Equivalence between Group and AddGroup #
This file contains two equivalences:
groupAddGroupEquivalence: the equivalence betweenGrpandAddGrpby sendingX : GrptoAdditive XandY : AddGrptoMultiplicative Y.commGroupAddCommGroupEquivalence: the equivalence betweenCommGrpandAddCommGrpby sendingX : CommGrptoAdditive XandY : AddCommGrptoMultiplicative Y.
The functor Grp ⥤ AddGrp by sending X ↦ Additive X and f ↦ f.
Equations
- Grp.toAddGrp = { obj := fun (X : Grp) => AddGrp.of (Additive ↑X), map := fun {x x_1 : Grp} => ⇑MonoidHom.toAdditive, map_id := Grp.toAddGrp.proof_1, map_comp := @Grp.toAddGrp.proof_2 }
Instances For
@[simp]
theorem
Grp.toAddGrp_map
{x✝ x✝¹ : Grp}
(a : ↑x✝ →* ↑x✝¹)
:
Grp.toAddGrp.map a = MonoidHom.toAdditive a
The functor CommGrp ⥤ AddCommGrp 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
@[simp]
theorem
CommGrp.toAddCommGrp_obj
(X : CommGrp)
:
CommGrp.toAddCommGrp.obj X = AddCommGrp.of (Additive ↑X)
The functor AddGrp ⥤ Grp 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 AddCommGrp ⥤ CommGrp 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
@[simp]
theorem
AddCommGrp.toCommGrp_obj
(X : AddCommGrp)
:
AddCommGrp.toCommGrp.obj X = CommGrp.of (Multiplicative ↑X)
@[simp]
@[simp]
theorem
groupAddGroupEquivalence_counitIso :
groupAddGroupEquivalence.counitIso = CategoryTheory.Iso.refl (AddGrp.toGrp.comp Grp.toAddGrp)
@[simp]
@[simp]
The equivalence of categories between CommGrp and AddCommGrp.
Equations
- One or more equations did not get rendered due to their size.
Instances For
@[simp]
@[simp]
@[simp]