Skip to content

Commit

Permalink
chore(AdicCompletion): move to RingTheory and make folder (#12511)
Browse files Browse the repository at this point in the history
Move `AdicCompletion` from `LinearAlgebra` into its own folder in `RingTheory` as it seems to fit better there.
  • Loading branch information
chrisflav committed Apr 29, 2024
1 parent 9cbb31e commit 283ea7e
Show file tree
Hide file tree
Showing 4 changed files with 3 additions and 3 deletions.
2 changes: 1 addition & 1 deletion Mathlib.lean
Original file line number Diff line number Diff line change
Expand Up @@ -2549,7 +2549,6 @@ import Mathlib.Lean.Meta.Simp
import Mathlib.Lean.Name
import Mathlib.Lean.PrettyPrinter.Delaborator
import Mathlib.Lean.Thunk
import Mathlib.LinearAlgebra.AdicCompletion
import Mathlib.LinearAlgebra.AffineSpace.AffineEquiv
import Mathlib.LinearAlgebra.AffineSpace.AffineMap
import Mathlib.LinearAlgebra.AffineSpace.AffineSubspace
Expand Down Expand Up @@ -3336,6 +3335,7 @@ import Mathlib.RepresentationTheory.GroupCohomology.Resolution
import Mathlib.RepresentationTheory.Invariants
import Mathlib.RepresentationTheory.Maschke
import Mathlib.RepresentationTheory.Rep
import Mathlib.RingTheory.AdicCompletion.Basic
import Mathlib.RingTheory.Adjoin.Basic
import Mathlib.RingTheory.Adjoin.FG
import Mathlib.RingTheory.Adjoin.Field
Expand Down
File renamed without changes.
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/DiscreteValuationRing/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,7 @@ Authors: Kevin Buzzard
import Mathlib.RingTheory.PrincipalIdealDomain
import Mathlib.RingTheory.Ideal.LocalRing
import Mathlib.RingTheory.Valuation.PrimeMultiplicity
import Mathlib.LinearAlgebra.AdicCompletion
import Mathlib.RingTheory.AdicCompletion.Basic

#align_import ring_theory.discrete_valuation_ring.basic from "leanprover-community/mathlib"@"c163ec99dfc664628ca15d215fce0a5b9c265b68"

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/Henselian.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,7 @@ Authors: Johan Commelin
-/
import Mathlib.Algebra.Polynomial.Taylor
import Mathlib.RingTheory.Ideal.LocalRing
import Mathlib.LinearAlgebra.AdicCompletion
import Mathlib.RingTheory.AdicCompletion.Basic

#align_import ring_theory.henselian from "leanprover-community/mathlib"@"d1accf4f9cddb3666c6e8e4da0ac2d19c4ed73f0"

Expand Down

0 comments on commit 283ea7e

Please sign in to comment.