aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-01-27 18:25:29 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-01-27 18:25:29 +0000
commitdf11643333c808596891d1c9ec4ba070934bb135 (patch)
treeda773debcdf0ef160ce4fd75d7b65d84c4327c31 /kernel
parent51dc457086fb5eee17c824f792363d327e15feab (diff)
make doc
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1286 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'kernel')
-rw-r--r--kernel/inductive.mli33
1 files changed, 16 insertions, 17 deletions
diff --git a/kernel/inductive.mli b/kernel/inductive.mli
index 547979fde..47d98e608 100644
--- a/kernel/inductive.mli
+++ b/kernel/inductive.mli
@@ -161,19 +161,18 @@ val find_rectype : env -> 'a evar_map -> constr -> inductive_type
from some inductive type already analysed as an [inductive_family];
global parameters are already instanciated in the constructor
types; the resulting summaries are valid in the environment where
- [indf] is valid the names of the products of the constructors types
+ [indf] is valid; the names of the products of the constructors types
are not renamed when [Anonymous] *)
val get_constructors : inductive_family -> constructor_summary array
val get_constructor : inductive_family -> int -> constructor_summary
-(* [get_arity inf] returns the product and the sort of the
- arity of the inductive family described by [is]; global parameters are
- already instanciated; [indf] must be defined w.r.t. [env] and [sigma];
- the products signature is relative to [env] and [sigma]; the names
- of the products of the constructors types are not renamed when
- [Anonymous] *)
+(* [get_arity indf] returns the product and the sort of the arity of
+ the inductive family described by [indf]; global parameters are
+ already instanciated; the products signature is relative to the
+ environment definition of [indf]; the names of the products of the
+ constructors types are not renamed when [Anonymous] *)
val get_arity : inductive_family -> arity
@@ -186,24 +185,24 @@ Inductive listn [A:Set] : nat -> Set :=
\end{verbatim}
has been defined. Then in some env containing ['x:nat'],
+\begin{quote}
+[find_rectype env sigma (listn bool (S x))] returns [IndType (indf, '(S x)')]
+\end{quote}
+where [indf = IndFamily ('listn',['bool'])].
-[find_inductive env sigma (listn bool (S x))] returns
-
-[is = {mind = 'listn'; params = 'bool'; realargs = '(S x)';
- nparams = 1; nrealargs = 1; nconstr = 2 }]
-
-then [get_constructors env sigma is] returns
-
+Then, [get_constructors indf] returns
+\begin{quote}
[[| { cs_cstr = 'niln'; cs_params = 'bool'; cs_nargs = 0;
cs_args = []; cs_concl_realargs = [|O|]};
{ cs_cstr = 'consn'; cs_params = 'bool'; cs_nargs = 3;
cs_args = [(Anonymous,'(listn A n)'),(Anonymous,'A'),(Name n,'nat')];
cs_concl_realargs = [|'(S n)'|]} |]]
-
-and [get_arity env sigma is] returns [[(Anonymous,'nat')],'Set'].
+\end{quote}
+and [get_arity indf] returns [[(Anonymous,'nat')],'Set'].
+\smallskip
*)
-(* Cases info *)
+(*s [Cases] info *)
val make_case_info : inductive_instance -> case_style option
-> pattern_source array -> case_info