aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>1999-11-30 12:06:00 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>1999-11-30 12:06:00 +0000
commit788402887777136c180a177ac41909b09727e159 (patch)
tree502b0d22865893747864e8111201353eff38dd6f /pretyping
parentc1d8ad80c5a877b2fae061b492af23e523d40ccf (diff)
ocamlweb
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@165 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'pretyping')
-rw-r--r--pretyping/coercion.mli5
-rw-r--r--pretyping/evarutil.mli11
-rw-r--r--pretyping/multcase.mli5
-rw-r--r--pretyping/pretype_errors.mli2
4 files changed, 17 insertions, 6 deletions
diff --git a/pretyping/coercion.mli b/pretyping/coercion.mli
index 2eeafa15b..3fc8dfb91 100644
--- a/pretyping/coercion.mli
+++ b/pretyping/coercion.mli
@@ -1,12 +1,15 @@
-(* $:Id$ *)
+(* $Id$ *)
+(*i*)
open Evd
open Term
open Sign
open Environ
open Evarutil
+(*i*)
+(* Coercions. *)
val inh_app_fun :
unsafe_env -> 'a evar_defs -> unsafe_judgment -> unsafe_judgment
diff --git a/pretyping/evarutil.mli b/pretyping/evarutil.mli
index c8d6b91ac..3cbf887c5 100644
--- a/pretyping/evarutil.mli
+++ b/pretyping/evarutil.mli
@@ -1,15 +1,18 @@
-(* This modules provides useful functions for unification algorithms.
- * Used in Trad and Progmach
- * This interface will have to be improved.
- *)
+(* $Id$ *)
+(*i*)
open Names
open Term
open Sign
open Evd
open Environ
open Reduction
+(*i*)
+
+(* This modules provides useful functions for unification algorithms.
+ * Used in Trad and Progmach
+ * This interface will have to be improved. *)
val filter_unique : 'a list -> 'a list
val distinct_id_list : identifier list -> identifier list
diff --git a/pretyping/multcase.mli b/pretyping/multcase.mli
index 7819915d9..68e68c1b4 100644
--- a/pretyping/multcase.mli
+++ b/pretyping/multcase.mli
@@ -1,14 +1,17 @@
(* $Id$ *)
+(*i*)
open Names
open Term
open Evd
open Environ
open Rawterm
open Evarutil
+(*i*)
+
+(* Compilation of pattern-matching. *)
-(* used by trad.ml *)
val compile_multcase :
(trad_constraint -> unsafe_env -> rawconstr -> unsafe_judgment)
* 'a evar_defs -> trad_constraint -> unsafe_env ->
diff --git a/pretyping/pretype_errors.mli b/pretyping/pretype_errors.mli
index ac605f196..4e37b18a7 100644
--- a/pretyping/pretype_errors.mli
+++ b/pretyping/pretype_errors.mli
@@ -1,6 +1,7 @@
(* $Id$ *)
+(*i*)
open Pp
open Names
open Term
@@ -8,6 +9,7 @@ open Sign
open Environ
open Type_errors
open Rawterm
+(*i*)
(* The type of errors raised by the pretyper *)