lean2/tests/lean/simp17.lean.expected.out

14 lines
416 B
Text
Raw Normal View History

Set: pp::colors
Set: pp::unicode
Assumed: a
Assumed: b
Assumed: c
trans (and_congrr
(λ C::1 : b = 0 ∧ c = 1,
congr (congr2 neq (congr1 0 (congr2 Nat::add (and_elimr C::1))))
(congr1 1 (congr2 Nat::add (and_eliml C::1))))
(λ C::7 : ⊥, refl (b = 0 ∧ c = 1)))
(and_falser (b = 0 ∧ c = 1))
(c + 0 ≠ b + 1 ∧ b = 0 ∧ c = 1) = ⊥