lean2/tests/lean/run/tactic4.lean
Leonardo de Moura 7593ee1468 refactor(library/standard): remove parameter from 'tactic' inductive type
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-07-02 08:09:24 -07:00

11 lines
210 B
Text

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