aboutsummaryrefslogtreecommitdiffhomepage
path: root/test-suite/bugs/opened/3336.v
blob: d469a13a3418efc231de1d1a14fa7ae1803bb792 (plain)
1
2
3
4
5
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. *)