CW complexes #
This file defines (relative) CW complexes and proves basic properties about them.
A CW complex is a topological space that is made by gluing closed disks of different dimensions together.
Main definitions #
RelCWComplex C D
: the class of CW structures on a subspaceC
relative to a base setD
of a topological spaceX
.CWComplex C
: an abbreviation forRelCWComplex C ∅
. The class of CW structures on a subspaceC
of the topological spaceX
.openCell n
: indexed family of all open cells of dimensionn
.closedCell n
: indexed family of all closed cells of dimensionn
.cellFrontier n
: indexed family of the boundaries of cells of dimensionn
.skeleton C n
: then
-skeleton of the (relative) CW complexC
.
Main statements #
iUnion_openCell_eq_skeleton
: the skeletons can also be seen as a union of open cells.cellFrontier_subset_finite_openCell
: the edge of a cell is contained in a finite union of open cells of a lower dimension.
Implementation notes #
- We use the historical definition of CW complexes, due to Whitehead: a CW complex is a collection of cells with attaching maps - all cells are subspaces of one ambient topological space. This way, we avoid having to work with a lot of different topological spaces. On the other hand, it requires the union of all cells to be closed. If that is not the case, you need to consider that union as a subspace of itself.
- The definition
RelCWComplex
does not requireX
to be a Hausdorff space. A lot of the lemmas will however require this property. - This definition is a class to ease working with different constructions and their properties. Overall this means the being a CW complex is treated more like a property than data.
- For statements, the auxiliary construction
skeletonLT
is preferred overskeleton
as it makes the base case of inductions easier. The statement aboutskeleton
should then be derived from the one aboutskeletonLT
.
References #
A CW complex of a topological space X
relative to another subspace D
is the data of its
n
-cells cell n i
for each n : ℕ
along with attaching maps that satisfy a number of
properties with the most important being closure-finiteness (mapsTo
) and weak topology
(closed'
). Note that this definition requires C
and D
to be closed subspaces.
If C
is not closed choose X
to be C
.
The indexing type of the cells of dimension
n
.The characteristic map of the
n
-cell given by the indexi
. This map is a bijection when restricting toball 0 1
, where we consider(Fin n → ℝ)
endowed with the maximum metric.The source of every charactersitic map of dimension
n
is(ball 0 1 : Set (Fin n → ℝ))
.The characteristic maps are continuous when restricting to
closedBall 0 1
.The inverse of the restriction to
ball 0 1
is continuous on the image.- pairwiseDisjoint' : Set.univ.PairwiseDisjoint fun (ni : (n : ℕ) × cell C n) => ↑(map ni.fst ni.snd) '' Metric.ball 0 1
The open cells are pairwise disjoint. Use
RelCWComplex.pairwiseDisjoint
orRelCWComplex.disjoint_openCell_of_ne
instead. All open cells are disjoint with the base. Use
RelCWComplex.disjointBase
instead.- mapsTo (n : ℕ) (i : cell C n) : ∃ (I : (m : ℕ) → Finset (cell C m)), Set.MapsTo (↑(map n i)) (Metric.sphere 0 1) (D ∪ ⋃ (m : ℕ), ⋃ (_ : m < n), ⋃ j ∈ I m, ↑(map m j) '' Metric.closedBall 0 1)
The boundary of a cell is contained in a finite union of closed cells of a lower dimension. Use
RelCWComplex.cellFrontier_subset_finite_closedCell
instead. - closed' (A : Set X) (asubc : A ⊆ C) : (∀ (n : ℕ) (j : cell C n), IsClosed (A ∩ ↑(map n j) '' Metric.closedBall 0 1)) ∧ IsClosed (A ∩ D) → IsClosed A
A CW complex has weak topology, i.e. a set
A
inX
is closed iff its intersection with every closed cell andD
is closed. UseRelCWComplex.closed
instead. - isClosedBase : IsClosed D
The base
D
is closed. The union of all closed cells equals
C
. UseRelCWComplex.union
instead.
Instances
Alias of Topology.RelCWComplex.mapsTo
.
The boundary of a cell is contained in a finite union of closed cells of a lower dimension.
Use RelCWComplex.cellFrontier_subset_finite_closedCell
instead.
Characterizing when a subspace C
of a topological space X
is a CW complex. Note that this
requires C
to be closed. If C
is not closed choose X
to be C
.
Equations
Instances For
A constructor for CWComplex
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The open n
-cell given by the index i
. Use this instead of map n i '' ball 0 1
whenever
possible.
Equations
- Topology.RelCWComplex.openCell n i = ↑(Topology.RelCWComplex.map n i) '' Metric.ball 0 1
Instances For
The closed n
-cell given by the index i
. Use this instead of map n i '' closedBall 0 1
whenever possible.
Equations
Instances For
The boundary of the n
-cell given by the index i
. Use this instead of map n i '' sphere 0 1
whenever possible.
Equations
- Topology.RelCWComplex.cellFrontier n i = ↑(Topology.RelCWComplex.map n i) '' Metric.sphere 0 1
Instances For
Alias of Topology.CWComplex.mapsTo
.
A non-standard definition of the n
-skeleton of a CW complex for n ∈ ℕ ∪ {∞}
.
This allows the base case of induction to be about the base instead of being about the union of
the base and some points.
The standard skeleton
is defined in terms of skeletonLT
. skeletonLT
is preferred
in statements. You should then derive the statement about skeleton
.
Equations
- Topology.RelCWComplex.skeletonLT C n = D ∪ ⋃ (m : ℕ), ⋃ (_ : ↑m < n), ⋃ (j : Topology.RelCWComplex.cell C m), Topology.RelCWComplex.closedCell m j
Instances For
The n
-skeleton of a CW complex, for n ∈ ℕ ∪ {∞}
. For statements use skeletonLT
instead
and then derive the statement about skeleton
.