lean2/tests/lean/extra/rec3.lean

9 lines
229 B
Text
Raw Normal View History

set_option pp.implicit true
set_option pp.notation false
definition symm : Π {A : Type} {a b : A}, a = b → b = a,
symm rfl := rfl
definition trans : Π {A : Type} {a b c : A}, a = b → b = c → a = c,
trans rfl rfl := rfl