The category of coalgebras over a commutative ring #
We introduce the bundled category CoalgebraCat
of coalgebras over a fixed commutative ring R
along with the forgetful functor to ModuleCat
.
This file mimics Mathlib.LinearAlgebra.QuadraticForm.QuadraticModuleCat
.
The category of R
-coalgebras.
- isAddCommGroup : AddCommGroup ↑self.toModuleCat
- isModule : Module R ↑self.toModuleCat
- instCoalgebra : Coalgebra R ↑self.toModuleCat
Instances For
Equations
- CoalgebraCat.instCoeSortType = { coe := fun (x : CoalgebraCat R) => ↑x.toModuleCat }
@[simp]
@[reducible, inline]
abbrev
CoalgebraCat.of
(R : Type u)
[CommRing R]
(X : Type v)
[AddCommGroup X]
[Module R X]
[Coalgebra R X]
:
The object in the category of R
-coalgebras associated to an R
-coalgebra.
Equations
- CoalgebraCat.of R X = { toModuleCat := ModuleCat.of R X, instCoalgebra := inferInstance }
Instances For
@[simp]
theorem
CoalgebraCat.of_comul
{R : Type u}
[CommRing R]
{X : Type v}
[AddCommGroup X]
[Module R X]
[Coalgebra R X]
:
@[simp]
theorem
CoalgebraCat.of_counit
{R : Type u}
[CommRing R]
{X : Type v}
[AddCommGroup X]
[Module R X]
[Coalgebra R X]
:
theorem
CoalgebraCat.Hom.ext
{R : Type u}
{inst✝ : CommRing R}
{V W : CoalgebraCat R}
{x y : V.Hom W}
(toCoalgHom' : x.toCoalgHom' = y.toCoalgHom')
:
Equations
instance
CoalgebraCat.concreteCategory
{R : Type u}
[CommRing R]
:
CategoryTheory.ConcreteCategory (CoalgebraCat R) fun (x1 x2 : CoalgebraCat R) => ↑x1.toModuleCat →ₗc[R] ↑x2.toModuleCat
Equations
- One or more equations did not get rendered due to their size.
@[reducible, inline]
Turn a morphism in CoalgebraCat
back into a CoalgHom
.
Equations
Instances For
@[reducible, inline]
abbrev
CoalgebraCat.ofHom
{R : Type u}
[CommRing R]
{X Y : Type v}
[AddCommGroup X]
[Module R X]
[AddCommGroup Y]
[Module R Y]
[Coalgebra R X]
[Coalgebra R Y]
(f : X →ₗc[R] Y)
:
Typecheck a CoalgHom
as a morphism in CoalgebraCat R
.
Equations
Instances For
theorem
CoalgebraCat.hom_ext
{R : Type u}
[CommRing R]
{M N : CoalgebraCat R}
(f g : M ⟶ N)
(h : Hom.toCoalgHom f = Hom.toCoalgHom g)
:
@[simp]
theorem
CoalgebraCat.toCoalgHom_comp
{R : Type u}
[CommRing R]
{M N U : CoalgebraCat R}
(f : M ⟶ N)
(g : N ⟶ U)
:
@[simp]
Equations
- One or more equations did not get rendered due to their size.
@[simp]
@[simp]
def
CoalgEquiv.toCoalgebraCatIso
{R : Type u}
[CommRing R]
{X Y : Type v}
[AddCommGroup X]
[Module R X]
[AddCommGroup Y]
[Module R Y]
[Coalgebra R X]
[Coalgebra R Y]
(e : X ≃ₗc[R] Y)
:
Build an isomorphism in the category CoalgebraCat R
from a
CoalgEquiv
.
Equations
- e.toCoalgebraCatIso = { hom := CoalgebraCat.ofHom ↑e, inv := CoalgebraCat.ofHom ↑e.symm, hom_inv_id := ⋯, inv_hom_id := ⋯ }
Instances For
@[simp]
theorem
CoalgEquiv.toCoalgebraCatIso_inv
{R : Type u}
[CommRing R]
{X Y : Type v}
[AddCommGroup X]
[Module R X]
[AddCommGroup Y]
[Module R Y]
[Coalgebra R X]
[Coalgebra R Y]
(e : X ≃ₗc[R] Y)
:
@[simp]
theorem
CoalgEquiv.toCoalgebraCatIso_hom
{R : Type u}
[CommRing R]
{X Y : Type v}
[AddCommGroup X]
[Module R X]
[AddCommGroup Y]
[Module R Y]
[Coalgebra R X]
[Coalgebra R Y]
(e : X ≃ₗc[R] Y)
:
@[simp]
theorem
CoalgEquiv.toCoalgebraCatIso_refl
{R : Type u}
[CommRing R]
{X : Type v}
[AddCommGroup X]
[Module R X]
[Coalgebra R X]
:
@[simp]
theorem
CoalgEquiv.toCoalgebraCatIso_symm
{R : Type u}
[CommRing R]
{X Y : Type v}
[AddCommGroup X]
[Module R X]
[AddCommGroup Y]
[Module R Y]
[Coalgebra R X]
[Coalgebra R Y]
(e : X ≃ₗc[R] Y)
:
@[simp]
theorem
CoalgEquiv.toCoalgebraCatIso_trans
{R : Type u}
[CommRing R]
{X Y Z : Type v}
[AddCommGroup X]
[Module R X]
[AddCommGroup Y]
[Module R Y]
[AddCommGroup Z]
[Module R Z]
[Coalgebra R X]
[Coalgebra R Y]
[Coalgebra R Z]
(e : X ≃ₗc[R] Y)
(f : Y ≃ₗc[R] Z)
:
Build a CoalgEquiv
from an isomorphism in the category
CoalgebraCat R
.
Equations
- i.toCoalgEquiv = { toCoalgHom := CoalgebraCat.Hom.toCoalgHom i.hom, invFun := ⇑(CoalgebraCat.Hom.toCoalgHom i.inv), left_inv := ⋯, right_inv := ⋯ }
Instances For
@[simp]
theorem
CategoryTheory.Iso.toCoalgEquiv_toCoalgHom
{R : Type u}
[CommRing R]
{X Y : CoalgebraCat R}
(i : X ≅ Y)
:
@[simp]
@[simp]
theorem
CategoryTheory.Iso.toCoalgEquiv_symm
{R : Type u}
[CommRing R]
{X Y : CoalgebraCat R}
(e : X ≅ Y)
:
@[simp]
theorem
CategoryTheory.Iso.toCoalgEquiv_trans
{R : Type u}
[CommRing R]
{X Y Z : CoalgebraCat R}
(e : X ≅ Y)
(f : Y ≅ Z)
: