180be5c4a2
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
17 lines
761 B
Text
17 lines
761 B
Text
Set: pp::colors
|
||
Set: pp::unicode
|
||
Assumed: a
|
||
Assumed: b
|
||
Assumed: c
|
||
a = 1 ∧ (¬ b = 0 ∨ c ≠ 0)
|
||
and_congr
|
||
(refl (a = 1))
|
||
(λ C::1 : a = 1,
|
||
trans (or_congr (or_congr (refl (¬ b = 0)) (λ C::2 : ¬ ¬ b = 0, congr2 (neq c) (not_not_elim C::2)))
|
||
(λ C::2 : ¬ (¬ b = 0 ∨ c ≠ 0),
|
||
congr (congr2 Nat::gt
|
||
(congr (congr2 Nat::add (not_not_elim (and_eliml (not_or_elim C::2))))
|
||
(not_neq_elim (and_elimr (not_or_elim C::2)))))
|
||
C::1))
|
||
(or_falsel (¬ b = 0 ∨ c ≠ 0)))
|
||
a = 1 ∧ ((¬ b = 0 ∨ c ≠ b) ∨ b + c > a) ↔ a = 1 ∧ (¬ b = 0 ∨ c ≠ 0)
|