aboutsummaryrefslogtreecommitdiffhomepage
path: root/pretyping/cases.mli
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-05-18 08:14:28 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2000-05-18 08:14:28 +0000
commitaaa56145f319b58300ed7f914b35eb11321838e4 (patch)
treea24271d50a26991be09ab5bb1440289e7beaf8e5 /pretyping/cases.mli
parentb71bb95005c9a9db0393bcafc2d43383335c69bf (diff)
Effets de bords suite à la restructuration des inductives (cf Inductive)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@442 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'pretyping/cases.mli')
-rw-r--r--pretyping/cases.mli3
1 files changed, 2 insertions, 1 deletions
diff --git a/pretyping/cases.mli b/pretyping/cases.mli
index 3dbe65ff8..fbf77e402 100644
--- a/pretyping/cases.mli
+++ b/pretyping/cases.mli
@@ -6,6 +6,7 @@ open Names
open Term
open Evd
open Environ
+open Inductive
open Rawterm
open Evarutil
(*i*)
@@ -13,7 +14,7 @@ open Evarutil
(* Used for old cases in pretyping *)
val branch_scheme :
- env -> 'a evar_defs -> bool -> int -> inductive * constr list -> constr
+ env -> 'a evar_defs -> bool -> int -> inductive_family -> constr
(* Compilation of pattern-matching. *)