We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
1 parent 0c52b45 commit 260dcb3Copy full SHA for 260dcb3
Mathlib/Order/Interval/Finset/Box.lean
@@ -85,7 +85,7 @@ end Prod
85
namespace Int
86
variable {x : ℤ × ℤ}
87
88
-attribute [norm_cast] toNat_ofNat
+attribute [norm_cast] toNat_natCast
89
90
lemma card_box : ∀ {n}, n ≠ 0 → #(box n : Finset (ℤ × ℤ)) = 8 * n
91
| n + 1, _ => by
0 commit comments