lean2/tests/lean/simp17.lean.expected.out
Leonardo de Moura c56df132b8 refactor(kernel): remove semantic attachments from the kernel
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
2014-02-02 14:48:27 -08:00

14 lines
463 B
Text

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