Commit 2024-11-20 11:43 b6fb044a

View on Github →

chore(RingTheory): split UniqueFactorizationDomain.lean (#19256) This PR splits the big file UniqueFactorizationDomain.lean into many smaller files:

  • UniqueFactorizationDomain.Defs contains the definition of WfDvdMonoid, UniqueFactorizationMonoid and factors
  • UniqueFactorizationDomain.Basic contains basic results on the previous definition such as the equivalence between UniqueFactorizationMonoid and the existence of prime factors
  • UniqueFactorizationDomain.NormalizedFactors defines UniqueFactorizationMonoid.normalizedFactors and contains basic results. (Or should we merge it into Defs/Basic?)
  • UniqueFactorizationDomain.FactorSet defines Associates.FactorSet and Associates.factors
  • UniqueFactorizationDomain.Finite proves that elements of a UFM with finitely many units have finitely many divisors. (This could be moved to Basic.lean but I find it niche enough to deserve its own file.)
  • UniqueFactorizationDomain.Finsupp defines UniqueFactorizationMonoid.factorization as a Finsupp version of factors
  • UniqueFactorizationDomain.GCDMonoid defines a GCD on a UFM
  • UniqueFactorizationDomain.Ideal shows UFDs satisfy the ascending chain condition on ideals
  • UniqueFactorizationDomain.Multiplicative contains results on multiplicative properties and functions.
  • UniqueFactorizationDomain.Multiplicity relates factors.count and multiplicity
  • UniqueFactorizationDomain.Nat contains the UniqueFactorizationMonoid Nat instance

Estimated changes

deleted def Associates.bcount
deleted def Associates.count
deleted theorem Associates.count_mul
deleted theorem Associates.count_pow
deleted theorem Associates.count_self
deleted theorem Associates.count_some
deleted theorem Associates.count_zero
deleted theorem Associates.dvd_count_pow
deleted theorem Associates.factors'_cong
deleted theorem Associates.factors_le
deleted theorem Associates.factors_mk
deleted theorem Associates.factors_mono
deleted theorem Associates.factors_mul
deleted theorem Associates.factors_one
deleted theorem Associates.factors_prod
deleted theorem Associates.factors_self
deleted theorem Associates.factors_zero
deleted theorem Associates.pow_factors
deleted theorem Associates.prod_add
deleted theorem Associates.prod_coe
deleted theorem Associates.prod_factors
deleted theorem Associates.prod_le
deleted theorem Associates.prod_mono
deleted theorem Associates.prod_top
deleted theorem Associates.sup_mul_inf
deleted theorem Associates.unique'
deleted theorem Nat.factors_eq
deleted theorem factorization_eq_count
deleted theorem factorization_mul
deleted theorem factorization_one
deleted theorem factorization_pow
deleted theorem factorization_zero
deleted theorem prime_factors_irreducible
deleted theorem prime_factors_unique
deleted theorem support_factorization
deleted theorem ufm_of_gcd_of_wfDvdMonoid
deleted theorem wellFounded_dvdNotUnit
added theorem Associates.unique'
added theorem prime_factors_unique
added def Associates.count
added theorem Associates.count_mul
added theorem Associates.count_pow
added theorem Associates.count_self
added theorem Associates.count_some
added theorem Associates.count_zero
added theorem Associates.factors_le
added theorem Associates.factors_mk
added theorem Associates.factors_mul
added theorem Associates.factors_one
added theorem Associates.pow_factors
added theorem Associates.prod_add
added theorem Associates.prod_coe
added theorem Associates.prod_le
added theorem Associates.prod_mono
added theorem Associates.prod_top
added theorem Associates.sup_mul_inf