aboutsummaryrefslogtreecommitdiff
path: root/kernel/term.mli
diff options
context:
space:
mode:
authorherbelin2001-09-19 16:55:41 +0000
committerherbelin2001-09-19 16:55:41 +0000
commitf83572bc45b9ab6b72688eb22d125896541ccf16 (patch)
tree37e08a39ea53751d9fdd7dff4449f4125e3f7bfd /kernel/term.mli
parent3607bb83605ff596445e0f18016d1fbb3d66d584 (diff)
Type 'sorts_family' (ex elimination_sorts) pour caractériser les familles des sortes (InProp, InSet, InType)
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2009 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'kernel/term.mli')
-rw-r--r--kernel/term.mli14
1 files changed, 11 insertions, 3 deletions
diff --git a/kernel/term.mli b/kernel/term.mli
index 76daa96f0a..ca0bae8385 100644
--- a/kernel/term.mli
+++ b/kernel/term.mli
@@ -27,6 +27,14 @@ val mk_Prop : sorts
val print_sort : sorts -> std_ppcmds
+(*s The sorts family of CCI. *)
+
+type sorts_family = InProp | InSet | InType
+
+val family_of_sort : sorts -> sorts_family
+val new_sort_in_family : sorts_family -> sorts
+
+(*s Useful types *)
type existential_key = int
@@ -38,7 +46,7 @@ type case_printing =
(* the integer is the number of real args, needed for reduction *)
type case_info = int * case_printing
-(* Concrete type for making pattern-matching. *)
+(*s Concrete type for making pattern-matching. *)
module Polymorph :
sig
(* [constr array] is an instance matching definitional [named_context] in
@@ -58,7 +66,7 @@ type ('constr, 'types) cofixpoint =
de Bruijn indices. *)
end
-(********************************************************************)
+(*s*******************************************************************)
(* type of global reference *)
type global_reference =
@@ -67,7 +75,7 @@ type global_reference =
| IndRef of inductive_path
| ConstructRef of constructor_path
-(********************************************************************)
+(*s*******************************************************************)
(* The type of constructions *)
type constr