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>
5 lines
218 B
Text
5 lines
218 B
Text
Set: pp::colors
|
||
Set: pp::unicode
|
||
Proved: T
|
||
Theorem T (a b : Bool) : a ∨ b ⇒ ¬ b ⇒ a :=
|
||
Discharge (λ H : a ∨ b, Discharge (λ H::1 : ¬ b, DisjCases H (λ H : a, H) (λ H : b, AbsurdElim a H H::1)))
|