aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs
diff options
context:
space:
mode:
authorGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-07-25 13:16:32 +0000
committerGravatar msozeau <msozeau@85f007b7-540e-0410-9357-904b9bb8a0f7>2008-07-25 13:16:32 +0000
commit26d532da9063cdac9c693ebed29551662158bbb3 (patch)
tree519ce11d54168e091dc5f48f5b130d4132f87402 /test-suite/bugs
parentbe9c3dc93413a76d188724d4a06739d9bb238b72 (diff)
A better test for relations being setoids or not: do leibniz rewrite iff
the applied relation is an abbreviation for @eq. Fixes bug #1915. git-svn-id: svn+ssh://scm.gforge.inria.fr/svn/coq/trunk@11264 85f007b7-540e-0410-9357-904b9bb8a0f7
Diffstat (limited to 'test-suite/bugs')
-rw-r--r--test-suite/bugs/closed/shouldfail/1915.v6
1 files changed, 6 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/shouldfail/1915.v b/test-suite/bugs/closed/shouldfail/1915.v
new file mode 100644
index 000000000..a96a482c6
--- /dev/null
+++ b/test-suite/bugs/closed/shouldfail/1915.v
@@ -0,0 +1,6 @@
+
+Require Import Setoid.
+
+Goal forall x, impl True (x = 0) -> x = 0 -> False.
+intros x H E.
+rewrite H in E. \ No newline at end of file