Documentation

Mathlib.Algebra.Category.GroupWithZeroCat

The category of groups with zero #

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

def GroupWithZeroCat :
Type (u_1 + 1)

The category of groups with zero.

Instances For

    Construct a bundled GroupWithZeroCat from a GroupWithZero.

    Instances For
      @[simp]
      theorem GroupWithZeroCat.Iso.mk_hom {α : GroupWithZeroCat} {β : GroupWithZeroCat} (e : α ≃* β) :
      def GroupWithZeroCat.Iso.mk {α : GroupWithZeroCat} {β : GroupWithZeroCat} (e : α ≃* β) :
      α β

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

      Instances For