summaryrefslogtreecommitdiff
path: root/test-suite/bugs/closed/3338.v
blob: 076cd5e6ea9bfb680597ddf43dcac341844694f5 (plain)
1
2
3
4
Require Import Setoid.
Goal forall x y : Set, x = y -> y = y.
intros x y H.
rewrite_strat try topdown terms H.