summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/3336.v
blob: dc358c6004f89f5351a4267259a420eff198127b (plain)
1
2
3
4
5
6
7
8
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. *)