summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/3487.v
diff options
context:
space:
mode:
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 00000000..03c60a8b
--- /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).
+Definition baz1 := prod ((_ : baz) = (_ : baz)) (foo = foo).