Skip to content

Commit dacfbcb

Browse files
chore: fix statement of PNat.pow_coe (#4298)
1 parent 9b45a6f commit dacfbcb

File tree

1 file changed

+3
-6
lines changed

1 file changed

+3
-6
lines changed

Mathlib/Data/PNat/Basic.lean

Lines changed: 3 additions & 6 deletions
Original file line numberDiff line numberDiff line change
@@ -23,6 +23,8 @@ It is defined in `Data.PNat.Defs`, but most of the development is deferred to he
2323
that `Data.PNat.Defs` can have very few imports.
2424
-/
2525

26+
local macro_rules | `($x ^ $y) => `(HPow.hPow $x $y) -- Porting note: See issue #2220
27+
2628
deriving instance AddLeftCancelSemigroup, AddRightCancelSemigroup, AddCommSemigroup,
2729
LinearOrderedCancelCommMonoid, Add, Mul, Distrib for PNat
2830

@@ -272,13 +274,8 @@ theorem coe_bit1 (a : ℕ+) : ((bit1 a : ℕ+) : ℕ) = bit1 (a : ℕ) :=
272274

273275
end deprecated
274276

275-
-- Porting note:
276-
-- mathlib3 statement was
277-
-- `((m ^ n : ℕ+) : ℕ) = (m : ℕ) ^ n`
278-
-- where the left `^ : ℕ+ → ℕ → ℕ+` was `monoid.has_pow`.
279-
-- Atm writing `m ^ n` means automatically `(↑m) ^ n`.
280277
@[simp, norm_cast]
281-
theorem pow_coe (m : ℕ+) (n : ℕ) : ((Pow.pow m n : ℕ+) : ℕ) = (m : ℕ) ^ n :=
278+
theorem pow_coe (m : ℕ+) (n : ℕ) : (m ^ n : ℕ) = (m : ℕ) ^ n :=
282279
rfl
283280
#align pnat.pow_coe PNat.pow_coe
284281

0 commit comments

Comments
 (0)