aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/indrec.mli
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-12 14:41:39 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2003-09-12 14:41:39 +0000
commit53d23f52cd28c1373e784c278c8455cf9fa4eb67 (patch)
treefa4a9d60f052df1f400af1589e568ef0ed11ef45 /pretyping/indrec.mli
parent893231ce35ba826efe64e4601ae0af32f97ba575 (diff)
Déplacement de Declare juste à la fin de interp pour pouvoir accéder à interp
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@4365 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'pretyping/indrec.mli')
-rw-r--r--pretyping/indrec.mli3
1 files changed, 2 insertions, 1 deletions
diff --git a/pretyping/indrec.mli b/pretyping/indrec.mli
index 38d07d1d9..1ab429dcf 100644
--- a/pretyping/indrec.mli
+++ b/pretyping/indrec.mli
@@ -30,6 +30,8 @@ val make_case_gen : env -> evar_map -> inductive -> sorts_family -> constr
val build_indrec : env -> evar_map -> inductive -> constr
val instanciate_indrec_scheme : sorts -> int -> constr -> constr
+val instanciate_type_indrec_scheme : sorts -> int -> constr -> types ->
+ constr * types
(* This builds complex [Scheme] *)
@@ -49,7 +51,6 @@ val make_rec_branch_arg :
constr -> constructor_summary -> wf_paths list -> constr
(* *)
-val declare_eliminations : mutual_inductive -> unit
val lookup_eliminator : inductive -> sorts_family -> constr
val elimination_suffix : sorts_family -> string
val make_elimination_ident : identifier -> sorts_family -> identifier