lean2/tests/lean/tactic5.lean.expected.out
Leonardo de Moura f9874cd675 feat(library/tactic): add to_tactic_ext, it allows functions that return tactics to be used where a tactic is expected
For example, after this commit, we can write

simple_tac = REPEAT(ORELSE(imp_tactic, conj_tactic)) .. assumption_tactic

instead of

simple_tac = REPEAT(ORELSE(imp_tactic(), conj_tactic())) .. assumption_tactic()

Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2013-11-29 09:40:21 -08:00

5 lines
177 B
Text

Set: pp::colors
Set: pp::unicode
Proved: T4
Theorem T4 (a b : Bool) : a ⇒ b ⇒ a ∧ b ∧ a :=
Discharge (λ H : a, Discharge (λ H::1 : b, Conj H (Conj H::1 H)))