Zulip Chat Archive
Stream: lean4
Topic: Quesiton on equality and omega
Emmanuel Anaya Gonzalez (Sep 04 2024 at 06:07):
Why does the following snippet works, whereas using the commented line fails?
theorem lemma_small
(a b : Nat)
-- (sum : a + b == 2)
(sum : a + b = 2)
: (a = 0 ∧ b = 2) ∨ (a = 1 ∧ b = 1) ∨ (a = 2 ∧ b = 0)
:= by omega
Kim Morrison (Sep 04 2024 at 06:12):
omega
knows nothing about ==
.
Kim Morrison (Sep 04 2024 at 06:12):
by simp_all; omega
works.
Emmanuel Anaya Gonzalez (Sep 04 2024 at 06:14):
you are right! thanks :)
Last updated: May 02 2025 at 03:31 UTC