lean2/tests/lean/run/refine2.lean

9 lines
157 B
Text
Raw Normal View History

import logic
example {A : Type} (f : A → A) (a b : A) : f a = b → f (f a) = f b :=
begin
intro fa_eq_b,
refine (congr_arg f _),
exact fa_eq_b
end