Documentation

Mathlib.CategoryTheory.Groupoid.VertexGroup

Vertex group #

This file defines the vertex group (aka isotropy group) of a groupoid at a vertex.

Implementation notes #

Tags #

isotropy, vertex group, groupoid

The vertex group at c.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    theorem CategoryTheory.Groupoid.vertexGroup_inv {C : Type u} [Groupoid C] (c : C) (a✝ : Quiver.Hom c c) :
    Eq (Inv.inv a✝) (inv a✝)

    The inverse in the group is equal to the inverse given by CategoryTheory.inv.

    An arrow in the groupoid defines, by conjugation, an isomorphism of groups between its endpoints.

    Equations
    • One or more equations did not get rendered due to their size.
    Instances For

      A path in the groupoid defines an isomorphism between its endpoints.

      Equations
      Instances For

        A functor defines a morphism of vertex group.

        Equations
        Instances For
          theorem CategoryTheory.Groupoid.CategoryTheory.Functor.mapVertexGroup_apply {C : Type u} [Groupoid C] {D : Type v} [Groupoid D] (φ : Functor C D) (c : C) (a✝ : Quiver.Hom c c) :
          Eq (DFunLike.coe (mapVertexGroup φ c) a✝) (φ.map a✝)