summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/3804.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/bugs/closed/3804.v')
-rw-r--r--test-suite/bugs/closed/3804.v12
1 files changed, 12 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3804.v b/test-suite/bugs/closed/3804.v
new file mode 100644
index 00000000..da9290cb
--- /dev/null
+++ b/test-suite/bugs/closed/3804.v
@@ -0,0 +1,12 @@
+Set Universe Polymorphism.
+Module Foo.
+ Definition T : sigT (fun x => x).
+ Proof.
+ exists Set.
+ abstract exact nat.
+ Defined.
+End Foo.
+Module Bar.
+ Include Foo.
+End Bar.
+Definition foo := eq_refl : Foo.T = Bar.T.