Skip to content

Commit f904bf8

Browse files
committed
chore: Better names for (⌊a⌋₊ : α) = ⌊a⌋ again (#16001)
Also remove the six months old deprecated names
1 parent 431ff4c commit f904bf8

File tree

1 file changed

+6
-12
lines changed

1 file changed

+6
-12
lines changed

Mathlib/Algebra/Order/Floor.lean

Lines changed: 6 additions & 12 deletions
Original file line numberDiff line numberDiff line change
@@ -1492,26 +1492,20 @@ theorem Nat.ceil_int : (Nat.ceil : ℤ → ℕ) = Int.toNat :=
14921492

14931493
variable {a : α}
14941494

1495-
theorem Int.ofNat_floor_eq_floor (ha : 0 ≤ a) : (⌊a⌋₊ : ℤ) = ⌊a⌋ := by
1495+
theorem Int.natCast_floor_eq_floor (ha : 0 ≤ a) : (⌊a⌋₊ : ℤ) = ⌊a⌋ := by
14961496
rw [← Int.floor_toNat, Int.toNat_of_nonneg (Int.floor_nonneg.2 ha)]
14971497

1498-
theorem Int.ofNat_ceil_eq_ceil (ha : 0 ≤ a) : (⌈a⌉₊ : ℤ) = ⌈a⌉ := by
1498+
theorem Int.natCast_ceil_eq_ceil (ha : 0 ≤ a) : (⌈a⌉₊ : ℤ) = ⌈a⌉ := by
14991499
rw [← Int.ceil_toNat, Int.toNat_of_nonneg (Int.ceil_nonneg ha)]
15001500

15011501
theorem natCast_floor_eq_intCast_floor (ha : 0 ≤ a) : (⌊a⌋₊ : α) = ⌊a⌋ := by
1502-
rw [← Int.ofNat_floor_eq_floor ha, Int.cast_natCast]
1502+
rw [← Int.natCast_floor_eq_floor ha, Int.cast_natCast]
15031503

15041504
theorem natCast_ceil_eq_intCast_ceil (ha : 0 ≤ a) : (⌈a⌉₊ : α) = ⌈a⌉ := by
1505-
rw [← Int.ofNat_ceil_eq_ceil ha, Int.cast_natCast]
1505+
rw [← Int.natCast_ceil_eq_ceil ha, Int.cast_natCast]
15061506

1507-
@[deprecated (since := "2024-02-14")] alias Nat.cast_floor_eq_int_floor := Int.ofNat_floor_eq_floor
1508-
@[deprecated (since := "2024-02-14")] alias Nat.cast_ceil_eq_int_ceil := Int.ofNat_ceil_eq_ceil
1509-
1510-
@[deprecated (since := "2024-02-14")]
1511-
alias Nat.cast_floor_eq_cast_int_floor := natCast_floor_eq_intCast_floor
1512-
1513-
@[deprecated (since := "2024-02-14")]
1514-
alias Nat.cast_ceil_eq_cast_int_ceil := natCast_ceil_eq_intCast_ceil
1507+
@[deprecated (since := "2024-08-20")] alias Int.ofNat_floor_eq_floor := natCast_floor_eq_floor
1508+
@[deprecated (since := "2024-08-20")] alias Int.ofNat_ceil_eq_ceil := natCast_ceil_eq_ceil
15151509

15161510
end FloorRingToSemiring
15171511

0 commit comments

Comments
 (0)