aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel/indtypes.ml
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2014-07-03 23:45:01 +0200
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2014-07-03 23:45:01 +0200
commit23d30ddc2a7cdfa3f71e99f57d36818b16ad40b7 (patch)
treebdd895f74d2764e4e57a1c4aab65ba4408442190 /kernel/indtypes.ml
parent7e4925b78162226331c65ef77f2da681a0b8ee48 (diff)
Cleanup code related to the constraint solving, which sits now outside the
kernel in library/universes.ml.
Diffstat (limited to 'kernel/indtypes.ml')
-rw-r--r--kernel/indtypes.ml1
1 files changed, 0 insertions, 1 deletions
diff --git a/kernel/indtypes.ml b/kernel/indtypes.ml
index cc56428fa..ee4a404a7 100644
--- a/kernel/indtypes.ml
+++ b/kernel/indtypes.ml
@@ -320,7 +320,6 @@ let typecheck_inductive env ctx mie =
in
match s with
| Type u when expltype (* Explicitly polymorphic *) ->
- (* && no_upper_constraints u (Univ.UContext.constraints mie.mind_entry_universes) -> *)
(* The polymorphic level is a function of the level of the *)
(* conclusions of the parameters *)
(* We enforce [u >= lev] in case [lev] has a strict upper *)