Zulip Chat Archive

Stream: general

Topic: No refl?


Joseph O (Apr 22 2022 at 01:36):

How come in this proof i dont need refl. I had to write it in the Natural Number Game.

lemma add_succ_zero (a : nat) : a + succ(0) = succ(a) :=
begin
  rw add_succ,
  rw add_zero,
end

when i write refl, at the end, it tells me

tactic failed, there are no goals to be solved
state:
no goals

is it implicit now?

Julian Berman (Apr 22 2022 at 01:40):

The nng uses a simplified rw, essentially to make it a bit less confusing to learn

Julian Berman (Apr 22 2022 at 01:40):

But yes the real rw will basically automatically run refl after rewriting

Joseph O (Apr 22 2022 at 01:48):

Julian Berman said:

The nng uses a simplified rw, essentially to make it a bit less confusing to learn

what is the nng?

Joseph O (Apr 22 2022 at 01:48):

how can i use the real rw?

Alex J. Best (Apr 22 2022 at 01:49):

Nng= natural number game, outside of the game rw is the real rewrite and you don't need to do anything special to use it

Joseph O (Apr 22 2022 at 01:50):

oh right

Joseph O (Apr 22 2022 at 01:54):

like im surprised with real rw succ_eq_add_one is

lemma succ_eq_add_one (n : nat) : succ n = n + 1 :=
begin
  rw one_eq_succ_zero,
end

but with nng its

lemma succ_eq_add_one (n : nat) : succ n = n + 1 :=
begin
  rw one_eq_succ_zero,
  rw add_succ,
  rw add_zero,
  refl,
end

Alex J. Best (Apr 22 2022 at 02:47):

What happens if you try the first one in nng, just followed by refl?

Alex J. Best (Apr 22 2022 at 02:47):

Does it work then? If add_succ and add_zero are proved by refl in the first place then it should be basically the same to do that

Joseph O (Apr 22 2022 at 12:28):

Alex J. Best said:

Does it work then? If add_succ and add_zero are proved by refl in the first place then it should be basically the same to do that

it doesn't prove it without them. It also seems like nng's rwa is analogous to the real rw.


Last updated: Dec 20 2023 at 11:08 UTC