aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/3487.v
diff options
context:
space:
mode:
authorGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-11-30 02:36:19 +0100
committerGravatar Pierre-Marie Pédrot <pierre-marie.pedrot@inria.fr>2014-11-30 02:36:19 +0100
commit4586e904f8d2759c4f19e1ac3ad5c0447b353ae0 (patch)
treee62b817143d70bd18d5ec3f323f9754c1b9cece3 /test-suite/bugs/closed/3487.v
parent6566764abca36d661c5e403486458a326eeea4a4 (diff)
Test for bug #3487.
Diffstat (limited to 'test-suite/bugs/closed/3487.v')
-rw-r--r--test-suite/bugs/closed/3487.v8
1 files changed, 8 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3487.v b/test-suite/bugs/closed/3487.v
new file mode 100644
index 000000000..ba7a5c98f
--- /dev/null
+++ b/test-suite/bugs/closed/3487.v
@@ -0,0 +1,8 @@
+Notation bar := $(exact I)$.
+Notation foo := bar (only parsing).
+Class baz := { x : False }.
+Instance: baz.
+Admitted.
+Definition baz0 := ((_ : baz) = (_ : baz)).
+Definition foo1 := (foo = foo).
+Fail Definition baz1 := prod ((_ : baz) = (_ : baz)) (foo = foo).