Skip to content

Commit

Permalink
chore: move Topology.Support to Topology.Algebra.Support (#19651)
Browse files Browse the repository at this point in the history
to make it clear it's not pure topology. Indeed, the support is the preimage of `0`, which is an algebraic object. Sounds quite trivial like that, but the file actually imports `Module`!
  • Loading branch information
YaelDillies committed Dec 1, 2024
1 parent 65cc543 commit 2aefce6
Show file tree
Hide file tree
Showing 8 changed files with 11 additions and 11 deletions.
2 changes: 1 addition & 1 deletion Mathlib.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4994,6 +4994,7 @@ import Mathlib.Topology.Algebra.SeparationQuotient.Basic
import Mathlib.Topology.Algebra.SeparationQuotient.Section
import Mathlib.Topology.Algebra.Star
import Mathlib.Topology.Algebra.StarSubalgebra
import Mathlib.Topology.Algebra.Support
import Mathlib.Topology.Algebra.UniformConvergence
import Mathlib.Topology.Algebra.UniformField
import Mathlib.Topology.Algebra.UniformFilterBasis
Expand Down Expand Up @@ -5326,7 +5327,6 @@ import Mathlib.Topology.Sober
import Mathlib.Topology.Specialization
import Mathlib.Topology.Spectral.Hom
import Mathlib.Topology.StoneCech
import Mathlib.Topology.Support
import Mathlib.Topology.TietzeExtension
import Mathlib.Topology.Ultrafilter
import Mathlib.Topology.UniformSpace.AbsoluteValue
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Topology/Algebra/ConstMulAction.lean
Original file line number Diff line number Diff line change
Expand Up @@ -8,9 +8,9 @@ import Mathlib.Algebra.Order.Group.Synonym
import Mathlib.Data.Set.Pointwise.SMul
import Mathlib.GroupTheory.GroupAction.Defs
import Mathlib.Topology.Algebra.Constructions
import Mathlib.Topology.Algebra.Support
import Mathlib.Topology.Bases
import Mathlib.Topology.Homeomorph
import Mathlib.Topology.Support

/-!
# Monoid actions continuous in the second variable
Expand Down
File renamed without changes.
2 changes: 1 addition & 1 deletion Mathlib/Topology/ContinuousMap/CompactlySupported.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,9 +3,9 @@ Copyright (c) 2024 Yoh Tanimoto. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yoh Tanimoto
-/
import Mathlib.Topology.Algebra.Support
import Mathlib.Topology.ContinuousMap.CocompactMap
import Mathlib.Topology.ContinuousMap.ZeroAtInfty
import Mathlib.Topology.Support

/-!
# Compactly supported continuous functions
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Topology/Homeomorph.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: Johannes Hölzl, Patrick Massot, Sébastien Gouëzel, Zhouhang Zhou, Reid Barton
-/
import Mathlib.Logic.Equiv.Fin
import Mathlib.Topology.DenseEmbedding
import Mathlib.Topology.Support
import Mathlib.Topology.Algebra.Support
import Mathlib.Topology.Connected.LocallyConnected
import Mathlib.Topology.DenseEmbedding

/-!
# Homeomorphisms
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Topology/MetricSpace/ProperSpace.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: Sébastien Gouëzel
-/

import Mathlib.Topology.Order.IsLUB
import Mathlib.Topology.Support
import Mathlib.Topology.Algebra.Support
import Mathlib.Topology.MetricSpace.Pseudo.Basic
import Mathlib.Topology.MetricSpace.Pseudo.Lemmas
import Mathlib.Topology.MetricSpace.Pseudo.Pi
import Mathlib.Topology.Order.IsLUB

/-! ## Proper spaces
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Topology/Order/Compact.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,10 +3,10 @@ Copyright (c) 2021 Patrick Massot. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Patrick Massot, Yury Kudryashov
-/
import Mathlib.Topology.Order.LocalExtr
import Mathlib.Topology.Algebra.Support
import Mathlib.Topology.Order.IntermediateValue
import Mathlib.Topology.Support
import Mathlib.Topology.Order.IsLUB
import Mathlib.Topology.Order.LocalExtr

/-!
# Compactness of a closed interval
Expand Down
4 changes: 2 additions & 2 deletions Mathlib/Topology/UniformSpace/HeineCantor.lean
Original file line number Diff line number Diff line change
Expand Up @@ -3,9 +3,9 @@ Copyright (c) 2020 Patrick Massot. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Patrick Massot, Yury Kudryashov
-/
import Mathlib.Topology.UniformSpace.Equicontinuity
import Mathlib.Topology.Algebra.Support
import Mathlib.Topology.UniformSpace.Compact
import Mathlib.Topology.Support
import Mathlib.Topology.UniformSpace.Equicontinuity

/-!
# Compact separated uniform spaces
Expand Down

0 comments on commit 2aefce6

Please sign in to comment.