Documentation

Mathlib.Data.Nat.Factorization.Basic

Prime factorizations #

n.factorization is the finitely supported function ℕ →₀ ℕ mapping each prime factor of n to its multiplicity in n. For example, since 2000 = 2^4 * 5^3,

TODO #

n.factorization is the finitely supported function ℕ →₀ ℕ mapping each prime factor of n to its multiplicity in n.

Equations
Instances For
    @[simp]
    theorem Nat.support_factorization (n : ) :
    (Nat.factorization n).support = n.primeFactors

    The support of n.factorization is exactly n.primeFactors.

    @[simp]

    We can write both n.factorization p and n.factors.count p to represent the power of p in the factorization of n: we declare the former to be the simp-normal form.

    theorem Nat.multiplicity_eq_factorization {n : } {p : } (pp : Nat.Prime p) (hn : n 0) :

    Basic facts about factorization #

    @[simp]
    theorem Nat.factorization_prod_pow_eq_self {n : } (hn : n 0) :
    (Finsupp.prod (Nat.factorization n) fun (x x_1 : ) => x ^ x_1) = n
    theorem Nat.eq_of_factorization_eq {a : } {b : } (ha : a 0) (hb : b 0) (h : ∀ (p : ), (Nat.factorization a) p = (Nat.factorization b) p) :
    a = b

    Every nonzero natural number has a unique prime factorization

    Lemmas characterising when n.factorization p = 0 #

    theorem Nat.factorization_eq_zero_of_lt {n : } {p : } (h : n < p) :
    theorem Nat.dvd_of_factorization_pos {n : } {p : } (hn : (Nat.factorization n) p 0) :
    p n
    theorem Nat.Prime.factorization_pos_of_dvd {n : } {p : } (hp : Nat.Prime p) (hn : n 0) (h : p n) :
    theorem Nat.factorization_eq_zero_of_remainder {p : } {r : } (i : ) (hr : ¬p r) :
    (Nat.factorization (p * i + r)) p = 0
    theorem Nat.factorization_eq_zero_iff_remainder {p : } {r : } (i : ) (pp : Nat.Prime p) (hr0 : r 0) :
    ¬p r (Nat.factorization (p * i + r)) p = 0

    The only numbers with empty prime factorization are 0 and 1

    Lemmas about factorizations of products and powers #

    @[simp]
    theorem Nat.factorization_mul {a : } {b : } (ha : a 0) (hb : b 0) :

    For nonzero a and b, the power of p in a * b is the sum of the powers in a and b

    theorem Nat.prod_factorization_eq_prod_primeFactors {n : } {β : Type u_1} [CommMonoid β] (f : β) :
    Finsupp.prod (Nat.factorization n) f = Finset.prod n.primeFactors fun (p : ) => f p ((Nat.factorization n) p)

    A product over n.factorization can be written as a product over n.primeFactors;

    theorem Nat.prod_primeFactors_prod_factorization {n : } {β : Type u_1} [CommMonoid β] (f : β) :
    (Finset.prod n.primeFactors fun (p : ) => f p) = Finsupp.prod (Nat.factorization n) fun (p x : ) => f p

    A product over n.primeFactors can be written as a product over n.factorization;

    theorem Nat.factorization_prod {α : Type u_1} {S : Finset α} {g : α} (hS : xS, g x 0) :

    For any p : ℕ and any function g : α → ℕ that's non-zero on S : Finset α, the power of p in S.prod g equals the sum over x ∈ S of the powers of p in g x. Generalises factorization_mul, which is the special case where S.card = 2 and g = id.

    @[simp]

    For any p, the power of p in n^k is k times the power in n

    Lemmas about factorizations of primes and prime powers #

    @[simp]

    The only prime factor of prime p is p itself, with multiplicity 1

    @[simp]

    The multiplicity of prime p in p is 1

    For prime p the only prime factor of p^k is p with multiplicity k

    theorem Nat.eq_pow_of_factorization_eq_single {n : } {p : } {k : } (hn : n 0) (h : Nat.factorization n = Finsupp.single p k) :
    n = p ^ k

    If the factorization of n contains just one number p then n is a power of p

    theorem Nat.Prime.eq_of_factorization_pos {p : } {q : } (hp : Nat.Prime p) (h : (Nat.factorization p) q 0) :
    p = q

    The only prime factor of prime p is p itself.

    Equivalence between ℕ+ and ℕ →₀ ℕ with support in the primes. #

    theorem Nat.prod_pow_factorization_eq_self {f : →₀ } (hf : pf.support, Nat.Prime p) :
    Nat.factorization (Finsupp.prod f fun (x x_1 : ) => x ^ x_1) = f

    Any Finsupp f : ℕ →₀ ℕ whose support is in the primes is equal to the factorization of the product ∏ (a : ℕ) in f.support, a ^ f a.

    theorem Nat.eq_factorization_iff {n : } {f : →₀ } (hn : n 0) (hf : pf.support, Nat.Prime p) :
    f = Nat.factorization n (Finsupp.prod f fun (x x_1 : ) => x ^ x_1) = n
    def Nat.factorizationEquiv :
    ℕ+ {f : →₀ | pf.support, Nat.Prime p}

    The equiv between ℕ+ and ℕ →₀ ℕ with support in the primes.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      theorem Nat.factorizationEquiv_apply (n : ℕ+) :
      (Nat.factorizationEquiv n) = Nat.factorization n
      theorem Nat.factorizationEquiv_inv_apply {f : →₀ } (hf : pf.support, Nat.Prime p) :
      (Nat.factorizationEquiv.symm { val := f, property := hf }) = Finsupp.prod f fun (x x_1 : ) => x ^ x_1

      Generalisation of the "even part" and "odd part" of a natural number #

      We introduce the notations ord_proj[p] n for the largest power of the prime p that divides n and ord_compl[p] n for the complementary part. The ord naming comes from the $p$-adic order/valuation of a number, and proj and compl are for the projection and complementary projection. The term n.factorization p is the $p$-adic order itself. For example, ord_proj[2] n is the even part of n and ord_compl[2] n is the odd part.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          @[simp]
          theorem Nat.ord_proj_of_not_prime (n : ) (p : ) (hp : ¬Nat.Prime p) :
          @[simp]
          theorem Nat.ord_compl_of_not_prime (n : ) (p : ) (hp : ¬Nat.Prime p) :
          n / p ^ (Nat.factorization n) p = n
          theorem Nat.ord_proj_dvd (n : ) (p : ) :
          theorem Nat.ord_compl_dvd (n : ) (p : ) :
          n / p ^ (Nat.factorization n) p n
          theorem Nat.ord_proj_pos (n : ) (p : ) :
          theorem Nat.ord_proj_le {n : } (p : ) (hn : n 0) :
          theorem Nat.ord_compl_pos {n : } (p : ) (hn : n 0) :
          0 < n / p ^ (Nat.factorization n) p
          theorem Nat.ord_compl_le (n : ) (p : ) :
          n / p ^ (Nat.factorization n) p n
          theorem Nat.ord_proj_mul {a : } {b : } (p : ) (ha : a 0) (hb : b 0) :
          theorem Nat.ord_compl_mul (a : ) (b : ) (p : ) :
          a * b / p ^ (Nat.factorization (a * b)) p = a / p ^ (Nat.factorization a) p * (b / p ^ (Nat.factorization b) p)

          Factorization and divisibility #

          theorem Nat.factorization_lt {n : } (p : ) (hn : n 0) :

          A crude upper bound on n.factorization p

          theorem Nat.factorization_le_of_le_pow {n : } {p : } {b : } (hb : n p ^ b) :

          An upper bound on n.factorization p

          theorem Nat.factorization_le_iff_dvd {d : } {n : } (hd : d 0) (hn : n 0) :
          theorem Nat.factorization_prime_le_iff_dvd {d : } {n : } (hd : d 0) (hn : n 0) :
          (∀ (p : ), Nat.Prime p(Nat.factorization d) p (Nat.factorization n) p) d n
          theorem Nat.pow_succ_factorization_not_dvd {n : } {p : } (hn : n 0) (hp : Nat.Prime p) :
          ¬p ^ ((Nat.factorization n) p + 1) n
          theorem Nat.Prime.pow_dvd_iff_le_factorization {p : } {k : } {n : } (pp : Nat.Prime p) (hn : n 0) :
          p ^ k n k (Nat.factorization n) p
          theorem Nat.Prime.pow_dvd_iff_dvd_ord_proj {p : } {k : } {n : } (pp : Nat.Prime p) (hn : n 0) :
          p ^ k n p ^ k p ^ (Nat.factorization n) p
          theorem Nat.Prime.dvd_iff_one_le_factorization {p : } {n : } (pp : Nat.Prime p) (hn : n 0) :
          theorem Nat.exists_factorization_lt_of_lt {a : } {b : } (ha : a 0) (hab : a < b) :
          ∃ (p : ), (Nat.factorization a) p < (Nat.factorization b) p
          theorem Nat.dvd_ord_proj_of_dvd {n : } {p : } (hn : n 0) (pp : Nat.Prime p) (h : p n) :
          theorem Nat.not_dvd_ord_compl {n : } {p : } (hp : Nat.Prime p) (hn : n 0) :
          theorem Nat.coprime_ord_compl {n : } {p : } (hp : Nat.Prime p) (hn : n 0) :
          theorem Nat.dvd_ord_compl_of_dvd_not_dvd {p : } {d : } {n : } (hdn : d n) (hpd : ¬p d) :
          d n / p ^ (Nat.factorization n) p
          theorem Nat.exists_eq_pow_mul_and_not_dvd {n : } (hn : n 0) (p : ) (hp : p 1) :
          ∃ (e : ) (n' : ), ¬p n' n = p ^ e * n'

          If n is a nonzero natural number and p ≠ 1, then there are natural numbers e and n' such that n' is not divisible by p and n = p^e * n'.

          theorem Nat.ord_proj_dvd_ord_proj_of_dvd {a : } {b : } (hb0 : b 0) (hab : a b) (p : ) :
          theorem Nat.ord_proj_dvd_ord_proj_iff_dvd {a : } {b : } (ha0 : a 0) (hb0 : b 0) :
          (∀ (p : ), p ^ (Nat.factorization a) p p ^ (Nat.factorization b) p) a b
          theorem Nat.ord_compl_dvd_ord_compl_of_dvd {a : } {b : } (hab : a b) (p : ) :
          theorem Nat.ord_compl_dvd_ord_compl_iff_dvd (a : ) (b : ) :
          (∀ (p : ), a / p ^ (Nat.factorization a) p b / p ^ (Nat.factorization b) p) a b
          theorem Nat.dvd_iff_prime_pow_dvd_dvd (n : ) (d : ) :
          d n ∀ (p k : ), Nat.Prime pp ^ k dp ^ k n
          theorem Nat.prod_primeFactors_dvd (n : ) :
          (Finset.prod n.primeFactors fun (p : ) => p) n
          theorem Nat.factorization_gcd {a : } {b : } (ha_pos : a 0) (hb_pos : b 0) :

          If a = ∏ pᵢ ^ nᵢ and b = ∏ pᵢ ^ mᵢ, then factorizationLCMLeft = ∏ pᵢ ^ kᵢ, where kᵢ = nᵢ if mᵢ ≤ nᵢ and 0 otherwise. Note that the product is over the divisors of lcm a b, so if one of a or b is 0 then the result is 1.

          Equations
          Instances For

            If a = ∏ pᵢ ^ nᵢ and b = ∏ pᵢ ^ mᵢ, then factorizationLCMRight = ∏ pᵢ ^ kᵢ, where kᵢ = mᵢ if nᵢ < mᵢ and 0 otherwise. Note that the product is over the divisors of lcm a b, so if one of a or b is 0 then the result is 1.

            Note that factorizationLCMRight a b is not factorizationLCMLeft b a: the difference is that in factorizationLCMLeft a b there are the primes whose exponent in a is bigger or equal than the exponent in b, while in factorizationLCMRight a b there are the primes primes whose exponent in b is strictly bigger than in a. For example factorizationLCMLeft 2 2 = 2, but factorizationLCMRight 2 2 = 1.

            Equations
            Instances For
              theorem Nat.sum_primeFactors_gcd_add_sum_primeFactors_mul {β : Type u_1} [AddCommMonoid β] (m : ) (n : ) (f : β) :
              Finset.sum (Nat.gcd m n).primeFactors f + Finset.sum (m * n).primeFactors f = Finset.sum m.primeFactors f + Finset.sum n.primeFactors f
              theorem Nat.prod_primeFactors_gcd_mul_prod_primeFactors_mul {β : Type u_1} [CommMonoid β] (m : ) (n : ) (f : β) :
              Finset.prod (Nat.gcd m n).primeFactors f * Finset.prod (m * n).primeFactors f = Finset.prod m.primeFactors f * Finset.prod n.primeFactors f
              theorem Nat.setOf_pow_dvd_eq_Icc_factorization {n : } {p : } (pp : Nat.Prime p) (hn : n 0) :
              {i : | i 0 p ^ i n} = Set.Icc 1 ((Nat.factorization n) p)
              theorem Nat.Icc_factorization_eq_pow_dvd (n : ) {p : } (pp : Nat.Prime p) :
              Finset.Icc 1 ((Nat.factorization n) p) = Finset.filter (fun (i : ) => p ^ i n) (Finset.Ico 1 n)

              The set of positive powers of prime p that divide n is exactly the set of positive natural numbers up to n.factorization p.

              theorem Nat.factorization_eq_card_pow_dvd (n : ) {p : } (pp : Nat.Prime p) :
              (Nat.factorization n) p = (Finset.filter (fun (i : ) => p ^ i n) (Finset.Ico 1 n)).card
              theorem Nat.Ico_filter_pow_dvd_eq {n : } {p : } {b : } (pp : Nat.Prime p) (hn : n 0) (hb : n p ^ b) :
              Finset.filter (fun (i : ) => p ^ i n) (Finset.Ico 1 n) = Finset.filter (fun (i : ) => p ^ i n) (Finset.Icc 1 b)

              Factorization and coprimes #

              For coprime a and b, the power of p in a * b is the sum of the powers in a and b

              For coprime a and b, the power of p in a * b is the sum of the powers in a and b

              theorem Nat.factorization_eq_of_coprime_left {p : } {a : } {b : } (hab : Nat.Coprime a b) (hpa : p Nat.factors a) :

              If p is a prime factor of a then the power of p in a is the same that in a * b, for any b coprime to a.

              theorem Nat.factorization_eq_of_coprime_right {p : } {a : } {b : } (hab : Nat.Coprime a b) (hpb : p Nat.factors b) :

              If p is a prime factor of b then the power of p in b is the same that in a * b, for any a coprime to b.

              Induction principles involving factorizations #

              def Nat.recOnPrimePow {P : Sort u_1} (h0 : P 0) (h1 : P 1) (h : (a p n : ) → Nat.Prime p¬p a0 < nP aP (p ^ n * a)) (a : ) :
              P a

              Given P 0, P 1 and a way to extend P a to P (p ^ n * a) for prime p not dividing a, we can define P for all natural numbers.

              Equations
              • One or more equations did not get rendered due to their size.
              Instances For
                def Nat.recOnPosPrimePosCoprime {P : Sort u_1} (hp : (p n : ) → Nat.Prime p0 < nP (p ^ n)) (h0 : P 0) (h1 : P 1) (h : (a b : ) → 1 < a1 < bNat.Coprime a bP aP bP (a * b)) (a : ) :
                P a

                Given P 0, P 1, and P (p ^ n) for positive prime powers, and a way to extend P a and P b to P (a * b) when a, b are positive coprime, we can define P for all natural numbers.

                Equations
                • One or more equations did not get rendered due to their size.
                Instances For
                  def Nat.recOnPrimeCoprime {P : Sort u_1} (h0 : P 0) (hp : (p n : ) → Nat.Prime pP (p ^ n)) (h : (a b : ) → 1 < a1 < bNat.Coprime a bP aP bP (a * b)) (a : ) :
                  P a

                  Given P 0, P (p ^ n) for all prime powers, and a way to extend P a and P b to P (a * b) when a, b are positive coprime, we can define P for all natural numbers.

                  Equations
                  Instances For
                    def Nat.recOnMul {P : Sort u_1} (h0 : P 0) (h1 : P 1) (hp : (p : ) → Nat.Prime pP p) (h : (a b : ) → P aP bP (a * b)) (a : ) :
                    P a

                    Given P 0, P 1, P p for all primes, and a way to extend P a and P b to P (a * b), we can define P for all natural numbers.

                    Equations
                    • One or more equations did not get rendered due to their size.
                    Instances For
                      theorem Nat.multiplicative_factorization {β : Type u_1} [CommMonoid β] (f : β) (h_mult : ∀ (x y : ), Nat.Coprime x yf (x * y) = f x * f y) (hf : f 1 = 1) {n : } :
                      n 0f n = Finsupp.prod (Nat.factorization n) fun (p k : ) => f (p ^ k)

                      For any multiplicative function f with f 1 = 1 and any n ≠ 0, we can evaluate f n by evaluating f at p ^ k over the factorization of n

                      theorem Nat.multiplicative_factorization' {n : } {β : Type u_1} [CommMonoid β] (f : β) (h_mult : ∀ (x y : ), Nat.Coprime x yf (x * y) = f x * f y) (hf0 : f 0 = 1) (hf1 : f 1 = 1) :
                      f n = Finsupp.prod (Nat.factorization n) fun (p k : ) => f (p ^ k)

                      For any multiplicative function f with f 1 = 1 and f 0 = 1, we can evaluate f n by evaluating f at p ^ k over the factorization of n

                      theorem Nat.eq_iff_prime_padicValNat_eq (a : ) (b : ) (ha : a 0) (hb : b 0) :
                      a = b ∀ (p : ), Nat.Prime ppadicValNat p a = padicValNat p b

                      Two positive naturals are equal if their prime padic valuations are equal

                      theorem Nat.prod_pow_prime_padicValNat (n : ) (hn : n 0) (m : ) (pr : n < m) :

                      Lemmas about factorizations of particular functions #

                      theorem Nat.card_multiples (n : ) (p : ) :
                      (Finset.filter (fun (e : ) => p e + 1) (Finset.range n)).card = n / p

                      Exactly n / p naturals in [1, n] are multiples of p. See Nat.card_multiples' for an alternative spelling of the statement.

                      theorem Nat.Ioc_filter_dvd_card_eq_div (n : ) (p : ) :
                      (Finset.filter (fun (x : ) => p x) (Finset.Ioc 0 n)).card = n / p

                      Exactly n / p naturals in (0, n] are multiples of p.

                      theorem Nat.card_multiples' (N : ) (n : ) :
                      (Finset.filter (fun (k : ) => k 0 n k) (Finset.range (Nat.succ N))).card = N / n

                      There are exactly ⌊N/n⌋ positive multiples of n that are ≤ N. See Nat.card_multiples for a "shifted-by-one" version.