Skip to content

Commit

Permalink
chore: Split RingTheory.FractionalIdeal.Basic (#9854)
Browse files Browse the repository at this point in the history
The file `RingTheory.FractionalIdeal.Basic` is more than 1600 lines long. This PR splits it into two files: `Basic` and `Operations` following the model of `RingTheory.Ideal.Basic` and `RingTheory.Ideal.Operations`

 

Co-authored-by: Mario Carneiro <mcarneir@andrew.cmu.edu>
Co-authored-by: Jz Pan <acme_pjz@hotmail.com>
  • Loading branch information
3 people committed Jan 19, 2024
1 parent 50388bc commit de9c7b5
Show file tree
Hide file tree
Showing 4 changed files with 984 additions and 954 deletions.
1 change: 1 addition & 0 deletions Mathlib.lean
Expand Up @@ -3117,6 +3117,7 @@ import Mathlib.RingTheory.Fintype
import Mathlib.RingTheory.Flat
import Mathlib.RingTheory.FractionalIdeal.Basic
import Mathlib.RingTheory.FractionalIdeal.Norm
import Mathlib.RingTheory.FractionalIdeal.Operations
import Mathlib.RingTheory.FreeCommRing
import Mathlib.RingTheory.FreeRing
import Mathlib.RingTheory.GradedAlgebra.Basic
Expand Down
6 changes: 2 additions & 4 deletions Mathlib/RingTheory/DedekindDomain/Ideal.lean
Expand Up @@ -6,11 +6,9 @@ Authors: Kenji Nakagawa, Anne Baanen, Filippo A. E. Nuccio
import Mathlib.Algebra.Algebra.Subalgebra.Pointwise
import Mathlib.AlgebraicGeometry.PrimeSpectrum.Maximal
import Mathlib.AlgebraicGeometry.PrimeSpectrum.Noetherian
import Mathlib.Order.Hom.Basic
import Mathlib.RingTheory.DedekindDomain.Basic
import Mathlib.RingTheory.FractionalIdeal.Basic
import Mathlib.RingTheory.PrincipalIdealDomain
import Mathlib.RingTheory.ChainOfDivisors
import Mathlib.RingTheory.DedekindDomain.Basic
import Mathlib.RingTheory.FractionalIdeal.Operations

#align_import ring_theory.dedekind_domain.ideal from "leanprover-community/mathlib"@"2bbc7e3884ba234309d2a43b19144105a753292e"

Expand Down

0 comments on commit de9c7b5

Please sign in to comment.