aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel/typeops.mli
diff options
context:
space:
mode:
authorGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>1999-10-18 13:51:32 +0000
committerGravatar filliatr <filliatr@85f007b7-540e-0410-9357-904b9bb8a0f7>1999-10-18 13:51:32 +0000
commit154f0fc69c79383cc75795554eb7e0256c8299d8 (patch)
treed39ed1dbe4d0c555a8373592162eee3043583a1a /kernel/typeops.mli
parent22e4ceb13d18c8b941f6a27cc83f547dd90104b8 (diff)
- déplacement (encore une fois !) des variables existentielles : elles sont
toujours dans le noyau (en ce sens que Reduction et Typeops les connaissent) mais dans un argument supplémentaire A COTE de l'environnement (de type unsafe_env) - Indtypes et Typing n'utilisent strictement que Evd.empty git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@106 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'kernel/typeops.mli')
-rw-r--r--kernel/typeops.mli35
1 files changed, 20 insertions, 15 deletions
diff --git a/kernel/typeops.mli b/kernel/typeops.mli
index 0a4419a60..f87601299 100644
--- a/kernel/typeops.mli
+++ b/kernel/typeops.mli
@@ -5,6 +5,7 @@
open Names
open Univ
open Term
+open Evd
open Environ
(*i*)
@@ -19,22 +20,25 @@ val j_val_only : unsafe_judgment -> constr
constructs the typed type $t:s$, while [assumption_of_judgement env j]
cosntructs the type type $c:t$, checking that $t$ is a sort. *)
-val typed_type_of_judgment : unsafe_env -> unsafe_judgment -> typed_type
-val assumption_of_judgment : unsafe_env -> unsafe_judgment -> typed_type
+val typed_type_of_judgment :
+ unsafe_env -> 'a evar_map -> unsafe_judgment -> typed_type
+val assumption_of_judgment :
+ unsafe_env -> 'a evar_map -> unsafe_judgment -> typed_type
val relative : unsafe_env -> int -> unsafe_judgment
-val type_of_constant : unsafe_env -> constr -> typed_type
+val type_of_constant : unsafe_env -> 'a evar_map -> constr -> typed_type
-val type_of_inductive : unsafe_env -> constr -> typed_type
+val type_of_inductive : unsafe_env -> 'a evar_map -> constr -> typed_type
-val type_of_constructor : unsafe_env -> constr -> constr
+val type_of_constructor : unsafe_env -> 'a evar_map -> constr -> constr
-val type_of_case : unsafe_env -> unsafe_judgment -> unsafe_judgment
- -> unsafe_judgment array -> unsafe_judgment
+val type_of_case : unsafe_env -> 'a evar_map
+ -> unsafe_judgment -> unsafe_judgment
+ -> unsafe_judgment array -> unsafe_judgment
val type_case_branches :
- unsafe_env -> constr -> constr -> constr -> constr
+ unsafe_env -> 'a evar_map -> constr -> constr -> constr -> constr
-> constr * constr array * constr
val type_of_prop_or_set : contents -> unsafe_judgment
@@ -42,22 +46,23 @@ val type_of_prop_or_set : contents -> unsafe_judgment
val type_of_type : universe -> unsafe_judgment * constraints
val abs_rel :
- unsafe_env -> name -> typed_type -> unsafe_judgment
+ unsafe_env -> 'a evar_map -> name -> typed_type -> unsafe_judgment
-> unsafe_judgment * constraints
val gen_rel :
- unsafe_env -> name -> typed_type -> unsafe_judgment
+ unsafe_env -> 'a evar_map -> name -> typed_type -> unsafe_judgment
-> unsafe_judgment * constraints
val cast_rel :
- unsafe_env -> unsafe_judgment -> unsafe_judgment -> unsafe_judgment
+ unsafe_env -> 'a evar_map -> unsafe_judgment -> unsafe_judgment
+ -> unsafe_judgment
val apply_rel_list :
- unsafe_env -> bool -> unsafe_judgment list -> unsafe_judgment
+ unsafe_env -> 'a evar_map -> bool -> unsafe_judgment list -> unsafe_judgment
-> unsafe_judgment * constraints
-val check_fix : unsafe_env -> Spset.t -> constr -> unit
-val check_cofix : unsafe_env -> Spset.t -> constr -> unit
+val check_fix : unsafe_env -> 'a evar_map -> Spset.t -> constr -> unit
+val check_cofix : unsafe_env -> 'a evar_map -> Spset.t -> constr -> unit
-val type_fixpoint : unsafe_env -> name list -> typed_type array
+val type_fixpoint : unsafe_env -> 'a evar_map -> name list -> typed_type array
-> unsafe_judgment array -> constraints