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.
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
.
- ι : Type w
the index type of the cells
- π : self.ι → α
for each
i : ι
, we shall attach a cell given by the morphismg (π i)
. - cofan₁ : CategoryTheory.Limits.Cofan fun (i : self.ι) => A (self.π i)
a colimit cofan which gives the coproduct of the object
A (π i)
- cofan₂ : CategoryTheory.Limits.Cofan fun (i : self.ι) => B (self.π i)
a colimit cofan which gives the coproduct of the object
B (π i)
- isColimit₁ : CategoryTheory.Limits.IsColimit self.cofan₁
cofan₁
is colimit - isColimit₂ : CategoryTheory.Limits.IsColimit self.cofan₂
cofan₂
is colimit the coproduct of the maps
g (π i) : A (π i) ⟶ B (π i)
for alli : ι
.- hm (i : self.ι) : CategoryTheory.CategoryStruct.comp (self.cofan₁.inj i) self.m = CategoryTheory.CategoryStruct.comp (g (self.π i)) (self.cofan₂.inj i)
the top morphism of the pushout square
the bottom morphism of the pushout square
- isPushout : CategoryTheory.IsPushout self.g₁ self.m f self.g₂
Instances For
The inclusion of a cell.
Instances For
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
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
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.