aboutsummaryrefslogtreecommitdiffhomepage
path: root/kernel/reduction.ml
diff options
context:
space:
mode:
authorGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-11-17 18:09:48 +0100
committerGravatar Hugo Herbelin <Hugo.Herbelin@inria.fr>2014-11-19 18:52:13 +0100
commit090fffa57b2235f70d4355f5dc85d73fa2634655 (patch)
treed07b76c4f97d2c1266563ccdb8f5ee1c86143054 /kernel/reduction.ml
parent51c8b16816ad0e9bdfaab0314fa6a0db5f4528f5 (diff)
Option -type-in-type continued (deactivate test for inferred sort of
inductive types + deactivate test for equality of sort + deactivate the check that the constraints Prop/Set <= Type are declared).
Diffstat (limited to 'kernel/reduction.ml')
-rw-r--r--kernel/reduction.ml5
1 files changed, 3 insertions, 2 deletions
diff --git a/kernel/reduction.ml b/kernel/reduction.ml
index 64964f85e..704b345bd 100644
--- a/kernel/reduction.ml
+++ b/kernel/reduction.ml
@@ -573,13 +573,14 @@ let check_sort_cmp_universes env pb s0 s1 univs =
end
| (Prop c1, Prop c2) -> if c1 != c2 then raise NotConvertible
| (Prop c1, Type u) ->
- let u0 = univ_of_sort s0 in
+ if not (type_in_type env) then
+ let u0 = univ_of_sort s0 in
(match pb with
| CUMUL -> check_leq univs u0 u
| CONV -> check_eq univs u0 u)
| (Type u, Prop c) -> raise NotConvertible
| (Type u1, Type u2) ->
- if not (type_in_type env) then
+ if not (type_in_type env) then
(match pb with
| CUMUL -> check_leq univs u1 u2
| CONV -> check_eq univs u1 u2)