Skip to content

Commit 260dcb3

Browse files
committed
deprecation
1 parent 0c52b45 commit 260dcb3

File tree

1 file changed

+1
-1
lines changed

1 file changed

+1
-1
lines changed

Mathlib/Order/Interval/Finset/Box.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -85,7 +85,7 @@ end Prod
8585
namespace Int
8686
variable {x : ℤ × ℤ}
8787

88-
attribute [norm_cast] toNat_ofNat
88+
attribute [norm_cast] toNat_natCast
8989

9090
lemma card_box : ∀ {n}, n ≠ 0 → #(box n : Finset (ℤ × ℤ)) = 8 * n
9191
| n + 1, _ => by

0 commit comments

Comments
 (0)