Documentation

Mathlib.Algebra.Category.Grp.EquivalenceGroupAddGroup

Equivalence between Group and AddGroup #

This file contains two equivalences:

The functor GrpAddGrp by sending X ↦ Additive X and f ↦ f.

Equations
Instances For
    @[simp]
    theorem Grp.toAddGrp_obj (X : Grp) :
    @[simp]
    theorem Grp.toAddGrp_map {x✝ x✝¹ : Grp} (a : x✝ →* x✝¹) :
    Grp.toAddGrp.map a = MonoidHom.toAdditive a

    The functor CommGrpAddCommGrp by sending X ↦ Additive X and f ↦ f.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For
      @[simp]
      theorem CommGrp.toAddCommGrp_map {x✝ x✝¹ : CommGrp} (a : x✝ →* x✝¹) :
      CommGrp.toAddCommGrp.map a = MonoidHom.toAdditive a

      The functor AddGrpGrp by sending X ↦ Multiplicative Y and f ↦ f.

      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        @[simp]
        theorem AddGrp.toGrp_map {x✝ x✝¹ : AddGrp} (a : x✝ →+ x✝¹) :
        AddGrp.toGrp.map a = AddMonoidHom.toMultiplicative a
        @[simp]

        The functor AddCommGrpCommGrp by sending X ↦ Multiplicative Y and f ↦ f.

        Equations
        • One or more equations did not get rendered due to their size.
        Instances For
          @[simp]
          theorem AddCommGrp.toCommGrp_map {x✝ x✝¹ : AddCommGrp} (a : x✝ →+ x✝¹) :
          AddCommGrp.toCommGrp.map a = AddMonoidHom.toMultiplicative a

          The equivalence of categories between Grp and AddGrp

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

            The equivalence of categories between CommGrp and AddCommGrp.

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