Documentation

Mathlib.AlgebraicTopology.RelativeCellComplex.AttachCells

Attaching cells #

Given a family of morphisms g a : A a ⟶ B a and a morphism f : X₁ ⟶ X₂, we introduce a structure AttachCells g f which expresses that X₂ is obtained from X₁ by attaching cells of the form g a. It means that there is a pushout diagram of the form

⨿ i, A (π i) -----> X₁
  |                 |f
  v                 v
⨿ i, B (π i) -----> X₂

In other words, the morphism f is a pushout of coproducts of morphisms of the form g a : A a ⟶ B a, see nonempty_attachCells_iff.

See the file Mathlib.AlgebraicTopology.RelativeCellComplex.Basic for transfinite compositions of morphisms f with AttachCells g f structures.

structure HomotopicalAlgebra.AttachCells {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} (g : (a : α) → A a B a) {X₁ X₂ : C} (f : X₁ X₂) :
Type (max (max (max t u) v) (w + 1))

Given a family of morphisms g a : A a ⟶ B a and a morphism f : X₁ ⟶ X₂, this structure contains the data and properties which expresses that X₂ is obtained from X₁ by attaching cells of the form g a.

Instances For
    @[simp]
    theorem HomotopicalAlgebra.AttachCells.hm_assoc {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (self : AttachCells g f) (i : self.ι) {Z : C} (h : self.cofan₂.pt Z) :
    def HomotopicalAlgebra.AttachCells.cell {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) (i : c.ι) :
    B (c.π i) X₂

    The inclusion of a cell.

    Equations
    Instances For
      theorem HomotopicalAlgebra.AttachCells.cell_def {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) (i : c.ι) :
      theorem HomotopicalAlgebra.AttachCells.cell_def_assoc {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) (i : c.ι) {Z : C} (h : X₂ Z) :
      theorem HomotopicalAlgebra.AttachCells.hom_ext {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {Z : C} {φ φ' : X₂ Z} (h₀ : CategoryTheory.CategoryStruct.comp f φ = CategoryTheory.CategoryStruct.comp f φ') (h : ∀ (i : c.ι), CategoryTheory.CategoryStruct.comp (c.cell i) φ = CategoryTheory.CategoryStruct.comp (c.cell i) φ') :
      φ = φ'
      def HomotopicalAlgebra.AttachCells.ofArrowIso {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {Y₁ Y₂ : C} {f' : Y₁ Y₂} (e : CategoryTheory.Arrow.mk f CategoryTheory.Arrow.mk f') :

      If f and f' are isomorphic morphisms and the target of f is obtained by attaching cells to the source of f, then the same holds for f'.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[simp]
        theorem HomotopicalAlgebra.AttachCells.ofArrowIso_m {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {Y₁ Y₂ : C} {f' : Y₁ Y₂} (e : CategoryTheory.Arrow.mk f CategoryTheory.Arrow.mk f') :
        (c.ofArrowIso e).m = c.m
        @[simp]
        theorem HomotopicalAlgebra.AttachCells.ofArrowIso_cofan₁ {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {Y₁ Y₂ : C} {f' : Y₁ Y₂} (e : CategoryTheory.Arrow.mk f CategoryTheory.Arrow.mk f') :
        @[simp]
        theorem HomotopicalAlgebra.AttachCells.ofArrowIso_ι {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {Y₁ Y₂ : C} {f' : Y₁ Y₂} (e : CategoryTheory.Arrow.mk f CategoryTheory.Arrow.mk f') :
        (c.ofArrowIso e).ι = c.ι
        @[simp]
        theorem HomotopicalAlgebra.AttachCells.ofArrowIso_isColimit₂ {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {Y₁ Y₂ : C} {f' : Y₁ Y₂} (e : CategoryTheory.Arrow.mk f CategoryTheory.Arrow.mk f') :
        @[simp]
        theorem HomotopicalAlgebra.AttachCells.ofArrowIso_isColimit₁ {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {Y₁ Y₂ : C} {f' : Y₁ Y₂} (e : CategoryTheory.Arrow.mk f CategoryTheory.Arrow.mk f') :
        @[simp]
        theorem HomotopicalAlgebra.AttachCells.ofArrowIso_g₂ {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {Y₁ Y₂ : C} {f' : Y₁ Y₂} (e : CategoryTheory.Arrow.mk f CategoryTheory.Arrow.mk f') :
        @[simp]
        theorem HomotopicalAlgebra.AttachCells.ofArrowIso_cofan₂ {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {Y₁ Y₂ : C} {f' : Y₁ Y₂} (e : CategoryTheory.Arrow.mk f CategoryTheory.Arrow.mk f') :
        @[simp]
        theorem HomotopicalAlgebra.AttachCells.ofArrowIso_g₁ {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {Y₁ Y₂ : C} {f' : Y₁ Y₂} (e : CategoryTheory.Arrow.mk f CategoryTheory.Arrow.mk f') :
        @[simp]
        theorem HomotopicalAlgebra.AttachCells.ofArrowIso_π {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {Y₁ Y₂ : C} {f' : Y₁ Y₂} (e : CategoryTheory.Arrow.mk f CategoryTheory.Arrow.mk f') (a✝ : c.ι) :
        (c.ofArrowIso e).π a✝ = c.π a✝
        def HomotopicalAlgebra.AttachCells.reindex {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {ι' : Type w'} (e : ι' c.ι) :

        This definition allows the replacement of the ι field of a AttachCells g f structure by an equivalent type.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          @[simp]
          theorem HomotopicalAlgebra.AttachCells.reindex_ι {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {ι' : Type w'} (e : ι' c.ι) :
          (c.reindex e).ι = ι'
          @[simp]
          theorem HomotopicalAlgebra.AttachCells.reindex_isColimit₁ {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {ι' : Type w'} (e : ι' c.ι) :
          @[simp]
          theorem HomotopicalAlgebra.AttachCells.reindex_cofan₁ {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {ι' : Type w'} (e : ι' c.ι) :
          @[simp]
          theorem HomotopicalAlgebra.AttachCells.reindex_g₂ {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {ι' : Type w'} (e : ι' c.ι) :
          (c.reindex e).g₂ = c.g₂
          @[simp]
          theorem HomotopicalAlgebra.AttachCells.reindex_isColimit₂ {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {ι' : Type w'} (e : ι' c.ι) :
          @[simp]
          theorem HomotopicalAlgebra.AttachCells.reindex_m {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {ι' : Type w'} (e : ι' c.ι) :
          (c.reindex e).m = c.m
          @[simp]
          theorem HomotopicalAlgebra.AttachCells.reindex_g₁ {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {ι' : Type w'} (e : ι' c.ι) :
          (c.reindex e).g₁ = c.g₁
          @[simp]
          theorem HomotopicalAlgebra.AttachCells.reindex_cofan₂ {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {ι' : Type w'} (e : ι' c.ι) :
          @[simp]
          theorem HomotopicalAlgebra.AttachCells.reindex_π {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {ι' : Type w'} (e : ι' c.ι) (i' : ι') :
          (c.reindex e).π i' = c.π (e i')
          def HomotopicalAlgebra.AttachCells.reindexCellTypes {C : Type u} [CategoryTheory.Category.{v, u} C] {α : Type t} {A B : αC} {g : (a : α) → A a B a} {X₁ X₂ : C} {f : X₁ X₂} (c : AttachCells g f) {α' : Type t'} {A' B' : α'C} (g' : (i' : α') → A' i' B' i') (a : αα') (ha : (i : α) → CategoryTheory.Arrow.mk (g i) CategoryTheory.Arrow.mk (g' (a i))) :

          If a family of maps g is contained in another family g' (up to isomorphisms), if f : X₁ ⟶ X₂ is a morphism, and X₂ is obtained from X₁ by attaching cells of the form g, then it is also obtained by attaching cells of the form g'.

          Equations
          • One or more equations did not get rendered due to their size.
          Instances For