lean2/tests/lean/tactic14.lean.expected.out

6 lines
186 B
Text
Raw Normal View History

Set: pp::colors
Set: pp::unicode
Proved: T1
Theorem T1 (a b : ) (f : ) (assumption : a = b) : (f (f a)) = (f (f b)) :=
Congr (Refl f) (Congr (Refl f) assumption)