aboutsummaryrefslogtreecommitdiff
path: root/kernel/inductive.mli
diff options
context:
space:
mode:
authorfilliatr1999-08-30 07:27:52 +0000
committerfilliatr1999-08-30 07:27:52 +0000
commit19d21ec59b69a7bd5a8e4e77794e85fed6b48d39 (patch)
tree4d6a784866d8b8da5a8c4378b3ce3fdf9d159186 /kernel/inductive.mli
parent72681a66688b1b81309582cfaf979a7096a118c2 (diff)
un petit effort de presentation dans les interfaces
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@31 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'kernel/inductive.mli')
-rw-r--r--kernel/inductive.mli15
1 files changed, 14 insertions, 1 deletions
diff --git a/kernel/inductive.mli b/kernel/inductive.mli
index c60c3cf4e8..a08136424a 100644
--- a/kernel/inductive.mli
+++ b/kernel/inductive.mli
@@ -1,9 +1,11 @@
(* $Id$ *)
+(*i*)
open Names
open Term
open Sign
+(*i*)
(* Inductive types (internal representation). *)
@@ -74,10 +76,21 @@ type inductive_error =
exception InductiveError of inductive_error
+(* [mind_check_names] checks the names of an inductive types declaration
+ i.e. that all the types and constructors names are distinct.
+ It raises an exception [InductiveError _] if it is not the case. *)
+
val mind_check_names : mutual_inductive_entry -> unit
-val mind_extract_params : int -> constr -> (name * constr) list * constr
+(* [mind_extract_and_check_params] extracts the parameters of an inductive
+ types declaration. It raises an exception [InductiveError _] if there is
+ not enough abstractions in any of the terms of the field
+ [mind_entry_inds]. *)
+
val mind_extract_and_check_params :
mutual_inductive_entry -> (name * constr) list
+val mind_extract_params : int -> constr -> (name * constr) list * constr
+
+
val mind_check_lc : (name * constr) list -> mutual_inductive_entry -> unit