aboutsummaryrefslogtreecommitdiff
path: root/kernel
diff options
context:
space:
mode:
authorherbelin2001-09-20 16:31:09 +0000
committerherbelin2001-09-20 16:31:09 +0000
commit6aeea41c8a94233cb8b3ae15db1b20c75397610e (patch)
tree07446933f33ed70d3cf11020e9b4187efad3df6d /kernel
parent500e89caeb3cb614cf2d51a2765cc42d0e10fed0 (diff)
Nettoyage des commentaires
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@2031 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'kernel')
-rw-r--r--kernel/closure.mli12
-rw-r--r--kernel/univ.mli15
2 files changed, 1 insertions, 26 deletions
diff --git a/kernel/closure.mli b/kernel/closure.mli
index e755f28d98..b7ded4a9f9 100644
--- a/kernel/closure.mli
+++ b/kernel/closure.mli
@@ -32,18 +32,6 @@ type evaluable_global_reference =
Rem: reduction of a Rel/Var bound to a term is Delta, but reduction of
a LetIn expression is Letin reduction *)
-(*
-type red_kind =
- | BETA
- | DELTA
- | ZETA
- | EVAR
- | IOTA
- | CONST of section_path list
- | CONSTBUT of section_path list
- | VAR of identifier
- | VARBUT of identifier
-*)
(* Sets of reduction kinds. *)
module type RedFlagsSig = sig
type reds
diff --git a/kernel/univ.mli b/kernel/univ.mli
index e677b765ce..da66f4aed5 100644
--- a/kernel/univ.mli
+++ b/kernel/univ.mli
@@ -16,15 +16,9 @@ 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
@@ -38,11 +32,7 @@ val initial_universes : universes
(*s Constraints. *)
-(*
-type constraint_type = Gt | Geq | Eq
-*)
-
-type univ_constraint (* = universe * constraint_type * universe *)
+type univ_constraint
module Constraint : Set.S with type elt = univ_constraint
@@ -50,9 +40,6 @@ 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