Multiplicity in Number Theory #
This file contains results in number theory relating to multiplicity.
Main statements #
multiplicity.Int.pow_sub_pow
is the lifting the exponent lemma for odd primes. We also prove several variations of the lemma.
References #
- [Wikipedia, Lifting-the-exponent lemma] (https://en.wikipedia.org/wiki/Lifting-the-exponent_lemma)
theorem
Int.two_pow_sub_pow
{x y : ℤ}
{n : ℕ}
(hxy : 2 ∣ x - y)
(hx : ¬2 ∣ x)
(hn : Even n)
:
emultiplicity 2 (x ^ n - y ^ n) + 1 = emultiplicity 2 (x + y) + emultiplicity 2 (x - y) + emultiplicity 2 ↑n
Lifting the exponent lemma for p = 2
theorem
Nat.two_pow_sub_pow
{x y : ℕ}
(hxy : 2 ∣ x - y)
(hx : ¬2 ∣ x)
{n : ℕ}
(hn : Even n)
:
emultiplicity 2 (x ^ n - y ^ n) + 1 = emultiplicity 2 (x + y) + emultiplicity 2 (x - y) + emultiplicity 2 n