d6692264e8
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
13 lines
355 B
Text
13 lines
355 B
Text
Set: pp::colors
|
|
Set: pp::unicode
|
|
Assumed: a
|
|
Assumed: b
|
|
Assumed: c
|
|
⊥
|
|
trans (and_congr
|
|
(refl (a = 1))
|
|
(λ C::1 : a = 1,
|
|
trans (and_congr (refl (b = 0)) (λ C::2 : b = 0, congr (congr2 Nat::gt C::2) C::1))
|
|
(and_falsel (b = 0))))
|
|
(and_falsel (a = 1))
|
|
(a = 1 ∧ b = 0 ∧ b > a) = ⊥
|