Documentation

Mathlib.Algebra.Category.CoalgebraCat.Basic

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.

structure CoalgebraCat (R : Type u) [CommRing R] extends ModuleCat R :
Type (max u (v + 1))

The category of R-coalgebras.

Instances For
    @[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
    Instances For
      structure CoalgebraCat.Hom {R : Type u} [CommRing R] (V W : CoalgebraCat R) :

      A type alias for CoalgHom to avoid confusion between the categorical and algebraic spellings of composition.

      Instances For
        theorem CoalgebraCat.Hom.ext {R : Type u} {inst✝ : CommRing R} {V W : CoalgebraCat R} {x y : V.Hom W} (toCoalgHom' : x.toCoalgHom' = y.toCoalgHom') :
        x = y
        Equations
        • One or more equations did not get rendered due to their size.
        @[reducible, inline]
        abbrev CoalgebraCat.Hom.toCoalgHom {R : Type u} [CommRing R] {X Y : CoalgebraCat R} (f : X.Hom Y) :

        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) :
          of R X of 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) :
            f = g
            Equations
            • One or more equations did not get rendered due to their size.

            Build an isomorphism in the category CoalgebraCat R from a CoalgEquiv.

            Equations
            Instances For

              Build a CoalgEquiv from an isomorphism in the category CoalgebraCat R.

              Equations
              Instances For
                @[simp]