lean2/tests/lean/tactic6.lean
Leonardo de Moura 0c059a9917 feat(library/tactic): use _tac suffix instead of _tactic like Isabelle
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2013-12-05 20:06:32 -08:00

21 lines
No EOL
601 B
Text

Theorem T (a b c : Bool): a => b /\ c => c /\ a /\ b := _.
apply imp_tac
apply imp_tac
apply conj_hyp_tac
apply conj_tac
apply (** FOCUS(THEN(show_tac, conj_tac, show_tac, assumption_tac), 2) **)
apply assumption_tac
done
Theorem T2 (a b c : Bool): a => b /\ c => c /\ a /\ b := _.
apply imp_tac
apply imp_tac
apply conj_hyp_tac
apply conj_tac
apply show_tac
apply (** FOCUS(THEN(show_tac, conj_tac, FOCUS(assumption_tac, 1)), 2) **)
apply show_tac
apply (** FOCUS(assumption_tac, 1) **)
apply show_tac
apply (** FOCUS(assumption_tac, 1) **)
done