aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/closed/3336.v
diff options
context:
space:
mode:
authorGravatar Matthieu Sozeau <mattam@mattam.org>2014-06-20 16:03:52 +0200
committerGravatar Matthieu Sozeau <mattam@mattam.org>2014-06-20 16:03:52 +0200
commit6133a43c30e03656696a897bcedaf0cfb2cec70d (patch)
treeedda5b719763000d714a3eb097a15d6a8efccb64 /test-suite/bugs/closed/3336.v
parent45bcb4c7ad7aad8c2c63287870666339fe2ac1f2 (diff)
Allow more relaxed conversion between the types of the two terms of a rewrite
equation, fix uncaught exception in setoid_rewrite (bug #3336).
Diffstat (limited to 'test-suite/bugs/closed/3336.v')
-rw-r--r--test-suite/bugs/closed/3336.v9
1 files changed, 9 insertions, 0 deletions
diff --git a/test-suite/bugs/closed/3336.v b/test-suite/bugs/closed/3336.v
new file mode 100644
index 000000000..dc358c600
--- /dev/null
+++ b/test-suite/bugs/closed/3336.v
@@ -0,0 +1,9 @@
+Require Import Setoid.
+
+Goal forall x y : Type, x = y -> x = y.
+intros x y H.
+setoid_rewrite H.
+reflexivity.
+Defined.
+(* Toplevel input, characters 0-16:
+Anomaly: Uncaught exception Reduction.NotConvertible(_). Please report. *)