Skip to content

Commit 4b14586

Browse files
grunwegplp127
andcommitted
chore(Topology/Homeomorph): split out the basic definitions (#22681)
Move `Homeomorph.lean` to `Homeomorph/Lemmas.lean`, and split out a new file `Homeomorph/Defs.lean` which contains just the basic definitions and properties. The definitions file intentionally has very minimal imports. All declarations which require heavier imports are kept in `Lemmas.lean`: this can be split in future commits. Future PRs will build on this split to dissolve `Homeomorph/Lemmas.lean` further, such as by moving the homeomorphism about direct sums next to their construction. This is also necessary to break an import cycle in #22137. This PR gives a modest import reduction - but is a pre-requisite to more far-reaching reductions by dissolving `Homeomorph/Lemmas.lean`. Co-authored-by: Aaron Liu <aaronliu2008@outlook.com>
1 parent 6715e25 commit 4b14586

28 files changed

+442
-401
lines changed

Mathlib.lean

Lines changed: 2 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -5767,7 +5767,8 @@ import Mathlib.Topology.Gluing
57675767
import Mathlib.Topology.Hom.ContinuousEval
57685768
import Mathlib.Topology.Hom.ContinuousEvalConst
57695769
import Mathlib.Topology.Hom.Open
5770-
import Mathlib.Topology.Homeomorph
5770+
import Mathlib.Topology.Homeomorph.Defs
5771+
import Mathlib.Topology.Homeomorph.Lemmas
57715772
import Mathlib.Topology.Homotopy.Basic
57725773
import Mathlib.Topology.Homotopy.Contractible
57735774
import Mathlib.Topology.Homotopy.Equiv

Mathlib/Topology/Algebra/ConstMulAction.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -10,7 +10,7 @@ import Mathlib.GroupTheory.GroupAction.Defs
1010
import Mathlib.Topology.Algebra.Constructions
1111
import Mathlib.Topology.Algebra.Support
1212
import Mathlib.Topology.Bases
13-
import Mathlib.Topology.Homeomorph
13+
import Mathlib.Topology.Homeomorph.Lemmas
1414

1515
/-!
1616
# Monoid actions continuous in the second variable

Mathlib/Topology/Algebra/Constructions.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@ Copyright (c) 2021 Nicolò Cavalleri. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Nicolò Cavalleri
55
-/
6-
import Mathlib.Topology.Homeomorph
6+
import Mathlib.Topology.Homeomorph.Lemmas
77

88
/-!
99
# Topological space structure on the opposite monoid and on the units group

Mathlib/Topology/Algebra/Constructions/DomMulAct.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@ Copyright (c) 2024 Yury Kudryashov. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Yury Kudryashov
55
-/
6-
import Mathlib.Topology.Homeomorph
6+
import Mathlib.Topology.Homeomorph.Lemmas
77
import Mathlib.GroupTheory.GroupAction.DomAct.Basic
88

99
/-!

Mathlib/Topology/Algebra/GroupWithZero.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -6,7 +6,7 @@ Authors: Yury Kudryashov
66
import Mathlib.Algebra.Group.Pi.Lemmas
77
import Mathlib.Algebra.GroupWithZero.Units.Equiv
88
import Mathlib.Topology.Algebra.Monoid
9-
import Mathlib.Topology.Homeomorph
9+
import Mathlib.Topology.Homeomorph.Lemmas
1010

1111
/-!
1212
# Topological group with zero

Mathlib/Topology/Algebra/Support.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -6,7 +6,7 @@ Authors: Floris van Doorn, Patrick Massot
66
import Mathlib.Algebra.GroupWithZero.Indicator
77
import Mathlib.Algebra.Module.Basic
88
import Mathlib.Algebra.Order.Group.Unbundled.Abs
9-
import Mathlib.Topology.Homeomorph
9+
import Mathlib.Topology.Homeomorph.Defs
1010
import Mathlib.Topology.Separation.Hausdorff
1111

1212
/-!

Mathlib/Topology/Category/TopCat/Limits/Products.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -9,6 +9,7 @@ import Mathlib.CategoryTheory.Limits.Shapes.Products
99
import Mathlib.CategoryTheory.Limits.ConcreteCategory.Basic
1010
import Mathlib.Data.Set.Subsingleton
1111
import Mathlib.Tactic.CategoryTheory.Elementwise
12+
import Mathlib.Topology.Homeomorph.Lemmas
1213

1314
/-!
1415
# Products and coproducts in the category of topological spaces

Mathlib/Topology/Category/TopCat/ULift.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Joël Riou
55
-/
66
import Mathlib.Topology.Category.TopCat.Basic
7+
import Mathlib.Topology.Homeomorph.Lemmas
78

89
/-!
910
# Lifting topological spaces to a higher universe

Mathlib/Topology/CompactOpen.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -5,6 +5,7 @@ Authors: Reid Barton
55
-/
66
import Mathlib.Topology.Hom.ContinuousEval
77
import Mathlib.Topology.ContinuousMap.Basic
8+
import Mathlib.Topology.Homeomorph.Lemmas
89

910
/-!
1011
# The compact-open topology

Mathlib/Topology/Compactification/OnePoint.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -4,6 +4,7 @@ Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Yourong Zang, Yury Kudryashov
55
-/
66
import Mathlib.Data.Fintype.Option
7+
import Mathlib.Topology.Homeomorph.Lemmas
78
import Mathlib.Topology.Sets.Opens
89

910
/-!

0 commit comments

Comments
 (0)