aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/opened
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-03-03 22:32:02 +0100
committerGravatar Matthieu Sozeau <matthieu.sozeau@inria.fr>2015-03-03 22:32:02 +0100
commitc1a330b28cd1417099183a1cb0a86b6a606b7ae9 (patch)
treed7d7cc78b9109f4295b1daf706f825e440666dec /test-suite/bugs/opened
parentf51efdd18b01c7f3fce026c32c0cd21ff4f6ca02 (diff)
Add missing test-suite files and update gitignore.
Diffstat (limited to 'test-suite/bugs/opened')
-rw-r--r--test-suite/bugs/opened/3794.v7
1 files changed, 7 insertions, 0 deletions
diff --git a/test-suite/bugs/opened/3794.v b/test-suite/bugs/opened/3794.v
new file mode 100644
index 000000000..511a92b2a
--- /dev/null
+++ b/test-suite/bugs/opened/3794.v
@@ -0,0 +1,7 @@
+Hint Extern 10 ((?X = ?Y) -> False) => intros; discriminate.
+Hint Unfold not : core.
+
+Goal true<>false.
+Set Typeclasses Debug.
+typeclasses eauto with core.
+Qed. \ No newline at end of file