Documentation

Mathlib.Geometry.Manifold.Bordism

(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 #

Main results #

Implementation notes #

TODO #

Tags #

singular manifold, bordism, bordism group

structure SingularManifold (X : Type u_1) [TopologicalSpace X] (k : WithTop ℕ∞) {E : Type u_2} {H : Type u_3} [NormedAddCommGroup E] [NormedSpace E] [FiniteDimensional E] [TopologicalSpace H] (I : ModelWithCorners E H) :
Type (max (max (u + 1) u_1) u_3)

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.

Instances For
    noncomputable def SingularManifold.map {X : Type u_7} {Y : Type u_8} [TopologicalSpace X] [TopologicalSpace Y] {k : WithTop ℕ∞} {E : Type u_9} {H : Type u_10} [NormedAddCommGroup E] [NormedSpace E] [FiniteDimensional E] [TopologicalSpace H] {I : ModelWithCorners E H} (s : SingularManifold X k I) {φ : XY} ( : Continuous φ) :

    A map of topological spaces induces a corresponding map of singular manifolds.

    Equations
    Instances For
      @[simp]
      theorem SingularManifold.map_f {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] {k : WithTop ℕ∞} {E : Type u_4} {H : Type u_5} [NormedAddCommGroup E] [NormedSpace E] [FiniteDimensional E] [TopologicalSpace H] {I : ModelWithCorners E H} (s : SingularManifold X k I) {φ : XY} ( : Continuous φ) :
      (s.map ).f = φ s.f
      @[simp]
      theorem SingularManifold.map_M {X : Type u_1} {Y : Type u_2} [TopologicalSpace X] [TopologicalSpace Y] {k : WithTop ℕ∞} {E : Type u_4} {H : Type u_5} [NormedAddCommGroup E] [NormedSpace E] [FiniteDimensional E] [TopologicalSpace H] {I : ModelWithCorners E H} (s : SingularManifold X k I) {φ : XY} ( : Continuous φ) :
      (s.map ).M = s.M
      theorem SingularManifold.map_comp {X : Type u_1} {Y : Type u_2} {Z : Type u_3} [TopologicalSpace X] [TopologicalSpace Y] [TopologicalSpace Z] {k : WithTop ℕ∞} {E : Type u_4} {H : Type u_5} [NormedAddCommGroup E] [NormedSpace E] [FiniteDimensional E] [TopologicalSpace H] {I : ModelWithCorners E H} (s : SingularManifold X k I) {φ : XY} {ψ : YZ} ( : Continuous φ) ( : Continuous ψ) :
      ((s.map ).map ).f = (ψ φ) s.f

      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
        noncomputable def SingularManifold.comap {X : Type u_1} [TopologicalSpace X] {k : WithTop ℕ∞} {E : Type u_4} {H : Type u_5} {M : Type u_6} [NormedAddCommGroup E] [NormedSpace E] [FiniteDimensional E] [TopologicalSpace H] {I : ModelWithCorners E H} [TopologicalSpace M] [ChartedSpace H M] [IsManifold I k M] [CompactSpace M] [BoundarylessManifold I M] (s : SingularManifold X k I) {φ : Ms.M} ( : Continuous φ) :

        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
        • s.comap = { M := M, topSpaceM := inst✝⁴, chartedSpace := inst✝³, isManifold := inst✝², compactSpace := inst✝¹, boundaryless := inst✝, f := s.f φ, hf := }
        Instances For
          @[simp]
          theorem SingularManifold.comap_M {X : Type u_1} [TopologicalSpace X] {k : WithTop ℕ∞} {E : Type u_4} {H : Type u_5} {M : Type u_6} [NormedAddCommGroup E] [NormedSpace E] [FiniteDimensional E] [TopologicalSpace H] {I : ModelWithCorners E H} [TopologicalSpace M] [ChartedSpace H M] [IsManifold I k M] [CompactSpace M] [BoundarylessManifold I M] (s : SingularManifold X k I) {φ : Ms.M} ( : Continuous φ) :
          (s.comap ).M = M
          @[simp]
          theorem SingularManifold.comap_f {X : Type u_1} [TopologicalSpace X] {k : WithTop ℕ∞} {E : Type u_4} {H : Type u_5} {M : Type u_6} [NormedAddCommGroup E] [NormedSpace E] [FiniteDimensional E] [TopologicalSpace H] {I : ModelWithCorners E H} [TopologicalSpace M] [ChartedSpace H M] [IsManifold I k M] [CompactSpace M] [BoundarylessManifold I M] (s : SingularManifold X k I) {φ : Ms.M} ( : Continuous φ) :
          (s.comap ).f = s.f φ

          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
            @[simp]
            theorem SingularManifold.empty_M {X : Type u_1} [TopologicalSpace X] {k : WithTop ℕ∞} {E : Type u_4} {H : Type u_5} {M : Type u_6} [NormedAddCommGroup E] [NormedSpace E] [FiniteDimensional E] [TopologicalSpace H] {I : ModelWithCorners E H} [TopologicalSpace M] [ChartedSpace H M] [IsManifold I k M] [IsEmpty M] :
            (empty X M I).M = M

            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
                noncomputable def SingularManifold.sum {X : Type u_1} [TopologicalSpace X] {k : WithTop ℕ∞} {E : Type u_4} {H : Type u_5} [NormedAddCommGroup E] [NormedSpace E] [FiniteDimensional E] [TopologicalSpace H] {I : ModelWithCorners E H} (s : SingularManifold X k I) (t : SingularManifold X k I) :

                The disjoint union of two singular I-manifolds on X is a singular I-manifold on X.

                Equations
                Instances For
                  @[simp]
                  theorem SingularManifold.sum_M {X : Type u_1} [TopologicalSpace X] {k : WithTop ℕ∞} {E : Type u_4} {H : Type u_5} [NormedAddCommGroup E] [NormedSpace E] [FiniteDimensional E] [TopologicalSpace H] {I : ModelWithCorners E H} (s : SingularManifold X k I) (t : SingularManifold X k I) :
                  (s.sum t).M = (s.M t.M)
                  @[simp]