aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/evd.mli
diff options
context:
space:
mode:
Diffstat (limited to 'pretyping/evd.mli')
-rw-r--r--pretyping/evd.mli8
1 files changed, 4 insertions, 4 deletions
diff --git a/pretyping/evd.mli b/pretyping/evd.mli
index 3b58910e1..1393a33d3 100644
--- a/pretyping/evd.mli
+++ b/pretyping/evd.mli
@@ -117,6 +117,9 @@ val map_evar_info : (constr -> constr) -> evar_info -> evar_info
(** {6 Unification state} **)
+type evar_universe_context
+(** The universe context associated to an evar map *)
+
type evar_map
(** Type of unification state. Essentially a bunch of state-passing data needed
to handle incremental term construction. *)
@@ -128,7 +131,7 @@ val progress_evar_map : evar_map -> evar_map -> bool
val empty : evar_map
(** The empty evar map. *)
-val from_env : ?ctx:Univ.universe_context_set -> env -> evar_map
+val from_env : ?ctx:evar_universe_context -> env -> evar_map
(** The empty evar map with given universe context, taking its initial
universes from env. *)
@@ -408,9 +411,6 @@ val univ_rigid : rigid
val univ_flexible : rigid
val univ_flexible_alg : rigid
-(** The universe context associated to an evar map *)
-type evar_universe_context
-
type 'a in_evar_universe_context = 'a * evar_universe_context
val evar_universe_context_set : evar_universe_context -> Univ.universe_context_set