aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/typing.mli
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-02-15 13:31:54 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2016-02-15 13:41:16 +0100
commit1a8c37ca352c95b4cd530efbbf47f0e7671d1fb3 (patch)
tree15aadd829fe3e8c3ee0a747de34a9b96614bfdba /pretyping/typing.mli
parent968dfdb15cc11d48783017b2a91147b25c854ad6 (diff)
Renaming functions in Typing to stick to the standard e_* scheme.
Diffstat (limited to 'pretyping/typing.mli')
-rw-r--r--pretyping/typing.mli6
1 files changed, 3 insertions, 3 deletions
diff --git a/pretyping/typing.mli b/pretyping/typing.mli
index dafd75231..e524edcca 100644
--- a/pretyping/typing.mli
+++ b/pretyping/typing.mli
@@ -24,16 +24,16 @@ val type_of : ?refresh:bool -> env -> evar_map -> constr -> evar_map * types
val e_type_of : ?refresh:bool -> env -> evar_map ref -> constr -> types
(** Typecheck a type and return its sort *)
-val sort_of : env -> evar_map ref -> types -> sorts
+val e_sort_of : env -> evar_map ref -> types -> sorts
(** Typecheck a term has a given type (assuming the type is OK) *)
-val check : env -> evar_map ref -> constr -> types -> unit
+val e_check : env -> evar_map ref -> constr -> types -> unit
(** Returns the instantiated type of a metavariable *)
val meta_type : evar_map -> metavariable -> types
(** Solve existential variables using typing *)
-val solve_evars : env -> evar_map ref -> constr -> constr
+val e_solve_evars : env -> evar_map ref -> constr -> constr
(** Raise an error message if incorrect elimination for this inductive *)
(** (first constr is term to match, second is return predicate) *)