lean2/tests/lean/apply_tac1.lean
Leonardo de Moura 029ef57abd feat(library/tactic): add apply_tactic
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2013-12-05 03:22:12 -08:00

18 lines
No EOL
506 B
Text

Variable f : Int -> Int -> Bool
Variable P : Int -> Int -> Bool
Axiom Ax1 (x y : Int) (H : P x y) : (f x y)
Theorem T1 (a : Int) : (P a a) => (f a a).
apply imp_tactic
apply (** apply_tactic("Ax1") **)
apply assumption_tactic
done
Variable b : Int
Axiom Ax2 (x : Int) : (f x b)
(**
simple_tac = REPEAT(ORELSE(imp_tactic, assumption_tactic, apply_tactic("Ax2"), apply_tactic("Ax1")))
**)
Theorem T2 (a : Int) : (P a a) => (f a a).
apply simple_tac
done
Show Environment 1.