Skip to content

Commit

Permalink
chore: move 2 files to a new folder (#6853)
Browse files Browse the repository at this point in the history
Later I'm going to split files like `Lipschitz` into 2: one in `EMetricSpace/`
and one in `MetricSpace/`.
  • Loading branch information
urkud committed Aug 31, 2023
1 parent bfb6bb7 commit dd781b4
Show file tree
Hide file tree
Showing 10 changed files with 10 additions and 10 deletions.
2 changes: 1 addition & 1 deletion Counterexamples/SorgenfreyLine.lean
Expand Up @@ -7,7 +7,7 @@ import Mathlib.Topology.Instances.Irrational
import Mathlib.Topology.Algebra.Order.Archimedean
import Mathlib.Topology.Paracompact
import Mathlib.Topology.MetricSpace.Metrizable
import Mathlib.Topology.MetricSpace.EMetricParacompact
import Mathlib.Topology.EMetricSpace.Paracompact
import Mathlib.Data.Set.Intervals.Monotone
import Mathlib.Topology.Separation.NotNormal

Expand Down
4 changes: 2 additions & 2 deletions Mathlib.lean
Expand Up @@ -3270,6 +3270,8 @@ import Mathlib.Topology.Covering
import Mathlib.Topology.DenseEmbedding
import Mathlib.Topology.DiscreteQuotient
import Mathlib.Topology.DiscreteSubset
import Mathlib.Topology.EMetricSpace.Basic
import Mathlib.Topology.EMetricSpace.Paracompact
import Mathlib.Topology.ExtendFrom
import Mathlib.Topology.ExtremallyDisconnected
import Mathlib.Topology.FiberBundle.Basic
Expand Down Expand Up @@ -3325,8 +3327,6 @@ import Mathlib.Topology.MetricSpace.Completion
import Mathlib.Topology.MetricSpace.Contracting
import Mathlib.Topology.MetricSpace.Dilation
import Mathlib.Topology.MetricSpace.DilationEquiv
import Mathlib.Topology.MetricSpace.EMetricParacompact
import Mathlib.Topology.MetricSpace.EMetricSpace
import Mathlib.Topology.MetricSpace.Equicontinuity
import Mathlib.Topology.MetricSpace.Gluing
import Mathlib.Topology.MetricSpace.GromovHausdorff
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Analysis/Fourier/RiemannLebesgueLemma.lean
Expand Up @@ -10,7 +10,7 @@ import Mathlib.MeasureTheory.Function.ContinuousMapDense
import Mathlib.MeasureTheory.Group.Integral
import Mathlib.MeasureTheory.Integral.SetIntegral
import Mathlib.MeasureTheory.Measure.Haar.NormedSpace
import Mathlib.Topology.MetricSpace.EMetricParacompact
import Mathlib.Topology.EMetricSpace.Paracompact

#align_import analysis.fourier.riemann_lebesgue_lemma from "leanprover-community/mathlib"@"fd5edc43dc4f10b85abfe544b88f82cf13c5f844"

Expand Down
File renamed without changes.
Expand Up @@ -5,7 +5,7 @@ Authors: Yury G. Kudryashov
-/
import Mathlib.SetTheory.Ordinal.Basic
import Mathlib.Tactic.GCongr
import Mathlib.Topology.MetricSpace.EMetricSpace
import Mathlib.Topology.EMetricSpace.Basic
import Mathlib.Topology.Paracompact

#align_import topology.metric_space.emetric_paracompact from "leanprover-community/mathlib"@"57ac39bd365c2f80589a700f9fbb664d3a1a30c2"
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Topology/MetricSpace/Basic.lean
Expand Up @@ -5,7 +5,7 @@ Authors: Jeremy Avigad, Robert Y. Lewis, Johannes Hölzl, Mario Carneiro, Sébas
-/
import Mathlib.Tactic.Positivity
import Mathlib.Topology.Algebra.Order.Compact
import Mathlib.Topology.MetricSpace.EMetricSpace
import Mathlib.Topology.EMetricSpace.Basic
import Mathlib.Topology.Bornology.Constructions

#align_import topology.metric_space.basic from "leanprover-community/mathlib"@"8047de4d911cdef39c2d646165eea972f7f9f539"
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Topology/MetricSpace/MetricSeparated.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2021 Yury Kudryashov. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yury Kudryashov
-/
import Mathlib.Topology.MetricSpace.EMetricSpace
import Mathlib.Topology.EMetricSpace.Basic

#align_import topology.metric_space.metric_separated from "leanprover-community/mathlib"@"57ac39bd365c2f80589a700f9fbb664d3a1a30c2"

Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Topology/MetricSpace/PartitionOfUnity.lean
Expand Up @@ -3,7 +3,7 @@ Copyright (c) 2022 Yury Kudryashov. All rights reserved.
Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yury Kudryashov
-/
import Mathlib.Topology.MetricSpace.EMetricParacompact
import Mathlib.Topology.EMetricSpace.Paracompact
import Mathlib.Analysis.Convex.PartitionOfUnity

#align_import topology.metric_space.partition_of_unity from "leanprover-community/mathlib"@"f2ce6086713c78a7f880485f7917ea547a215982"
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Topology/MetricSpace/ShrinkingLemma.lean
Expand Up @@ -4,7 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
Authors: Yury G. Kudryashov
-/
import Mathlib.Topology.MetricSpace.Basic
import Mathlib.Topology.MetricSpace.EMetricParacompact
import Mathlib.Topology.EMetricSpace.Paracompact
import Mathlib.Topology.ShrinkingLemma

#align_import topology.metric_space.shrinking_lemma from "leanprover-community/mathlib"@"f2ce6086713c78a7f880485f7917ea547a215982"
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/Topology/Paracompact.lean
Expand Up @@ -35,7 +35,7 @@ We also prove the following facts.
the instance graph.
* Every `EMetricSpace` is a paracompact space, see instance `EMetricSpace.ParacompactSpace` in
`Topology/MetricSpace/EMetricParacompact`.
`Topology/EMetricSpace/Paracompact`.
## TODO
Expand Down

0 comments on commit dd781b4

Please sign in to comment.