Skip to content

Commit

Permalink
chore: split Mathlib.Topology.Algebra.UniformGroup
Browse files Browse the repository at this point in the history
  • Loading branch information
kim-em committed Oct 28, 2024
1 parent 2061d03 commit dd28b47
Show file tree
Hide file tree
Showing 17 changed files with 559 additions and 416 deletions.
3 changes: 2 additions & 1 deletion Mathlib.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4669,7 +4669,8 @@ import Mathlib.Topology.Algebra.StarSubalgebra
import Mathlib.Topology.Algebra.UniformConvergence
import Mathlib.Topology.Algebra.UniformField
import Mathlib.Topology.Algebra.UniformFilterBasis
import Mathlib.Topology.Algebra.UniformGroup
import Mathlib.Topology.Algebra.UniformGroup.Basic
import Mathlib.Topology.Algebra.UniformGroup.Defs
import Mathlib.Topology.Algebra.UniformMulAction
import Mathlib.Topology.Algebra.UniformRing
import Mathlib.Topology.Algebra.Valued.NormedValued
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Analysis/Convex/TotallyBounded.lean
Original file line number Diff line number Diff line change
Expand Up @@ -6,7 +6,7 @@ Authors: Christopher Hoskin

import Mathlib.Topology.UniformSpace.Cauchy
import Mathlib.Analysis.Convex.Hull
import Mathlib.Topology.Algebra.UniformGroup
import Mathlib.Topology.Algebra.UniformGroup.Basic
import Mathlib.Topology.Algebra.Module.LocallyConvex

/-!
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Analysis/LocallyConvex/Bounded.lean
Original file line number Diff line number Diff line change
Expand Up @@ -9,7 +9,7 @@ import Mathlib.Analysis.LocallyConvex.BalancedCoreHull
import Mathlib.Analysis.Seminorm
import Mathlib.LinearAlgebra.Basis.VectorSpace
import Mathlib.Topology.Bornology.Basic
import Mathlib.Topology.Algebra.UniformGroup
import Mathlib.Topology.Algebra.UniformGroup.Basic
import Mathlib.Topology.UniformSpace.Cauchy
import Mathlib.Topology.Algebra.Module.Basic

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Analysis/Normed/Group/Uniform.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2018 Patrick Massot. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Patrick Massot, Johannes Hölzl, Yaël Dillies
-/
import Mathlib.Topology.Algebra.UniformGroup
import Mathlib.Topology.Algebra.UniformGroup.Basic
import Mathlib.Topology.MetricSpace.Algebra
import Mathlib.Topology.MetricSpace.IsometricSMul
import Mathlib.Analysis.Normed.Group.Basic
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Topology/Algebra/Equicontinuity.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Anatole Dedecker
-/
import Mathlib.Topology.Algebra.UniformConvergence
import Mathlib.Topology.UniformSpace.Equicontinuity

/-!
# Algebra-related equicontinuity criterions
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Topology/Algebra/GroupCompletion.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,7 +3,6 @@ Copyright (c) 2018 Patrick Massot. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Patrick Massot, Johannes Hölzl
-/
import Mathlib.Topology.Algebra.UniformGroup
import Mathlib.Topology.Algebra.UniformMulAction
import Mathlib.Topology.UniformSpace.Completion

Expand Down
3 changes: 2 additions & 1 deletion Mathlib/Topology/Algebra/InfiniteSum/Group.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,7 +5,8 @@ Authors: Johannes Hölzl
-/
import Mathlib.SetTheory.Cardinal.Finite
import Mathlib.Topology.Algebra.InfiniteSum.Basic
import Mathlib.Topology.Algebra.UniformGroup
import Mathlib.Topology.UniformSpace.Cauchy
import Mathlib.Topology.Algebra.UniformGroup.Defs

/-!
# Infinite sums and products in topological groups
Expand Down
3 changes: 2 additions & 1 deletion Mathlib/Topology/Algebra/Module/Basic.lean
Original file line number Diff line number Diff line change
Expand Up @@ -11,8 +11,9 @@ import Mathlib.LinearAlgebra.Pi
import Mathlib.LinearAlgebra.Projection
import Mathlib.Topology.Algebra.MulAction
import Mathlib.Topology.Algebra.Ring.Basic
import Mathlib.Topology.Algebra.UniformGroup
import Mathlib.Topology.UniformSpace.UniformEmbedding
import Mathlib.Topology.Algebra.Group.Quotient
import Mathlib.Topology.Algebra.UniformGroup.Defs

/-!
# Theory of topological modules and continuous linear maps.
Expand Down
1 change: 1 addition & 0 deletions Mathlib/Topology/Algebra/UniformConvergence.lean
Original file line number Diff line number Diff line change
Expand Up @@ -5,6 +5,7 @@ Authors: Anatole Dedecker
-/
import Mathlib.Topology.Algebra.UniformMulAction
import Mathlib.Algebra.Module.Pi
import Mathlib.Topology.UniformSpace.UniformConvergenceTopology

/-!
# Algebraic facts about the topology of uniform convergence
Expand Down
1 change: 0 additions & 1 deletion Mathlib/Topology/Algebra/UniformFilterBasis.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,6 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Patrick Massot
-/
import Mathlib.Topology.Algebra.FilterBasis
import Mathlib.Topology.Algebra.UniformGroup

/-!
# Uniform properties of neighborhood bases in topological algebra
Expand Down
Loading

0 comments on commit dd28b47

Please sign in to comment.