The category of bipointed types #
This defines Bipointed
, the category of bipointed types.
TODO #
Monoidal structure
Equations
- Bipointed.instCoeSortType = { coe := Bipointed.X }
@[reducible, inline]
Turns a bipointing into a bipointed type.
Equations
- Bipointed.of to_prod = { X := X, toProd := to_prod }
Instances For
Equations
- Bipointed.instInhabited = { default := Bipointed.of ((), ()) }
The identity morphism of X : Bipointed
.
Equations
- Bipointed.Hom.id X = { toFun := id, map_fst := ⋯, map_snd := ⋯ }
Instances For
Equations
- Bipointed.Hom.instInhabited X = { default := Bipointed.Hom.id X }
instance
Bipointed.instFunLikeHomSubtypeX
(X : Bipointed)
(Y : Bipointed)
:
FunLike (X.HomSubtype Y) X.X Y.X
Equations
- X.instFunLikeHomSubtypeX Y = { coe := fun (f : X.HomSubtype Y) => ↑f, coe_injective' := ⋯ }
Equations
- One or more equations did not get rendered due to their size.
Swaps the pointed elements of a bipointed type. Prod.swap
as a functor.
Equations
- One or more equations did not get rendered due to their size.
Instances For
BipointedToPointed_fst
is inverse to PointedToBipointed
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
theorem
pointedToBipointedCompBipointedToPointedFst_inv_app_toFun
(X : Pointed)
(a : ((CategoryTheory.Functor.id Pointed).obj X).X)
:
@[simp]
theorem
pointedToBipointedCompBipointedToPointedFst_hom_app_toFun
(X : Pointed)
(a : ((pointedToBipointed.comp bipointedToPointedFst).obj X).X)
:
BipointedToPointed_snd
is inverse to PointedToBipointed
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
theorem
pointedToBipointedCompBipointedToPointedSnd_hom_app_toFun
(X : Pointed)
(a : ((pointedToBipointed.comp bipointedToPointedSnd).obj X).X)
:
@[simp]
theorem
pointedToBipointedCompBipointedToPointedSnd_inv_app_toFun
(X : Pointed)
(a : ((CategoryTheory.Functor.id Pointed).obj X).X)
:
The free/forgetful adjunction between PointedToBipointed_fst
and BipointedToPointed_fst
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The free/forgetful adjunction between PointedToBipointed_snd
and BipointedToPointed_snd
.
Equations
- One or more equations did not get rendered due to their size.