Documentation

Mathlib.Algebra.Category.MonCat.Basic

Category instances for Monoid, AddMonoid, CommMonoid, and AddCommMmonoid. #

We introduce the bundled categories:

structure AddMonCat :
Type (u + 1)

The category of additive groups and group morphisms.

Instances For
    structure MonCat :
    Type (u + 1)

    The category of groups and group morphisms.

    Instances For
      @[reducible, inline]
      abbrev MonCat.of (M : Type u) [Monoid M] :

      Construct a bundled MonCat from the underlying type and typeclass.

      Equations
      Instances For
        @[reducible, inline]
        abbrev AddMonCat.of (M : Type u) [AddMonoid M] :

        Construct a bundled AddMonCat from the underlying type and typeclass.

        Equations
        Instances For
          structure AddMonCat.Hom (A B : AddMonCat) :

          The type of morphisms in AddMonCat R.

          Instances For
            theorem AddMonCat.Hom.ext {A B : AddMonCat} {x y : A.Hom B} (hom' : Eq x.hom' y.hom') :
            Eq x y
            theorem AddMonCat.Hom.ext_iff {A B : AddMonCat} {x y : A.Hom B} :
            Iff (Eq x y) (Eq x.hom' y.hom')
            structure MonCat.Hom (A B : MonCat) :

            The type of morphisms in MonCat R.

            Instances For
              theorem MonCat.Hom.ext_iff {A B : MonCat} {x y : A.Hom B} :
              Iff (Eq x y) (Eq x.hom' y.hom')
              theorem MonCat.Hom.ext {A B : MonCat} {x y : A.Hom B} (hom' : Eq x.hom' y.hom') :
              Eq x y
              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
                      @[reducible, inline]
                      abbrev MonCat.Hom.hom {X Y : MonCat} (f : X.Hom Y) :

                      Turn a morphism in MonCat back into a MonoidHom.

                      Equations
                      Instances For
                        @[reducible, inline]

                        Turn a morphism in AddMonCat back into an AddMonoidHom.

                        Equations
                        Instances For
                          @[reducible, inline]
                          abbrev MonCat.ofHom {X Y : Type u} [Monoid X] [Monoid Y] (f : MonoidHom X Y) :
                          Quiver.Hom (of X) (of Y)

                          Typecheck a MonoidHom as a morphism in MonCat.

                          Equations
                          Instances For
                            @[reducible, inline]
                            abbrev AddMonCat.ofHom {X Y : Type u} [AddMonoid X] [AddMonoid Y] (f : AddMonoidHom X Y) :
                            Quiver.Hom (of X) (of Y)

                            Typecheck an AddMonoidHom as a morphism in AddMonCat.

                            Equations
                            Instances For

                              Use the ConcreteCategory.hom projection for @[simps] lemmas.

                              Equations
                              Instances For

                                The results below duplicate the ConcreteCategory simp lemmas, but we can keep them for dsimp.

                                theorem MonCat.coe_of (M : Type u) [Monoid M] :
                                Eq (of M).carrier M
                                theorem AddMonCat.coe_of (M : Type u) [AddMonoid M] :
                                Eq (of M).carrier M
                                theorem MonCat.hom_ext {M N : MonCat} {f g : Quiver.Hom M N} (hf : Eq (Hom.hom f) (Hom.hom g)) :
                                Eq f g
                                theorem AddMonCat.hom_ext {M N : AddMonCat} {f g : Quiver.Hom M N} (hf : Eq (Hom.hom f) (Hom.hom g)) :
                                Eq f g
                                theorem MonCat.hom_ext_iff {M N : MonCat} {f g : Quiver.Hom M N} :
                                Iff (Eq f g) (Eq (Hom.hom f) (Hom.hom g))
                                theorem AddMonCat.hom_ext_iff {M N : AddMonCat} {f g : Quiver.Hom M N} :
                                Iff (Eq f g) (Eq (Hom.hom f) (Hom.hom g))
                                theorem MonCat.hom_ofHom {M N : Type u} [Monoid M] [Monoid N] (f : MonoidHom M N) :
                                Eq (Hom.hom (ofHom f)) f
                                theorem AddMonCat.hom_ofHom {M N : Type u} [AddMonoid M] [AddMonoid N] (f : AddMonoidHom M N) :
                                Eq (Hom.hom (ofHom f)) f
                                theorem MonCat.ofHom_hom {M N : MonCat} (f : Quiver.Hom M N) :
                                Eq (ofHom (Hom.hom f)) f
                                theorem AddMonCat.ofHom_hom {M N : AddMonCat} (f : Quiver.Hom M N) :
                                Eq (ofHom (Hom.hom f)) f
                                theorem MonCat.ofHom_comp {M N P : Type u} [Monoid M] [Monoid N] [Monoid P] (f : MonoidHom M N) (g : MonoidHom N P) :
                                Equations
                                Instances For
                                  Equations
                                  Instances For
                                    theorem MonCat.hom_one (X Y : MonCat) :
                                    Eq (Hom.hom 1) 1
                                    theorem MonCat.oneHom_apply (X Y : MonCat) (x : X.carrier) :
                                    theorem MonCat.one_of {A : Type u_1} [Monoid A] :
                                    Eq 1 1
                                    theorem AddMonCat.zero_of {A : Type u_1} [AddMonoid A] :
                                    Eq 0 0
                                    theorem MonCat.mul_of {A : Type u_1} [Monoid A] (a b : A) :
                                    Eq (HMul.hMul a b) (HMul.hMul a b)
                                    theorem AddMonCat.add_of {A : Type u_1} [AddMonoid A] (a b : A) :
                                    Eq (HAdd.hAdd a b) (HAdd.hAdd a b)

                                    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
                                        structure AddCommMonCat :
                                        Type (u + 1)

                                        The category of additive groups and group morphisms.

                                        Instances For
                                          structure CommMonCat :
                                          Type (u + 1)

                                          The category of groups and group morphisms.

                                          Instances For
                                            @[reducible, inline]

                                            Construct a bundled CommMonCat from the underlying type and typeclass.

                                            Equations
                                            Instances For
                                              @[reducible, inline]

                                              Construct a bundled AddCommMonCat from the underlying type and typeclass.

                                              Equations
                                              Instances For
                                                structure AddCommMonCat.Hom (A B : AddCommMonCat) :

                                                The type of morphisms in AddCommMonCat R.

                                                Instances For
                                                  theorem AddCommMonCat.Hom.ext_iff {A B : AddCommMonCat} {x y : A.Hom B} :
                                                  Iff (Eq x y) (Eq x.hom' y.hom')
                                                  theorem AddCommMonCat.Hom.ext {A B : AddCommMonCat} {x y : A.Hom B} (hom' : Eq x.hom' y.hom') :
                                                  Eq x y
                                                  structure CommMonCat.Hom (A B : CommMonCat) :

                                                  The type of morphisms in CommMonCat R.

                                                  Instances For
                                                    theorem CommMonCat.Hom.ext_iff {A B : CommMonCat} {x y : A.Hom B} :
                                                    Iff (Eq x y) (Eq x.hom' y.hom')
                                                    theorem CommMonCat.Hom.ext {A B : CommMonCat} {x y : A.Hom B} (hom' : Eq x.hom' y.hom') :
                                                    Eq x y
                                                    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
                                                            @[reducible, inline]

                                                            Turn a morphism in CommMonCat back into a MonoidHom.

                                                            Equations
                                                            Instances For
                                                              @[reducible, inline]

                                                              Turn a morphism in AddCommMonCat back into an AddMonoidHom.

                                                              Equations
                                                              Instances For
                                                                @[reducible, inline]
                                                                abbrev CommMonCat.ofHom {X Y : Type u} [CommMonoid X] [CommMonoid Y] (f : MonoidHom X Y) :
                                                                Quiver.Hom (of X) (of Y)

                                                                Typecheck a MonoidHom as a morphism in CommMonCat.

                                                                Equations
                                                                Instances For
                                                                  @[reducible, inline]
                                                                  abbrev AddCommMonCat.ofHom {X Y : Type u} [AddCommMonoid X] [AddCommMonoid Y] (f : AddMonoidHom X Y) :
                                                                  Quiver.Hom (of X) (of Y)

                                                                  Typecheck an AddMonoidHom as a morphism in AddCommMonCat.

                                                                  Equations
                                                                  Instances For

                                                                    Use the ConcreteCategory.hom projection for @[simps] lemmas.

                                                                    Equations
                                                                    Instances For

                                                                      Use the ConcreteCategory.hom projection for @[simps] lemmas.

                                                                      Equations
                                                                      Instances For

                                                                        The results below duplicate the ConcreteCategory simp lemmas, but we can keep them for dsimp.

                                                                        theorem CommMonCat.hom_ext {M N : CommMonCat} {f g : Quiver.Hom M N} (hf : Eq (Hom.hom f) (Hom.hom g)) :
                                                                        Eq f g
                                                                        theorem AddCommMonCat.hom_ext {M N : AddCommMonCat} {f g : Quiver.Hom M N} (hf : Eq (Hom.hom f) (Hom.hom g)) :
                                                                        Eq f g
                                                                        theorem CommMonCat.hom_ext_iff {M N : CommMonCat} {f g : Quiver.Hom M N} :
                                                                        Iff (Eq f g) (Eq (Hom.hom f) (Hom.hom g))
                                                                        theorem AddCommMonCat.hom_ext_iff {M N : AddCommMonCat} {f g : Quiver.Hom M N} :
                                                                        Iff (Eq f g) (Eq (Hom.hom f) (Hom.hom g))
                                                                        theorem CommMonCat.hom_ofHom {M N : Type u} [CommMonoid M] [CommMonoid N] (f : MonoidHom M N) :
                                                                        Eq (Hom.hom (ofHom f)) f
                                                                        theorem CommMonCat.ofHom_hom {M N : CommMonCat} (f : Quiver.Hom M N) :
                                                                        Eq (ofHom (Hom.hom f)) f
                                                                        theorem CommMonCat.coe_of (R : Type u) [CommMonoid R] :
                                                                        Eq (of R).carrier R
                                                                        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

                                                                            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 Monoids.

                                                                                Equations
                                                                                Instances For

                                                                                  Build an isomorphism in the category AddMonCat from an AddEquiv between AddMonoids.

                                                                                  Equations
                                                                                  Instances For

                                                                                    Build an isomorphism in the category CommMonCat from a MulEquiv between CommMonoids.

                                                                                    Equations
                                                                                    Instances For

                                                                                      Build an isomorphism in the category AddCommMonCat from an AddEquiv between AddCommMonoids.

                                                                                      Equations
                                                                                      Instances For

                                                                                        Build a MulEquiv from an isomorphism in the category MonCat.

                                                                                        Equations
                                                                                        Instances For

                                                                                          Build an AddEquiv from an isomorphism in the category AddMonCat.

                                                                                          Equations
                                                                                          Instances For

                                                                                            Build a MulEquiv from an isomorphism in the category CommMonCat.

                                                                                            Equations
                                                                                            Instances For

                                                                                              Build an AddEquiv from an isomorphism in the category AddCommMonCat.

                                                                                              Equations
                                                                                              Instances For

                                                                                                multiplicative equivalences between Monoids 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 AddMonoids 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 CommMonoids 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 AddCommMonoids 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.

                                                                                                        @[deprecated "Proven by `simp only [MonCat.hom_id, comp_id]`" (since := "2025-01-28")]
                                                                                                        @[deprecated "Proven by `simp only [MonCat.hom_id, comp_id]`" (since := "2025-01-28")]
                                                                                                        @[deprecated "Proven by `simp only [MonCat.hom_id, id_comp]`" (since := "2025-01-28")]
                                                                                                        @[deprecated "Proven by `simp only [MonCat.hom_id, id_comp]`" (since := "2025-01-28")]
                                                                                                        @[deprecated "Proven by `simp only [CommMonCat.hom_id, comp_id]`" (since := "2025-01-28")]
                                                                                                        @[deprecated "Proven by `simp only [CommMonCat.hom_id, comp_id]`" (since := "2025-01-28")]
                                                                                                        @[deprecated "Proven by `simp only [CommMonCat.hom_id, id_comp]`" (since := "2025-01-28")]
                                                                                                        @[deprecated "Proven by `simp only [CommMonCat.hom_id, id_comp]`" (since := "2025-01-28")]

                                                                                                        The equivalence between AddMonCat and MonCat.

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

                                                                                                          The equivalence between AddCommMonCat and CommMonCat.

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