Factorization of Binomial Coefficients #
This file contains a few results on the multiplicity of prime factors within certain size bounds in binomial coefficients. These include:
- Nat.factorization_choose_le_log: a logarithmic upper bound on the multiplicity of a prime in a binomial coefficient.
- Nat.factorization_choose_le_one: Primes above- sqrt nappear at most once in the factorization of- nchoose- k.
- Nat.factorization_centralBinom_of_two_mul_self_lt_three_mul: Primes from- 2 * n / 3to- ndo not appear in the factorization of the- nth central binomial coefficient.
- Nat.factorization_choose_eq_zero_of_lt: Primes greater than- ndo not appear in the factorization of- nchoose- k.
These results appear in the Erdős proof of Bertrand's postulate.
Legendre's Theorem
The multiplicity of a prime in n! is the sum of the quotients n / p ^ i. This sum is expressed
over the finset Ico 1 b where b is any bound greater than log p n.
The factorization of p in (p * (n + 1))! is one more than the sum of the factorizations of
p in (p * n)! and n + 1.
The factorization of p in (p * n)! is n more than that of n!.
Modified version of emultiplicity_le_emultiplicity_of_dvd_right
but for factorization.
A lower bound on the factorization of p in choose n k.
A logarithmic upper bound on the multiplicity of a prime in a binomial coefficient.
A pow form of Nat.factorization_choose_le
Primes greater than about sqrt n appear only to multiplicity 0 or 1
in the binomial coefficient.
If a prime p has positive multiplicity in the nth central binomial coefficient,
p is no more than 2 * n
Contrapositive form of Nat.factorization_centralBinom_eq_zero_of_two_mul_lt
A binomial coefficient is the product of its prime factors, which are at most n.
The nth central binomial coefficient is the product of its prime factors, which are
at most 2n.