Documentation

Mathlib.Algebra.Category.Grp.Preadditive

The category of additive commutative groups is preadditive. #

Equations
  • P.instAddCommGroupHom Q = inferInstance
@[simp]
theorem AddCommGrp.hom_add_apply {P : AddCommGrp} {Q : AddCommGrp} (f : P Q) (g : P Q) (x : P) :
(f + g) x = f x + g x