Zulip Chat Archive

Stream: new members

Topic: Unknown identifier in NNG Multiplication World 3/9


R Dong (Oct 21 2024 at 16:22):

I'm trying to figure out why I can't proceed with the proof:

induction b with b' h
repeat rw [mul_zero]
rw [add_zero]
rfl
repeat rw [mul_succ]
nth_rewrite 2 [succ_eq_add_one a]
rw [succ_eq_add_one b']
repeat rw [ add_assoc]

Lean says add_right_cancel is unknown. However, I can see that it's available (and not locked) from the panel to the right. Am I misunderstanding what theorems are available?

R Dong (Oct 21 2024 at 16:36):

It seems like I can't apply any theorem

R Dong (Oct 21 2024 at 16:37):

I solved it with only rewrite rules, but I feel like that's not the best way to do it...

Etienne Marion (Oct 21 2024 at 18:07):

I don't know why add_right_cancel is unknown, but here it won't help you anyway because what you want to prove is in the other direction

R Dong (Oct 21 2024 at 18:11):

image.png
Is this not exactly add_right_cancel?

R Dong (Oct 21 2024 at 18:13):

Isn't (a b n : ℕ) (a✝ : a + n = b + n) : a = b directly applicable?

R Dong (Oct 21 2024 at 18:15):

Ok, I see what you mean

Etienne Marion (Oct 21 2024 at 18:31):

Personally on this level I went for a full rw proof too

R Dong (Oct 21 2024 at 18:36):

I explored a different path where I tried to apply succ_inj and that one is unknown too

Etienne Marion (Oct 21 2024 at 19:15):

I think this is because these lemmas are introduced in worlds parallel to multiplication world and so are considered unknown even if you completed those worlds before

R Dong (Oct 21 2024 at 19:17):

But they are not locked/grayed out in the panel. I can also use all the other rewrite rules

Etienne Marion (Oct 21 2024 at 21:07):

You can't use all the rewrites

R Dong (Oct 21 2024 at 21:31):

Ok, I didn't try all the rewrite rules

Martin Dvořák (Oct 23 2024 at 17:35):

Maybe it is related to the bug:
#general > Bug in NNG?


Last updated: May 02 2025 at 03:31 UTC