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.

Equations
Instances For
    Equations
    • One or more equations did not get rendered due to their size.
    Equations
    • GroupWithZeroCat.instFunLikeHomGroupWithZeroCatToQuiverToCategoryStructInstLargeCategoryGroupWithZeroCatαGroupWithZero = { coe := fun (f : M N) => f.toFun, coe_injective' := }
    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.
    Equations
    • One or more equations did not get rendered due to their size.
    @[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.

    Equations
    Instances For