aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/detyping.mli
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-01-13 00:25:21 +0530
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-01-13 00:29:09 +0530
commitc60f40ccecf526b5c7ce5adfe5908fdac3f66771 (patch)
treecb0eb77577f7de305043d081dbf8e7ecacc02149 /pretyping/detyping.mli
parentd797153f3e44279dd61804c3d2e75ec7892f38bf (diff)
Fix issue in printing due to de Bruijn bug when constructing compatibility
constr for primitive records (not used anywhere else than printing). Problem reported by P. LeFanu Lumsdaine on HoTT/HoTT. Also add some minor fixes in detyping and pretty printing related to universes.
Diffstat (limited to 'pretyping/detyping.mli')
-rw-r--r--pretyping/detyping.mli8
1 files changed, 4 insertions, 4 deletions
diff --git a/pretyping/detyping.mli b/pretyping/detyping.mli
index b9fdb5cbe..725fff5b2 100644
--- a/pretyping/detyping.mli
+++ b/pretyping/detyping.mli
@@ -36,12 +36,12 @@ val detype_names : bool -> Id.t list -> names_context -> env -> evar_map -> cons
val detype : ?lax:bool -> bool -> Id.t list -> env -> evar_map -> constr -> glob_constr
val detype_case :
- bool -> ('a -> glob_constr) ->
- (constructor array -> bool list array -> 'a array ->
+ bool -> (constr -> glob_constr) ->
+ (constructor array -> bool list array -> constr array ->
(Loc.t * Id.t list * cases_pattern list * glob_constr) list) ->
- ('a -> bool list -> bool) ->
+ (constr -> bool list -> bool) ->
Id.t list -> inductive * case_style * bool list array * bool list ->
- 'a option -> 'a -> 'a array -> glob_constr
+ constr option -> constr -> constr array -> glob_constr
val detype_sort : sorts -> glob_sort