aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/3804.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2014-11-21 00:46:45 +0100
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2014-11-21 00:46:45 +0100
commit337800bee39698c888a5d32e6724efc1c12b3f3d (patch)
tree9fb060ada6715d22c3cae298fc82a81941184bd9 /test-suite/bugs/closed/3804.v
parent00d32afd7c6b270bab55671d7a5aeff125a1ca29 (diff)
Add test-suite file for bug #3804.
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 000000000..5dc0f7264
--- /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. (* Error: Conversion test raised an anomaly *) \ No newline at end of file