f9874cd675
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>
5 lines
177 B
Text
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)))
|