Skip to content

Commit

Permalink
chore(RingTheory/Ideal): split Quotient.lean into Defs and Basic (
Browse files Browse the repository at this point in the history
#18393)

This PR renames and splits files involved in the ideal quotient.
Changes:
* `RingTheory/Ideal/Quotient.lean` is split into
  - `RingTheory/Ideal/Quotient/Defs.lean` (definition of ideal quotient and ring structure)
 * `RingTheory/Ideal/Quotient/Basic.lean` (further results)
* `RingTheory/QuotientNilpotent.lean` is renamed to `RingTheory/Ideal/Quotient/Nilpotent.lean`
* `RingTheory/QuotientNoetherian.lean` is renamed to `Mathlib/RingTheory/Ideal/Quotient/Noetherian.lean`
* `RingTheory/Ideal/QuotientOperations.lean` is renamed to `Mathlib/RingTheory/Ideal/Quotient/Operations.lean`



Co-authored-by: Kim Morrison <[email protected]>
  • Loading branch information
Vierkantor and kim-em committed Oct 30, 2024
1 parent 3977332 commit abfa430
Show file tree
Hide file tree
Showing 39 changed files with 237 additions and 185 deletions.
9 changes: 5 additions & 4 deletions Mathlib.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4088,8 +4088,11 @@ import Mathlib.RingTheory.Ideal.Over
import Mathlib.RingTheory.Ideal.Pointwise
import Mathlib.RingTheory.Ideal.Prime
import Mathlib.RingTheory.Ideal.Prod
import Mathlib.RingTheory.Ideal.Quotient
import Mathlib.RingTheory.Ideal.QuotientOperations
import Mathlib.RingTheory.Ideal.Quotient.Basic
import Mathlib.RingTheory.Ideal.Quotient.Defs
import Mathlib.RingTheory.Ideal.Quotient.Nilpotent
import Mathlib.RingTheory.Ideal.Quotient.Noetherian
import Mathlib.RingTheory.Ideal.Quotient.Operations
import Mathlib.RingTheory.Ideal.Span
import Mathlib.RingTheory.Idempotents
import Mathlib.RingTheory.Int.Basic
Expand Down Expand Up @@ -4224,8 +4227,6 @@ import Mathlib.RingTheory.Prime
import Mathlib.RingTheory.PrimeSpectrum
import Mathlib.RingTheory.PrincipalIdealDomain
import Mathlib.RingTheory.QuotSMulTop
import Mathlib.RingTheory.QuotientNilpotent
import Mathlib.RingTheory.QuotientNoetherian
import Mathlib.RingTheory.Radical
import Mathlib.RingTheory.ReesAlgebra
import Mathlib.RingTheory.Regular.IsSMulRegular
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/CharP/MixedCharZero.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Jon Eugster
-/
import Mathlib.Algebra.CharP.LocalRing
import Mathlib.RingTheory.Ideal.Quotient
import Mathlib.RingTheory.Ideal.Quotient.Basic
import Mathlib.Tactic.FieldSimp

/-!
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/CharP/Quotient.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@ Authors: Kenny Lau, Eric Wieser
-/
import Mathlib.GroupTheory.OrderOfElement
import Mathlib.RingTheory.Ideal.Maps
import Mathlib.RingTheory.Ideal.Quotient
import Mathlib.RingTheory.Ideal.Quotient.Defs

/-!
# Characteristic of quotients rings
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Algebra/DirectLimit.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,7 +8,7 @@ import Mathlib.Data.Finset.Order
import Mathlib.LinearAlgebra.Quotient.Basic
import Mathlib.RingTheory.FreeCommRing
import Mathlib.RingTheory.Ideal.Maps
import Mathlib.RingTheory.Ideal.Quotient
import Mathlib.RingTheory.Ideal.Quotient.Defs
import Mathlib.Tactic.SuppressCompilation

/-!
Expand Down
4 changes: 3 additions & 1 deletion Mathlib/Algebra/RingQuot.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,9 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kim Morrison
-/
import Mathlib.Algebra.Algebra.Hom
import Mathlib.RingTheory.Ideal.Quotient
import Mathlib.RingTheory.Congruence.Basic
import Mathlib.RingTheory.Ideal.Quotient.Defs
import Mathlib.RingTheory.Ideal.Span

/-!
# Quotients of non-commutative rings
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Analysis/Normed/Group/Quotient.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@ Authors: Patrick Massot, Riccardo Brasca
-/
import Mathlib.Analysis.Normed.Module.Basic
import Mathlib.Analysis.Normed.Group.Hom
import Mathlib.RingTheory.Ideal.QuotientOperations
import Mathlib.RingTheory.Ideal.Quotient.Operations
import Mathlib.Topology.MetricSpace.HausdorffDistance

/-!
Expand Down
3 changes: 2 additions & 1 deletion Mathlib/Analysis/Normed/Ring/Units.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,8 +3,9 @@ Copyright (c) 2020 Heather Macbeth. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Heather Macbeth
-/
import Mathlib.Topology.Algebra.Ring.Ideal
import Mathlib.Analysis.SpecificLimits.Normed
import Mathlib.Topology.Algebra.Ring.Ideal
import Mathlib.RingTheory.Ideal.Basic

/-!
# The group of units of a complete normed ring
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Data/ZMod/Quotient.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,7 @@ Authors: Anne Baanen
import Mathlib.Algebra.Group.Equiv.TypeTags
import Mathlib.Data.ZMod.Basic
import Mathlib.GroupTheory.GroupAction.Quotient
import Mathlib.RingTheory.Ideal.QuotientOperations
import Mathlib.RingTheory.Ideal.Quotient.Operations
import Mathlib.RingTheory.Int.Basic
import Mathlib.RingTheory.ZMod

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/InvariantBasisNumber.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,8 +3,8 @@ Copyright (c) 2020 Markus Himmel. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Markus Himmel, Kim Morrison
-/
import Mathlib.RingTheory.Ideal.Quotient.Basic
import Mathlib.RingTheory.OrzechProperty
import Mathlib.RingTheory.Ideal.Quotient
import Mathlib.RingTheory.PrincipalIdealDomain

/-!
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/LinearAlgebra/SModEq.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Kenny Lau
-/
import Mathlib.Algebra.Polynomial.Eval
import Mathlib.RingTheory.Ideal.Quotient
import Mathlib.RingTheory.Ideal.Quotient.Defs

/-!
# modular equivalence for submodule
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/LinearAlgebra/Semisimple.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,10 +4,10 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Oliver Nash
-/
import Mathlib.FieldTheory.Perfect
import Mathlib.LinearAlgebra.Basis.VectorSpace
import Mathlib.LinearAlgebra.AnnihilatingPolynomial
import Mathlib.LinearAlgebra.Basis.VectorSpace
import Mathlib.RingTheory.Artinian
import Mathlib.RingTheory.QuotientNilpotent
import Mathlib.RingTheory.Ideal.Quotient.Nilpotent
import Mathlib.RingTheory.SimpleModule

/-!
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/LinearAlgebra/TensorProduct/Quotient.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,11 +4,11 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Antoine Chambert-Loir, Jujian Zhang
-/

import Mathlib.RingTheory.Ideal.Operations
import Mathlib.LinearAlgebra.TensorProduct.Basic
import Mathlib.LinearAlgebra.Quotient.Basic
import Mathlib.LinearAlgebra.Prod
import Mathlib.RingTheory.Ideal.Quotient
import Mathlib.RingTheory.Ideal.Operations
import Mathlib.RingTheory.Ideal.Quotient.Defs

/-!
Expand Down
3 changes: 2 additions & 1 deletion Mathlib/NumberTheory/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,8 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Johan Commelin, Kenny Lau
-/
import Mathlib.Algebra.GeomSum
import Mathlib.RingTheory.Ideal.Quotient
import Mathlib.RingTheory.Ideal.Quotient.Defs
import Mathlib.RingTheory.Ideal.Span

/-!
# Basic results in number theory
Expand Down
4 changes: 3 additions & 1 deletion Mathlib/NumberTheory/Multiplicity.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,9 +6,11 @@ Authors: Tian Chen, Mantas Bakšys
import Mathlib.Algebra.GeomSum
import Mathlib.Algebra.Order.Ring.Basic
import Mathlib.Algebra.Ring.Int
import Mathlib.Data.Nat.Choose.Sum
import Mathlib.Data.Nat.Prime.Int
import Mathlib.NumberTheory.Padics.PadicVal.Defs
import Mathlib.RingTheory.Ideal.Quotient
import Mathlib.RingTheory.Ideal.Quotient.Defs
import Mathlib.RingTheory.Ideal.Span

/-!
# Multiplicity in Number Theory
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/AdjoinRoot.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,9 +9,9 @@ import Mathlib.FieldTheory.Minpoly.Basic
import Mathlib.RingTheory.Adjoin.Basic
import Mathlib.RingTheory.FinitePresentation
import Mathlib.RingTheory.FiniteType
import Mathlib.RingTheory.Ideal.Quotient.Noetherian
import Mathlib.RingTheory.PowerBasis
import Mathlib.RingTheory.PrincipalIdealDomain
import Mathlib.RingTheory.QuotientNoetherian
import Mathlib.RingTheory.Polynomial.Quotient

/-!
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/Derivation/ToSquareZero.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Nicolò Cavalleri, Andrew Yang
-/
import Mathlib.RingTheory.Derivation.Basic
import Mathlib.RingTheory.Ideal.QuotientOperations
import Mathlib.RingTheory.Ideal.Quotient.Operations

/-!
# Results
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/RingTheory/EisensteinCriterion.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,9 +4,9 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Chris Hughes
-/
import Mathlib.Data.Nat.Cast.WithTop
import Mathlib.RingTheory.Prime
import Mathlib.RingTheory.Ideal.Quotient.Basic
import Mathlib.RingTheory.Polynomial.Content
import Mathlib.RingTheory.Ideal.Quotient
import Mathlib.RingTheory.Prime

/-!
# Eisenstein's criterion
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/Etale/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2022 Andrew Yang. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Andrew Yang
-/
import Mathlib.RingTheory.QuotientNilpotent
import Mathlib.RingTheory.Ideal.Quotient.Nilpotent
import Mathlib.RingTheory.Smooth.Basic
import Mathlib.RingTheory.Unramified.Basic

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/FinitePresentation.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,8 +4,8 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Johan Commelin
-/
import Mathlib.RingTheory.FiniteType
import Mathlib.RingTheory.Ideal.Quotient.Operations
import Mathlib.RingTheory.MvPolynomial.Tower
import Mathlib.RingTheory.Ideal.QuotientOperations

/-!
# Finiteness conditions in commutative algebra
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/FiniteType.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@ Authors: Johan Commelin
-/
import Mathlib.Algebra.FreeAlgebra
import Mathlib.RingTheory.Adjoin.Tower
import Mathlib.RingTheory.Ideal.QuotientOperations
import Mathlib.RingTheory.Ideal.Quotient.Operations

/-!
# Finiteness conditions in commutative algebra
Expand Down
3 changes: 2 additions & 1 deletion Mathlib/RingTheory/Flat/FaithfullyFlat.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,8 +4,9 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Judith Ludwig, Florent Schaffhauser, Yunzhou Xie, Jujian Zhang
-/

import Mathlib.RingTheory.Flat.Stability
import Mathlib.LinearAlgebra.TensorProduct.Quotient
import Mathlib.RingTheory.Flat.Stability
import Mathlib.RingTheory.Ideal.Quotient.Basic

/-!
# Faithfully flat modules
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/Ideal/AssociatedPrime.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@ Authors: Andrew Yang
-/
import Mathlib.LinearAlgebra.Span
import Mathlib.RingTheory.Ideal.IsPrimary
import Mathlib.RingTheory.Ideal.QuotientOperations
import Mathlib.RingTheory.Ideal.Quotient.Operations
import Mathlib.RingTheory.Noetherian

/-!
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/Ideal/IsPrincipalPowQuotient.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@ Authors: Yakov Pechersky
-/
import Mathlib.LinearAlgebra.Isomorphisms
import Mathlib.RingTheory.Ideal.Operations
import Mathlib.RingTheory.Ideal.Quotient
import Mathlib.RingTheory.Ideal.Quotient.Defs

/-!
# Quotients of powers of principal ideals
Expand Down
Loading

0 comments on commit abfa430

Please sign in to comment.