This file defines some extra lemmas for free groups, in particular about cyclically reduced words.
We show that free groups are (strongly) torsion-free in the sense of IsMulTorsionFree, i.e.,
taking powers by every non-zero element n : ℕ is injective.
Main declarations #
FreeGroup.IsCyclicallyReduced: the predicate for cyclically reduced words
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
- FreeGroup.IsCyclicallyReduced L = (FreeGroup.IsReduced L ∧ ∀ a ∈ L.getLast?, ∀ b ∈ L.head?, a.1 = b.1 → a.2 = b.2)
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
- FreeAddGroup.IsCyclicallyReduced L = (FreeAddGroup.IsReduced L ∧ ∀ a ∈ L.getLast?, ∀ b ∈ L.head?, a.1 = b.1 → a.2 = b.2)
Instances For
This function produces a subword of a word L by cancelling the first and last letters of L
as long as possible. If L is reduced, the resulting word will be cyclically reduced.
Equations
- One or more equations did not get rendered due to their size.
Instances For
This function produces a subword of a word L by cancelling the first and last
letters of L as long as possible. If L is reduced, the resulting word will be cyclically
reduced.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Partner function to reduceCyclically.
See reduceCyclically.conj_conjugator_reduceCyclically.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Partner function to reduceCyclically.
See reduceCyclically.conj_conjugator_reduceCyclically.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Free groups are torsion-free, i.e., taking powers is injective. Our proof idea is as follows:
if x ^ n = y ^ n, then also x ^ (2 * n) = y ^ (2 * n). We then compare the reduced words
representing the powers in terms of the cyclic reductions of x.toWord and y.toWord using
reduce_flatten_replicate. We conclude that the cyclic reductions of x.toWord and y.toWord must
have the same length, and in fact they have to agree.
Free additive groups are torsion free, i.e., scalar multiplication by every
non-zero element n : ℕ is injective. See the instance for free groups for an overview over the
proof.