aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/detyping.mli
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-01-17 20:17:17 +0530
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-01-18 00:16:44 +0530
commit237b569dd6539fc1730dbd1dda29f83e24ef8d0c (patch)
tree71c1eeaec02da28ae34f8428bab7ddcf7ecc251c /pretyping/detyping.mli
parent1c0110b40a9009aa6b56fafbf34a04e7ae59de0f (diff)
Univs: proper printing of global and local universe names (only
printing functions touched in the kernel).
Diffstat (limited to 'pretyping/detyping.mli')
-rw-r--r--pretyping/detyping.mli2
1 files changed, 1 insertions, 1 deletions
diff --git a/pretyping/detyping.mli b/pretyping/detyping.mli
index 725fff5b2..eb158686a 100644
--- a/pretyping/detyping.mli
+++ b/pretyping/detyping.mli
@@ -43,7 +43,7 @@ val detype_case :
Id.t list -> inductive * case_style * bool list array * bool list ->
constr option -> constr -> constr array -> glob_constr
-val detype_sort : sorts -> glob_sort
+val detype_sort : evar_map -> sorts -> glob_sort
val detype_rel_context : ?lax:bool -> constr option -> Id.t list -> (names_context * env) ->
evar_map -> rel_context -> glob_decl list