Documentation

Mathlib.Algebra.Category.GrpWithZero

The category of groups with zero #

This file defines GrpWithZero, the category of groups with zero.

structure GrpWithZero :
Type (u_1 + 1)

The category of groups with zero.

Instances For
    Equations
    • One or more equations did not get rendered due to their size.
    Equations
    • One or more equations did not get rendered due to their size.
    @[reducible, inline]
    abbrev GrpWithZero.ofHom {X Y : Type u} [GroupWithZero X] [GroupWithZero Y] (f : X →*₀ Y) :
    { carrier := X, str := inst✝ } { carrier := Y, str := inst✝¹ }

    Typecheck a MonoidWithZeroHom as a morphism in GrpWithZero.

    Equations
    Instances For
      Equations
      • One or more equations did not get rendered due to their size.
      Equations
      • One or more equations did not get rendered due to their size.
      def GrpWithZero.Iso.mk {α β : GrpWithZero} (e : α.carrier ≃* β.carrier) :
      α β

      Constructs an isomorphism of groups with zero from a group isomorphism between them.

      Equations
      Instances For
        @[simp]
        theorem GrpWithZero.Iso.mk_hom {α β : GrpWithZero} (e : α.carrier ≃* β.carrier) :
        (mk e).hom = ofHom e
        @[simp]
        theorem GrpWithZero.Iso.mk_inv {α β : GrpWithZero} (e : α.carrier ≃* β.carrier) :
        (mk e).inv = ofHom e.symm