I would make this a pull request, but I'm not sure it's a real typo (and I have pull-request-rejection anxiety :)
Here is an example from Section 7.4:
theorem succ_add (m n : nat) : succ m + n = succ (m + n) :=
nat.rec_on n rfl (λ n ih, by simp only [succ_add, ih])
Is the use of succ_add in the simp tactic okay? Maybe it's only used to establish the induction hypothesis...? Or was the proof supposed to use add_succ? That is,
theorem succ_add (m n : nat) : succ m + n = succ (m + n) :=
nat.rec_on n rfl (λ n ih, by simp only [add_succ, ih])
I would make this a pull request, but I'm not sure it's a real typo (and I have pull-request-rejection anxiety :)
Here is an example from Section 7.4:
Is the use of
succ_add
in thesimp
tactic okay? Maybe it's only used to establish the induction hypothesis...? Or was the proof supposed to useadd_succ
? That is,