lean2/tests/lean/run/tactic20.lean

13 lines
172 B
Text
Raw Normal View History

import standard
using tactic
definition assump := eassumption
theorem tst {A : Type} {a b c : A} (H1 : a = b) (H2 : b = c) : a = c
:= by apply trans; assump; assump