aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/failure
diff options
context:
space:
mode:
authorGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-04-22 11:11:46 +0000
committerGravatar barras <barras@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-04-22 11:11:46 +0000
commit9ac005d89776bf74e78875128f04620c40a9408b (patch)
tree4d9b3f5d9ee60a19cea42f09d09c984a40b791ac /test-suite/failure
parenta3540551dc3f889b0b0a76d61fc02ec87f6dfd49 (diff)
fixed universes bug related to module inclusion
git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@10828 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/failure')
-rw-r--r--test-suite/failure/univ_include.v7
1 files changed, 4 insertions, 3 deletions
diff --git a/test-suite/failure/univ_include.v b/test-suite/failure/univ_include.v
index fd17457f0..4be70d888 100644
--- a/test-suite/failure/univ_include.v
+++ b/test-suite/failure/univ_include.v
@@ -17,13 +17,14 @@ Module G (E : MU).
Include F E.
Print Universes. (* U <= T *)
End G.
-Print Universes. (* constraint lost! *)
+Print Universes. (* Check if constraint is lost *)
Module Mt.
- Definition t :=T.
+ Definition t := T.
End Mt.
-Module P := G Mt.
+Module P := G Mt. (* should yield Universe inconsistency *)
+(* ... otherwise the following command will show that T has type T! *)
Eval cbv delta [P.elt Mt.t] in P.elt.