summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/3337.v
blob: cd7891f11241a4fb20c7f2558306a1633e72eb4e (plain)
1
2
3
4
Require Import Setoid.
Goal forall x y : Set, x = y -> x = y.
intros x y H.
rewrite_strat subterms H.