aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel/univ.mli
diff options
context:
space:
mode:
authorGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-09-09 15:39:40 +0000
committerGravatar herbelin <herbelin@85f007b7-540e-0410-9357-904b9bb8a0f7>2001-09-09 15:39:40 +0000
commit382e4f6bb67bec64ea4a0ead5e9de232858a891e (patch)
tree99f79d0e8fa93366acb90788443aad2b0bc25043 /kernel/univ.mli
parent106d1c36ced53924f9dd3965e40536b2d1d3fb31 (diff)
Passage aux univers algébriques
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@1940 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'kernel/univ.mli')
-rw-r--r--kernel/univ.mli10
1 files changed, 9 insertions, 1 deletions
diff --git a/kernel/univ.mli b/kernel/univ.mli
index 0c405084d..e677b765c 100644
--- a/kernel/univ.mli
+++ b/kernel/univ.mli
@@ -16,11 +16,15 @@ open Names
type universe
+(*
val dummy_univ : universe
+*)
val implicit_univ : universe
val prop_univ : universe
+(*
val prop_univ_univ : universe
+*)
val set_module : dir_path -> unit
@@ -34,9 +38,11 @@ val initial_universes : universes
(*s Constraints. *)
+(*
type constraint_type = Gt | Geq | Eq
+*)
-type univ_constraint = universe * constraint_type * universe
+type univ_constraint (* = universe * constraint_type * universe *)
module Constraint : Set.S with type elt = univ_constraint
@@ -44,7 +50,9 @@ type constraints = Constraint.t
type constraint_function = universe -> universe -> constraints -> constraints
+(*
val enforce_gt : constraint_function
+*)
val enforce_geq : constraint_function
val enforce_eq : constraint_function