From 337800bee39698c888a5d32e6724efc1c12b3f3d Mon Sep 17 00:00:00 2001 From: Matthieu Sozeau Date: Fri, 21 Nov 2014 00:46:45 +0100 Subject: Add test-suite file for bug #3804. --- test-suite/bugs/closed/3804.v | 12 ++++++++++++ 1 file changed, 12 insertions(+) create mode 100644 test-suite/bugs/closed/3804.v (limited to 'test-suite/bugs/closed/3804.v') 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 -- cgit v1.2.3