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 b1d3f2c commit 47a6fc5Copy full SHA for 47a6fc5
Mathlib/Algebra/GroupPower/Lemmas.lean
@@ -733,7 +733,7 @@ end LinearOrderedRing
733
734
namespace Int
735
736
-lemma natAbs_sq (x : ℤ) : ↑(x.natAbs ^ 2) = x ^ 2 := by rw [sq, Int.natAbs_mul_self, sq]
+lemma natAbs_sq (x : ℤ) : (x.natAbs : ℤ) ^ 2 = x ^ 2 := by rw [sq, Int.natAbs_mul_self', sq]
737
#align int.nat_abs_sq Int.natAbs_sq
738
739
alias natAbs_sq ← natAbs_pow_two
0 commit comments