Skip to content

Commit 427742c

Browse files
Vierkantorkim-em
andcommitted
chore(RingTheory/Localization/Basic): split off Defs (#17735)
This PR splits off a `RingTheory.Localization.Defs` file that is supposed to contain the definition of `IsLocalization` and the ring structure on `Localization`, and some basic results that don't need further imports. I am quite sure that we can minimize the transitive imports a bit further but this seems like a decent point to stop for now. Co-authored-by: Kim Morrison <kim@tqft.net>
1 parent dbbb99a commit 427742c

File tree

7 files changed

+919
-797
lines changed

7 files changed

+919
-797
lines changed

Mathlib.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -4000,6 +4000,7 @@ import Mathlib.RingTheory.Localization.Away.Lemmas
40004000
import Mathlib.RingTheory.Localization.BaseChange
40014001
import Mathlib.RingTheory.Localization.Basic
40024002
import Mathlib.RingTheory.Localization.Cardinality
4003+
import Mathlib.RingTheory.Localization.Defs
40034004
import Mathlib.RingTheory.Localization.Finiteness
40044005
import Mathlib.RingTheory.Localization.FractionRing
40054006
import Mathlib.RingTheory.Localization.Ideal

Mathlib/Algebra/Module/LocalizedModule.lean

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -4,8 +4,9 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Andrew Yang, Jujian Zhang
55
-/
66
import Mathlib.Algebra.Algebra.Bilinear
7-
import Mathlib.RingTheory.Localization.Basic
87
import Mathlib.Algebra.Exact
8+
import Mathlib.Algebra.Algebra.Tower
9+
import Mathlib.RingTheory.Localization.Defs
910

1011
/-!
1112
# Localized Module

Mathlib/Algebra/Polynomial/Laurent.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -6,7 +6,7 @@ Authors: Damiano Testa
66
import Mathlib.Algebra.Polynomial.AlgebraMap
77
import Mathlib.Algebra.Polynomial.Reverse
88
import Mathlib.Algebra.Polynomial.Inductions
9-
import Mathlib.RingTheory.Localization.Basic
9+
import Mathlib.RingTheory.Localization.Defs
1010

1111
/-! # Laurent polynomials
1212

0 commit comments

Comments
 (0)