Factorization of Binomial Coefficients #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
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 abovesqrt nappear at most once in the factorization ofnchoosek.nat.factorization_central_binom_of_two_mul_self_lt_three_mul: Primes from2 * n / 3tondo not appear in the factorization of thenth central binomial coefficient.nat.factorization_choose_eq_zero_of_lt: Primes greater thanndo not appear in the factorization ofnchoosek.
These results appear in the Erdős proof of Bertrand's postulate.
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.
Primes greater than about 2 * n / 3 and less than n do not appear in the factorization of
central_binom n.
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_central_binom_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.