Documentation

Mathlib.Algebra.Category.CoalgCat.ComonEquivalence

The category equivalence between R-coalgebras and comonoid objects in R-Mod #

Given a commutative ring R, this file defines the equivalence of categories between R-coalgebras and comonoid objects in the category of R-modules.

We then use this to set up boilerplate for the Coalgebra instance on a tensor product of coalgebras defined in Mathlib.RingTheory.Coalgebra.TensorProduct.

Implementation notes #

We make the definition CoalgCat.instMonoidalCategoryAux in this file, which is the monoidal structure on CoalgCat induced by the equivalence with Comon(R-Mod). We use this to show the comultiplication and counit on a tensor product of coalgebras satisfy the coalgebra axioms, but our actual MonoidalCategory instance on CoalgCat is constructed in Mathlib.Algebra.Category.CoalgCat.Monoidal to have better definitional equalities.

noncomputable def CoalgCat.toComonObj {R : Type u} [CommRing R] (X : CoalgCat R) :

An R-coalgebra is a comonoid object in the category of R-modules.

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

    The natural functor from R-coalgebras to comonoid objects in the category of R-modules.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      @[simp]
      theorem CoalgCat.toComon_obj (R : Type u) [CommRing R] (X : CoalgCat R) :
      @[simp]
      theorem CoalgCat.toComon_map_hom (R : Type u) [CommRing R] {X✝ Y✝ : CoalgCat R} (f : X✝ Y✝) :
      noncomputable instance CoalgCat.ofComonObjCoalgebraStruct {R : Type u} [CommRing R] (X : Comon_ (ModuleCat R)) :

      A comonoid object in the category of R-modules has a natural comultiplication and counit.

      Equations
      noncomputable def CoalgCat.ofComonObj {R : Type u} [CommRing R] (X : Comon_ (ModuleCat R)) :

      A comonoid object in the category of R-modules has a natural R-coalgebra structure.

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

        The natural functor from comonoid objects in the category of R-modules to R-coalgebras.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          noncomputable def CoalgCat.comonEquivalence (R : Type u) [CommRing R] :

          The natural category equivalence between R-coalgebras and comonoid objects in the category of R-modules.

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

            The monoidal category structure on the category of R-coalgebras induced by the equivalence with Comon(R-Mod). This is just an auxiliary definition; the MonoidalCategory instance we make in Mathlib.Algebra.Category.CoalgCat.Monoidal has better definitional equalities.

            Equations
            Instances For