aboutsummaryrefslogtreecommitdiffhomepage
path: root/engine/eConstr.mli
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-11-30 15:06:42 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2017-02-14 17:30:44 +0100
commit4f66c854956bd05a24fd55c3d52fb669dbbb65e6 (patch)
treed0c34b7e8cab383e8c6869d8026d4a6a41a50d2d /engine/eConstr.mli
parentbe51c33a6bf91a00fdd5f3638ddb5b3cc3a2c626 (diff)
Moving evar-normalization functions to EConstr.
This removes code duplication between Evarutil and EConstr.
Diffstat (limited to 'engine/eConstr.mli')
-rw-r--r--engine/eConstr.mli3
1 files changed, 3 insertions, 0 deletions
diff --git a/engine/eConstr.mli b/engine/eConstr.mli
index 83536d6f8..7992c0633 100644
--- a/engine/eConstr.mli
+++ b/engine/eConstr.mli
@@ -34,6 +34,8 @@ val kind : Evd.evar_map -> t -> (t, t) Constr.kind_of_term
(** Same as {!Constr.kind} except that it expands evars and normalizes
universes on the fly. *)
+val kind_upto : Evd.evar_map -> Constr.t -> (Constr.t, Constr.t) Constr.kind_of_term
+
val to_constr : Evd.evar_map -> t -> Constr.t
(** Returns the evar-normal form of the argument. See {!Evarutil.nf_evar}. *)
@@ -146,6 +148,7 @@ val decompose_prod_assum : Evd.evar_map -> t -> rel_context * t
val decompose_prod_n_assum : Evd.evar_map -> int -> t -> rel_context * t
val existential_type : Evd.evar_map -> existential -> types
+val whd_evar : Evd.evar_map -> constr -> constr
(** {6 Equality} *)