lean2/tests/lean/run/tactic4.lean
Leonardo de Moura b2b76b078f feat(frontends/lean): remove build_tactic_cmds, and use expressions for representing tactics
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-07-01 20:43:53 -07:00

11 lines
212 B
Text

import standard
definition id {A : Type} (a : A) := a
definition simple_tac {A : Bool} : tactic A
:= unfold_tac @id.{1}; exact_tac
theorem tst {A B : Bool} (H1 : A) (H2 : B) : id A
:= by simple_tac
check tst