Zulip Chat Archive

Stream: PR reviews

Topic: !4#3320


Jeremy Tan (Apr 07 2023 at 04:16):

!4#3320 was created because of one of Eric's comments on !4#2450. I'd like a quick review so we can merge !4#2450 sooner

Kevin Buzzard (Apr 07 2023 at 04:27):

docs#fin.cast_succ_cast_lt

Jeremy Tan (Apr 07 2023 at 04:33):

@Kevin Buzzard in mathlib4 (currently):

@[simp]
theorem castSucc_cast_lt (i : Fin (n + 1)) (h : (i : ) < n) : castSucc (castLt i h) = i :=
  Fin.eq_of_veq rfl
#align fin.cast_succ_cast_lt Fin.castSucc_cast_lt

@[simp]
theorem cast_lt_castSucc {n : } (a : Fin n) (h : (a : ) < n) : castLt (castSucc a) h = a := by
  cases a; rfl
#align fin.cast_lt_cast_succ Fin.cast_lt_castSucc

Jeremy Tan (Apr 07 2023 at 04:34):

castLt is in the declaration, so castLt should be in the name too

Kevin Buzzard (Apr 07 2023 at 04:51):

Weekly reminder that I still have no understanding of the new naming convention

Kevin Buzzard (Apr 07 2023 at 04:51):

I thought "proof => mathlib3 style blah_blah_blah"

Mario Carneiro (Apr 07 2023 at 04:52):

I think it would be castSucc_castLt with that name

Kevin Buzzard (Apr 07 2023 at 04:52):

That's what the PR does

Mario Carneiro (Apr 07 2023 at 04:52):

although I think we're spelling it castLT and castLt is a mathportism

Kevin Buzzard (Apr 07 2023 at 04:53):

Kevin Buzzard said:

Weekly reminder that I still have no understanding of the new naming convention

Jeremy Tan (Apr 07 2023 at 04:53):

So should it be castLT everywhere?

Mario Carneiro (Apr 07 2023 at 04:53):

yeah

Kevin Buzzard (Apr 07 2023 at 04:54):

Is there anyone out there who can make a simple mathlib4 naming convention game? I'm serious.

Mario Carneiro (Apr 07 2023 at 04:56):

Mathlib.namingConvention_game

Jeremy Tan (Apr 07 2023 at 05:00):

@Mario Carneiro commit pushed


Last updated: Dec 20 2023 at 11:08 UTC