(Unoriented) bordism theory #
This file defines the beginnings of unoriented bordism theory. We define singular manifolds, the building blocks of unoriented bordism groups. Future pull requests will define bordisms and the bordism groups of a topological space, and prove these are abelian groups.
The basic notion of bordism theory is that of a bordism between smooth manifolds.
Two compact smooth n
-dimensional manifolds M
and N
are bordant if there exists a smooth
bordism between them: this is a compact n+1
-dimensional manifold W
whose boundary is
(diffeomorphic to) the disjoint union M ⊕ N
. Being bordant is an equivalence relation
(transitivity follows from the collar neighbourhood theorem). The set of equivalence classes has an
abelian group structure, with the group operation given as disjoint union of manifolds,
and is called the n
-th (unoriented) bordism group.
This construction can be generalised one step further, to produce an extraordinary homology theory.
Given a topological space X
, a singular manifold on X
is a closed smooth manifold M
together with a continuous map M → F
. (The word singular does not refer to singularities,
but is by analogy to singular chains in the definition of singular homology.)
Given two n
-dimensional singular manifolds s
and t
, an (oriented) bordism between s
and t
is a compact smooth n+1
-dimensional manifold W
whose boundary is (diffeomorphic to) the disjoint
union of s
and t
, together with a map W → X
which restricts to the maps on s
and t
.
We call s
and t
bordant if there exists a bordism between them: again, this defines an
equivalence relation. The n
-th bordism group of X
is the set of bordism classes of
n
-dimensional singular manifolds on X
. If X
is a single point, this recovers the bordism
groups from the preceding paragraph.
These absolute bordism groups can be generalised further to relative bordism groups, for each
topological pair (X, A)
; in fact, these define an extra-ordinary homology theory.
Main definitions #
- SingularManifold X k I: a singular manifold on a topological space
X
, is a pair(M, f)
of a closedC^k
-manifold manifoldM
modelled onI
together with a continuous mapM → X
. We don't assumeM
to be modelled onℝⁿ
, but add the model topological spaceH
, the vector spaceE
and the model with cornersI
as type parameters. If we wish to emphasize the model, with will speak of a singularI
-manifold. To define a disjoint unions of singular manifolds, we require their domains to be manifolds over the same model with corners: this is why we make the model explicit.
Main results #
SingularManifold.map
: a mapX → Y
of topological spaces induces a map between the spaces of singular manifolds. This will be used to define functoriality of bordism groups.SingularManifold.comap
: if(N, f)
is a singular manifold onX
andφ : M → N
is continuous, thecomap
of(N, f)
andφ
is the induced singular manifold(M, f ∘ φ)
onX
.SingularManifold.empty
: the empty setM
, viewed as a manifold, as a singular manifold over any spaceX
.SingularManifold.toPUnit
: a smooth manifold induces a singular manifold on the one-point space.SingularManifold.prod
: the product of a singularI
-manifold and a singularJ
-manifold on the one-point space, is a singularI.prod J
-manifold on the one-point space.SingularManifold.sum
: the disjoint union of two singularI
-manifolds is a singularI
-manifold.
Implementation notes #
- We choose a bundled design for singular manifolds (and also for bordisms): to construct the group structure on the set of bordism classes, having that be a type is useful.
- The underlying model with corners is a type parameter, as defining a disjoint union of singular
manifolds requires their domains to be manifolds over the same model with corners.
Thus, either we restrict to manifolds modelled over
𝓡n
(which we prefer not to), or the model must be a type parameter. - Having
SingularManifold
contain the typeM
as explicit structure field is not ideal, as this adds a universe parameter to the structure. However, this is the best solution we found: we generally cannot haveM
live in the same universe asX
(a common case isX
beingPUnit
), and determining the universe ofM
from the universes ofE
andH
would makeSingularManifold.map
painful to state (as that would requireULift
ingM
).
TODO #
- define bordisms and prove basic constructions (e.g. reflexivity, symmetry, transitivity) and operations (e.g. disjoint union, sum with the empty set)
- define the bordism relation and prove it is an equivalence relation
- define the unoriented bordism group (the set of bordism classes) and prove it is an abelian group
- for bordisms on a one-point space, define multiplication and prove the bordism ring structure
- define relative bordism groups (generalising the previous three points)
- prove that relative unoriented bordism groups define an extraordinary homology theory
Tags #
singular manifold, bordism, bordism group
A singular manifold on a topological space X
is a pair (M, f)
of a closed
C^k
-manifold manifold M
modelled on I
together with a continuous map M → X
.
If we wish to emphasize the model, with will speak of a singular I
-manifold.
In practice, one commonly wants to take k=∞
(as then e.g. the intersection form is a powerful tool
to compute bordism groups; for the definition, this makes no difference.)
This is parametrised on the universe M
lives in; ensure u
is the first universe argument.
- M : Type u
The manifold
M
of a singularn
-manifold(M, f)
- topSpaceM : TopologicalSpace self.M
The manifold
M
is a topological space. - chartedSpace : ChartedSpace H self.M
The manifold
M
is a charted space overH
. - isManifold : IsManifold I k self.M
M
is aC^k
manifold. - compactSpace : CompactSpace self.M
- boundaryless : BoundarylessManifold I self.M
- f : self.M → X
The underlying map
M → X
of a singularn
-manifold(M, f)
onX
- hf : Continuous self.f
Instances For
Equations
Equations
A map of topological spaces induces a corresponding map of singular manifolds.
Equations
Instances For
If M
is a closd C^k
manifold, it is a singular manifold over itself.
Equations
- SingularManifold.refl M I = { M := M, topSpaceM := inst✝⁴, chartedSpace := inst✝³, isManifold := inst✝², compactSpace := inst✝¹, boundaryless := inst✝, f := id, hf := ⋯ }
Instances For
If (N, f)
is a singular manifold on X
and M
another C^k
manifold,
a continuous map φ : M → N
induces a singular manifold structure (M, f ∘ φ)
on X
.
Equations
Instances For
The canonical singular manifold associated to the empty set (seen as a smooth manifold)
Equations
- SingularManifold.empty X M I = { M := M, topSpaceM := inst✝³, chartedSpace := inst✝², isManifold := inst✝¹, compactSpace := ⋯, boundaryless := ⋯, f := fun (x : M) => ⋯.elim, hf := ⋯ }
Instances For
A smooth manifold induces a singular manifold on the one-point space.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The product of a singular I
- and a singular J
-manifold into a one-point space
is a singular I.prod J
-manifold.
This construction is used to prove that the bordism group of PUnit
is a graded commutative ring.
NB. This definition as written makes sense more generally, for SingularManifold X k I
whenever X
is a topological (additive) group. However, this would not be the correct definition if X
is not
(P)Unit
: the bordism ring can be defined for every C^k
manifold X
, but the product of two
singular manifolds (M, f)
and (N, g)
is the fibre product of M
and N
w.r.t. f
and g
,
with its induced map into X
.
(If f
and g
intersect transversely, this fibre product is a smooth manifold, of dimension
dim M + dim N - dim X
. Otherwise, the transversality theorem proves that f
(or g
) admits an
arbitrarily small perturbation f'
so f'
and g
are transverse. One can prove that different
perturbations yield bordant manifolds.)
Equations
- One or more equations did not get rendered due to their size.
Instances For
The disjoint union of two singular I
-manifolds on X
is a singular I
-manifold on X
.