411ebbc3c1
This commit also adds several new theorems that are useful for implementing the simplifier. TODO: perhaps we should remove the declarations at basic_thms.h? Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
7 lines
220 B
Text
7 lines
220 B
Text
Set: pp::colors
|
||
Set: pp::unicode
|
||
Imported 'tactic'
|
||
Proved: T1
|
||
Proved: T2
|
||
Theorem T2 (a b : Bool) : a ∨ b ⇒ b ∨ a :=
|
||
Discharge (λ H : a ∨ b, DisjCases H (λ H : a, Disj2 b H) (λ H : b, Disj1 H a))
|