aboutsummaryrefslogtreecommitdiff
path: root/pretyping/indrec.mli
diff options
context:
space:
mode:
Diffstat (limited to 'pretyping/indrec.mli')
-rw-r--r--pretyping/indrec.mli14
1 files changed, 7 insertions, 7 deletions
diff --git a/pretyping/indrec.mli b/pretyping/indrec.mli
index 7e6dd8fa1b..e28331848c 100644
--- a/pretyping/indrec.mli
+++ b/pretyping/indrec.mli
@@ -21,30 +21,30 @@ open Evd
(* These functions build elimination predicate for Case tactic *)
-val make_case_dep : env -> 'a evar_map -> inductive -> sorts_family -> constr
-val make_case_nodep : env -> 'a evar_map -> inductive -> sorts_family -> constr
-val make_case_gen : env -> 'a evar_map -> inductive -> sorts_family -> constr
+val make_case_dep : env -> evar_map -> inductive -> sorts_family -> constr
+val make_case_nodep : env -> evar_map -> inductive -> sorts_family -> constr
+val make_case_gen : env -> evar_map -> inductive -> sorts_family -> constr
(* This builds an elimination scheme associated (using the own arity
of the inductive) *)
-val build_indrec : env -> 'a evar_map -> inductive -> constr
+val build_indrec : env -> evar_map -> inductive -> constr
val instanciate_indrec_scheme : sorts -> int -> constr -> constr
(* This builds complex [Scheme] *)
val build_mutual_indrec :
- env -> 'a evar_map ->
+ env -> evar_map ->
(inductive * mutual_inductive_body * one_inductive_body
* bool * sorts_family) list
-> constr list
(* These are for old Case/Match typing *)
-val type_rec_branches : bool -> env -> 'c evar_map -> inductive_type
+val type_rec_branches : bool -> env -> evar_map -> inductive_type
-> unsafe_judgment -> constr -> constr array * constr
val make_rec_branch_arg :
- env -> 'a evar_map ->
+ env -> evar_map ->
int * ('b * constr) option array * int ->
constr -> constructor_summary -> recarg list -> constr