Commit 2024-07-02 02:30 12473136

View on Github →

chore(Data/Nat): split Prime.lean (#14286) Splitting Prime.lean into Defs, Basic. The split aims at separation of defs and needed lemmas from everything else. With this split 13/18 Mathlib modules no longer import the whole Prime.lean. Prime/Defs.lean is about half the size. Motivation is a circular dependency that would prevent me from adding a lemma to Prime.lean. https://leanprover.zulipchat.com/#narrow/stream/287929-mathlib4/topic/split.20Nat.2FPrime.2Elean

Estimated changes

added theorem Int.prime_three
added theorem Int.prime_two
added theorem Nat.Prime.even_iff
added theorem Nat.Prime.even_sub_one
added theorem Nat.Prime.not_dvd_mul
added theorem Nat.Prime.pow_eq_iff
added theorem Nat.Prime.pow_inj
added theorem Nat.Prime.pow_minFac
added theorem Nat.Prime.pred_pos
added theorem Nat.coprime_of_dvd'
added theorem Nat.coprime_pow_primes
added theorem Nat.coprime_primes
added theorem Nat.coprime_two_left
added theorem Nat.coprime_two_right
added theorem Nat.dvd_prime_pow
added theorem Nat.factors_lemma
added theorem Nat.pow_minFac
added theorem Nat.succ_pred_prime
deleted theorem Int.prime_three
deleted theorem Int.prime_two
deleted theorem Nat.Prime.dvd_factorial
deleted theorem Nat.Prime.dvd_of_dvd_pow
deleted theorem Nat.Prime.eq_one_of_pow
deleted theorem Nat.Prime.eq_two_or_odd'
deleted theorem Nat.Prime.eq_two_or_odd
deleted theorem Nat.Prime.even_iff
deleted theorem Nat.Prime.even_sub_one
deleted theorem Nat.Prime.not_dvd_mul
deleted theorem Nat.Prime.not_prime_pow'
deleted theorem Nat.Prime.not_prime_pow
deleted theorem Nat.Prime.odd_of_ne_two
deleted theorem Nat.Prime.pow_eq_iff
deleted theorem Nat.Prime.pow_inj
deleted theorem Nat.Prime.pow_minFac
deleted theorem Nat.Prime.pred_pos
deleted theorem Nat.coprime_of_dvd'
deleted theorem Nat.coprime_of_lt_prime
deleted theorem Nat.coprime_pow_primes
deleted theorem Nat.coprime_primes
deleted theorem Nat.coprime_two_left
deleted theorem Nat.coprime_two_right
deleted theorem Nat.dvd_prime_pow
deleted theorem Nat.factors_lemma
deleted theorem Nat.irreducible_iff_prime
deleted theorem Nat.pow_minFac
deleted theorem Nat.prime_iff_prime_int
deleted theorem Nat.succ_pred_prime