Documentation

Mathlib.Topology.CWComplex.Abstract.Basic

CW-complexes #

This file defines (relative) CW-complexes.

Main definitions #

References #

@[reducible, inline]

For each n : ℕ, this is the family of morphisms which sends the unique element of Unit to diskBoundaryInclusion n : ∂𝔻 n ⟶ 𝔻 n.

Equations
Instances For
    @[reducible, inline]
    abbrev TopCat.RelativeCWComplex {X Y : TopCat} (f : X Y) :
    Type (u + 1)

    A relative CW-complex is a morphism f : X ⟶ Y equipped with data expressing that Y identifies to the colimit of a functor F : ℕ ⥤ TopCat with that F.obj 0 ≅ X and for any n : ℕ, F.obj (n + 1) is obtained from F.obj n by attaching n-disks.

    Equations
    Instances For
      @[reducible, inline]
      abbrev TopCat.CWComplex (X : TopCat) :
      Type (u + 1)

      A CW-complex is a topological space such that ⊥_ _ ⟶ X is a relative CW-complex.

      Equations
      Instances For