Category instances for Monoid
, AddMonoid
, CommMonoid
, and AddCommMmonoid
. #
We introduce the bundled categories:
MonCat
AddMonCat
CommMonCat
AddCommMonCat
along with the relevant forgetful functors between them.
Equations
- Eq MonCat.instCoeSortType { coe := MonCat.carrier }
Instances For
Equations
- Eq AddMonCat.instCoeSortType { coe := AddMonCat.carrier }
Instances For
Construct a bundled AddMonCat
from the underlying type and typeclass.
Equations
- Eq (AddMonCat.of M) { carrier := M, str := inst✝ }
Instances For
The type of morphisms in AddMonCat R
.
- hom' : AddMonoidHom A.carrier B.carrier
The underlying monoid homomorphism.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Typecheck a MonoidHom
as a morphism in MonCat
.
Equations
Instances For
Typecheck an AddMonoidHom
as a morphism in AddMonCat
.
Equations
Instances For
The results below duplicate the ConcreteCategory
simp lemmas, but we can keep them for dsimp
.
Equations
- Eq MonCat.instInhabited { default := MonCat.of PUnit }
Instances For
Equations
- Eq AddMonCat.instInhabited { default := AddMonCat.of PUnit }
Instances For
Equations
- Eq (X.instOneHom Y) { one := MonCat.ofHom 1 }
Instances For
Equations
- Eq (X.instZeroHom Y) { zero := AddMonCat.ofHom 0 }
Instances For
Universe lift functor for monoids.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Universe lift functor for additive monoids.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The category of additive groups and group morphisms.
- carrier : Type u
The underlying type.
- str : AddCommMonoid self.carrier
Instances For
The category of groups and group morphisms.
- carrier : Type u
The underlying type.
- str : CommMonoid self.carrier
Instances For
Equations
- Eq CommMonCat.instCoeSortType { coe := CommMonCat.carrier }
Instances For
Equations
- Eq AddCommMonCat.instCoeSortType { coe := AddCommMonCat.carrier }
Instances For
Construct a bundled CommMonCat
from the underlying type and typeclass.
Equations
- Eq (CommMonCat.of M) { carrier := M, str := inst✝ }
Instances For
Construct a bundled AddCommMonCat
from the underlying type and typeclass.
Equations
- Eq (AddCommMonCat.of M) { carrier := M, str := inst✝ }
Instances For
The type of morphisms in AddCommMonCat R
.
- hom' : AddMonoidHom A.carrier B.carrier
The underlying monoid homomorphism.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Turn a morphism in AddCommMonCat
back into an AddMonoidHom
.
Equations
Instances For
Typecheck a MonoidHom
as a morphism in CommMonCat
.
Equations
Instances For
Typecheck an AddMonoidHom
as a morphism in AddCommMonCat
.
Equations
Instances For
Use the ConcreteCategory.hom
projection for @[simps]
lemmas.
Equations
- Eq (CommMonCat.Hom.Simps.hom X Y f) f.hom
Instances For
Use the ConcreteCategory.hom
projection for @[simps]
lemmas.
Equations
- Eq (AddCommMonCat.Hom.Simps.hom X Y f) f.hom
Instances For
The results below duplicate the ConcreteCategory
simp lemmas, but we can keep them for dsimp
.
Equations
- Eq CommMonCat.instInhabited { default := CommMonCat.of PUnit }
Instances For
Equations
- Eq AddCommMonCat.instInhabited { default := AddCommMonCat.of PUnit }
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Instances For
Equations
- Eq CommMonCat.instCoeMonCat { coe := (CategoryTheory.forget₂ CommMonCat MonCat).obj }
Instances For
Equations
Instances For
Universe lift functor for commutative monoids.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Universe lift functor for additive commutative monoids.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Build an isomorphism in the category MonCat
from a MulEquiv
between Monoid
s.
Equations
- Eq e.toMonCatIso { hom := MonCat.ofHom e.toMonoidHom, inv := MonCat.ofHom e.symm.toMonoidHom, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
Build an isomorphism in the category AddMonCat
from
an AddEquiv
between AddMonoid
s.
Equations
- Eq e.toAddMonCatIso { hom := AddMonCat.ofHom e.toAddMonoidHom, inv := AddMonCat.ofHom e.symm.toAddMonoidHom, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
Build an isomorphism in the category CommMonCat
from a MulEquiv
between CommMonoid
s.
Equations
- Eq e.toCommMonCatIso { hom := CommMonCat.ofHom e.toMonoidHom, inv := CommMonCat.ofHom e.symm.toMonoidHom, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
Build an isomorphism in the category AddCommMonCat
from an AddEquiv
between AddCommMonoid
s.
Equations
- Eq e.toAddCommMonCatIso { hom := AddCommMonCat.ofHom e.toAddMonoidHom, inv := AddCommMonCat.ofHom e.symm.toAddMonoidHom, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
Build a MulEquiv
from an isomorphism in the category MonCat
.
Equations
- Eq i.monCatIsoToMulEquiv ((MonCat.Hom.hom i.hom).toMulEquiv (MonCat.Hom.hom i.inv) ⋯ ⋯)
Instances For
Build an AddEquiv
from an isomorphism in the category
AddMonCat
.
Equations
- Eq i.addMonCatIsoToAddEquiv ((AddMonCat.Hom.hom i.hom).toAddEquiv (AddMonCat.Hom.hom i.inv) ⋯ ⋯)
Instances For
Build a MulEquiv
from an isomorphism in the category CommMonCat
.
Equations
- Eq i.commMonCatIsoToMulEquiv ((CommMonCat.Hom.hom i.hom).toMulEquiv (CommMonCat.Hom.hom i.inv) ⋯ ⋯)
Instances For
Build an AddEquiv
from an isomorphism in the category
AddCommMonCat
.
Equations
- Eq i.commMonCatIsoToAddEquiv ((AddCommMonCat.Hom.hom i.hom).toAddEquiv (AddCommMonCat.Hom.hom i.inv) ⋯ ⋯)
Instances For
multiplicative equivalences between Monoid
s are the same as (isomorphic to) isomorphisms
in MonCat
Equations
- One or more equations did not get rendered due to their size.
Instances For
additive equivalences between AddMonoid
s are the same
as (isomorphic to) isomorphisms in AddMonCat
Equations
- One or more equations did not get rendered due to their size.
Instances For
multiplicative equivalences between CommMonoid
s are the same as (isomorphic to) isomorphisms
in CommMonCat
Equations
- One or more equations did not get rendered due to their size.
Instances For
additive equivalences between AddCommMonoid
s are
the same as (isomorphic to) isomorphisms in AddCommMonCat
Equations
- One or more equations did not get rendered due to their size.
Instances For
Ensure that forget₂ CommMonCat MonCat
automatically reflects isomorphisms.
We could have used CategoryTheory.HasForget.ReflectsIso
alternatively.
@[simp]
lemmas for MonoidHom.comp
and categorical identities.
The equivalence between AddCommMonCat
and CommMonCat
.
Equations
- One or more equations did not get rendered due to their size.