Documentation

Mathlib.GroupTheory.FreeGroup.CyclicallyReduced

This file defines some extra lemmas for free groups, in particular about cyclically reduced words.

Main declarations #

Predicate asserting that the word L is cyclically reduced, i.e., it is reduced and furthermore the first and the last letter of the word do not cancel. The empty word is by convention also cyclically reduced.

Equations
Instances For

    Predicate asserting that the word L is cyclically reduced, i.e., it is reduced and furthermore the first and the last letter of the word do not cancel. The empty word is by convention also cyclically reduced.

    Equations
    Instances For
      theorem FreeGroup.isCyclicallyReduced_iff {α : Type u} {L : List (α × Bool)} :
      IsCyclicallyReduced L IsReduced L aL.getLast?, bL.head?, a.1 = b.1a.2 = b.2
      theorem FreeAddGroup.isCyclicallyReduced_iff {α : Type u} {L : List (α × Bool)} :
      IsCyclicallyReduced L IsReduced L aL.getLast?, bL.head?, a.1 = b.1a.2 = b.2
      theorem FreeGroup.isCyclicallyReduced_cons_append_iff {α : Type u} {L : List (α × Bool)} {a b : α × Bool} :
      IsCyclicallyReduced (b :: L ++ [a]) IsReduced (b :: L ++ [a]) (a.1 = b.1a.2 = b.2)
      theorem FreeAddGroup.isCyclicallyReduced_cons_append_iff {α : Type u} {L : List (α × Bool)} {a b : α × Bool} :
      IsCyclicallyReduced (b :: L ++ [a]) IsReduced (b :: L ++ [a]) (a.1 = b.1a.2 = b.2)