aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/opened/3336.v
diff options
context:
space:
mode:
Diffstat (limited to 'test-suite/bugs/opened/3336.v')
-rw-r--r--test-suite/bugs/opened/3336.v6
1 files changed, 6 insertions, 0 deletions
diff --git a/test-suite/bugs/opened/3336.v b/test-suite/bugs/opened/3336.v
new file mode 100644
index 000000000..d469a13a3
--- /dev/null
+++ b/test-suite/bugs/opened/3336.v
@@ -0,0 +1,6 @@
+Require Import Setoid.
+Goal forall x y : Type, x = y -> x = y.
+intros x y H.
+Fail setoid_rewrite H.
+(* Toplevel input, characters 0-16:
+Anomaly: Uncaught exception Reduction.NotConvertible(_). Please report. *)