summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/7615.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/bugs/closed/7615.v')
-rw-r--r--test-suite/bugs/closed/7615.v19
1 files changed, 19 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/7615.v b/test-suite/bugs/closed/7615.v
new file mode 100644
index 00000000..cd8c4ad7
--- /dev/null
+++ b/test-suite/bugs/closed/7615.v
@@ -0,0 +1,19 @@
+Set Universe Polymorphism.
+
+Module Type S.
+Parameter Inline T@{i} : Type@{i+1}.
+End S.
+
+Module F (X : S).
+Definition X@{j i} : Type@{j} := X.T@{i}.
+End F.
+
+Module M.
+Definition T@{i} := Type@{i}.
+End M.
+
+Module N := F(M).
+
+Require Import Hurkens.
+
+Fail Definition eqU@{i j} : @eq Type@{j} N.X@{i Set} Type@{i} := eq_refl.