Skip to content

Commit

Permalink
feat: port Data.PNat.Factors (#1830)
Browse files Browse the repository at this point in the history
Co-authored-by: qawbecrdtey <qawbecrdtey@naver.com>
Co-authored-by: int-y1 <jason_yuen2007@hotmail.com>
Co-authored-by: Ruben Van de Velde <65514131+Ruben-VandeVelde@users.noreply.github.com>
Co-authored-by: Lukas Miaskiwskyi <lukas.mias@gmail.com>
  • Loading branch information
5 people committed Feb 6, 2023
1 parent 8e39855 commit 948f2ea
Show file tree
Hide file tree
Showing 4 changed files with 435 additions and 1 deletion.
1 change: 1 addition & 0 deletions Mathlib.lean
Expand Up @@ -509,6 +509,7 @@ import Mathlib.Data.PFun
import Mathlib.Data.PFunctor.Univariate.Basic
import Mathlib.Data.PNat.Basic
import Mathlib.Data.PNat.Defs
import Mathlib.Data.PNat.Factors
import Mathlib.Data.PNat.Find
import Mathlib.Data.PNat.Interval
import Mathlib.Data.PNat.Prime
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Data/Nat/Prime.lean
Expand Up @@ -768,6 +768,7 @@ theorem prime_iff_prime_int {p : ℕ} : p.Prime ↔ _root_.Prime (p : ℤ) :=
/-- The type of prime numbers -/
def Primes :=
{ p : ℕ // p.Prime }
deriving DecidableEq
#align nat.primes Nat.Primes

namespace Primes
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/PNat/Basic.lean
Expand Up @@ -278,7 +278,7 @@ end deprecated
-- where the left `^ : ℕ+ → ℕ → ℕ+` was `monoid.has_pow`.
-- Atm writing `m ^ n` means automatically `(↑m) ^ n`.
@[simp, norm_cast]
theorem pow_coe (m : ℕ+) (n : ℕ) : ((Monoid.Pow.pow m n : ℕ+) : ℕ) = (m : ℕ) ^ n :=
theorem pow_coe (m : ℕ+) (n : ℕ) : ((Pow.pow m n : ℕ+) : ℕ) = (m : ℕ) ^ n :=
rfl
#align pnat.pow_coe PNat.pow_coe

Expand Down

0 comments on commit 948f2ea

Please sign in to comment.