aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/detyping.mli
diff options
context:
space:
mode:
Diffstat (limited to 'pretyping/detyping.mli')
-rw-r--r--pretyping/detyping.mli6
1 files changed, 3 insertions, 3 deletions
diff --git a/pretyping/detyping.mli b/pretyping/detyping.mli
index 72379dfcf..d1e0d1049 100644
--- a/pretyping/detyping.mli
+++ b/pretyping/detyping.mli
@@ -30,9 +30,9 @@ val subst_rawconstr : substitution -> rawconstr -> rawconstr
val detype : bool -> identifier list -> names_context -> constr -> rawconstr
-val detype_case :
+val detype_case :
bool -> ('a -> rawconstr) ->
- (constructor array -> int array -> 'a array ->
+ (constructor array -> int array -> 'a array ->
(loc * identifier list * cases_pattern list * rawconstr) list) ->
('a -> int -> bool) ->
identifier list -> inductive * case_style * int * int array * int ->
@@ -54,7 +54,7 @@ val synthetize_type : unit -> bool
(* Utilities to transform kernel cases to simple pattern-matching problem *)
val it_destRLambda_or_LetIn_names : int -> rawconstr -> name list * rawconstr
-val simple_cases_matrix_of_branches :
+val simple_cases_matrix_of_branches :
inductive -> int list -> rawconstr list -> cases_clauses
val return_type_of_predicate :
inductive -> int -> int -> rawconstr -> predicate_pattern * rawconstr option