mathlib3 documentation

group_theory.free_group

Free groups #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

This file defines free groups over a type. Furthermore, it is shown that the free group construction is an instance of a monad. For the result that free_group is the left adjoint to the forgetful functor from groups to types, see algebra/category/Group/adjunctions.

Main definitions #

Main statements #

Implementation details #

First we introduce the one step reduction relation free_group.red.step: w * x * x⁻¹ * v ~> w * v, its reflexive transitive closure free_group.red.trans and prove that its join is an equivalence relation. Then we introduce free_group α as a quotient over free_group.red.step.

For the additive version we introduce the same relation under a different name so that we can distinguish the quotient types more easily.

Tags #

free group, Newman's diamond lemma, Church-Rosser theorem

inductive free_add_group.red.step {α : Type u} :
list × bool) list × bool) Prop

Reduction step for the additive free group relation: w + x + (-x) + v ~> w + v

inductive free_group.red.step {α : Type u} :
list × bool) list × bool) Prop

Reduction step for the multiplicative free group relation: w * x * x⁻¹ * v ~> w * v

def free_group.red {α : Type u} :
list × bool) list × bool) Prop

Reflexive-transitive closure of red.step

Equations
Instances for free_group.red
def free_add_group.red {α : Type u} :
list × bool) list × bool) Prop

Reflexive-transitive closure of red.step

Equations
@[refl]
theorem free_add_group.red.refl {α : Type u} {L : list × bool)} :
@[refl]
theorem free_group.red.refl {α : Type u} {L : list × bool)} :
@[trans]
theorem free_group.red.trans {α : Type u} {L₁ L₂ L₃ : list × bool)} :
free_group.red L₁ L₂ free_group.red L₂ L₃ free_group.red L₁ L₃
@[trans]
theorem free_add_group.red.trans {α : Type u} {L₁ L₂ L₃ : list × bool)} :
theorem free_group.red.step.length {α : Type u} {L₁ L₂ : list × bool)} :
free_group.red.step L₁ L₂ L₂.length + 2 = L₁.length

Predicate asserting that the word w₁ can be reduced to w₂ in one step, i.e. there are words w₃ w₄ and letter x such that w₁ = w₃xx⁻¹w₄ and w₂ = w₃w₄

theorem free_add_group.red.step.length {α : Type u} {L₁ L₂ : list × bool)} :
free_add_group.red.step L₁ L₂ L₂.length + 2 = L₁.length

Predicate asserting that the word w₁ can be reduced to w₂ in one step, i.e. there are words w₃ w₄ and letter x such that w₁ = w₃ + x + (-x) + w₄ and w₂ = w₃w₄

@[simp]
theorem free_add_group.red.step.bnot_rev {α : Type u} {L₁ L₂ : list × bool)} {x : α} {b : bool} :
free_add_group.red.step (L₁ ++ (x, !b) :: (x, b) :: L₂) (L₁ ++ L₂)
@[simp]
theorem free_group.red.step.bnot_rev {α : Type u} {L₁ L₂ : list × bool)} {x : α} {b : bool} :
free_group.red.step (L₁ ++ (x, !b) :: (x, b) :: L₂) (L₁ ++ L₂)
@[simp]
theorem free_add_group.red.step.cons_bnot {α : Type u} {L : list × bool)} {x : α} {b : bool} :
free_add_group.red.step ((x, b) :: (x, !b) :: L) L
@[simp]
theorem free_group.red.step.cons_bnot {α : Type u} {L : list × bool)} {x : α} {b : bool} :
free_group.red.step ((x, b) :: (x, !b) :: L) L
@[simp]
theorem free_add_group.red.step.cons_bnot_rev {α : Type u} {L : list × bool)} {x : α} {b : bool} :
free_add_group.red.step ((x, !b) :: (x, b) :: L) L
@[simp]
theorem free_group.red.step.cons_bnot_rev {α : Type u} {L : list × bool)} {x : α} {b : bool} :
free_group.red.step ((x, !b) :: (x, b) :: L) L
theorem free_group.red.step.append_left {α : Type u} {L₁ L₂ L₃ : list × bool)} :
free_group.red.step L₂ L₃ free_group.red.step (L₁ ++ L₂) (L₁ ++ L₃)
theorem free_add_group.red.step.append_left {α : Type u} {L₁ L₂ L₃ : list × bool)} :
free_add_group.red.step L₂ L₃ free_add_group.red.step (L₁ ++ L₂) (L₁ ++ L₃)
theorem free_group.red.step.cons {α : Type u} {L₁ L₂ : list × bool)} {x : α × bool} (H : free_group.red.step L₁ L₂) :
free_group.red.step (x :: L₁) (x :: L₂)
theorem free_add_group.red.step.cons {α : Type u} {L₁ L₂ : list × bool)} {x : α × bool} (H : free_add_group.red.step L₁ L₂) :
free_add_group.red.step (x :: L₁) (x :: L₂)
theorem free_add_group.red.step.append_right {α : Type u} {L₁ L₂ L₃ : list × bool)} :
free_add_group.red.step L₁ L₂ free_add_group.red.step (L₁ ++ L₃) (L₂ ++ L₃)
theorem free_group.red.step.append_right {α : Type u} {L₁ L₂ L₃ : list × bool)} :
free_group.red.step L₁ L₂ free_group.red.step (L₁ ++ L₃) (L₂ ++ L₃)
theorem free_group.red.step.cons_left_iff {α : Type u} {L₁ L₂ : list × bool)} {a : α} {b : bool} :
free_group.red.step ((a, b) :: L₁) L₂ ( (L : list × bool)), free_group.red.step L₁ L L₂ = (a, b) :: L) L₁ = (a, !b) :: L₂
theorem free_add_group.red.step.cons_left_iff {α : Type u} {L₁ L₂ : list × bool)} {a : α} {b : bool} :
free_add_group.red.step ((a, b) :: L₁) L₂ ( (L : list × bool)), free_add_group.red.step L₁ L L₂ = (a, b) :: L) L₁ = (a, !b) :: L₂
theorem free_group.red.not_step_singleton {α : Type u} {L : list × bool)} {p : α × bool} :
theorem free_add_group.red.step.cons_cons_iff {α : Type u} {L₁ L₂ : list × bool)} {p : α × bool} :
theorem free_group.red.step.cons_cons_iff {α : Type u} {L₁ L₂ : list × bool)} {p : α × bool} :
free_group.red.step (p :: L₁) (p :: L₂) free_group.red.step L₁ L₂
theorem free_add_group.red.step.append_left_iff {α : Type u} {L₁ L₂ : list × bool)} (L : list × bool)) :
theorem free_group.red.step.append_left_iff {α : Type u} {L₁ L₂ : list × bool)} (L : list × bool)) :
free_group.red.step (L ++ L₁) (L ++ L₂) free_group.red.step L₁ L₂
theorem free_add_group.red.step.diamond_aux {α : Type u} {L₁ L₂ L₃ L₄ : list × bool)} {x1 : α} {b1 : bool} {x2 : α} {b2 : bool} :
L₁ ++ (x1, b1) :: (x1, !b1) :: L₂ = L₃ ++ (x2, b2) :: (x2, !b2) :: L₄ (L₁ ++ L₂ = L₃ ++ L₄ (L₅ : list × bool)), free_add_group.red.step (L₁ ++ L₂) L₅ free_add_group.red.step (L₃ ++ L₄) L₅)
theorem free_group.red.step.diamond_aux {α : Type u} {L₁ L₂ L₃ L₄ : list × bool)} {x1 : α} {b1 : bool} {x2 : α} {b2 : bool} :
L₁ ++ (x1, b1) :: (x1, !b1) :: L₂ = L₃ ++ (x2, b2) :: (x2, !b2) :: L₄ (L₁ ++ L₂ = L₃ ++ L₄ (L₅ : list × bool)), free_group.red.step (L₁ ++ L₂) L₅ free_group.red.step (L₃ ++ L₄) L₅)
theorem free_group.red.step.diamond {α : Type u} {L₁ L₂ L₃ L₄ : list × bool)} :
free_group.red.step L₁ L₃ free_group.red.step L₂ L₄ L₁ = L₂ (L₃ = L₄ (L₅ : list × bool)), free_group.red.step L₃ L₅ free_group.red.step L₄ L₅)
theorem free_add_group.red.step.diamond {α : Type u} {L₁ L₂ L₃ L₄ : list × bool)} :
free_add_group.red.step L₁ L₃ free_add_group.red.step L₂ L₄ L₁ = L₂ (L₃ = L₄ (L₅ : list × bool)), free_add_group.red.step L₃ L₅ free_add_group.red.step L₄ L₅)
theorem free_add_group.red.step.to_red {α : Type u} {L₁ L₂ : list × bool)} :
theorem free_group.red.step.to_red {α : Type u} {L₁ L₂ : list × bool)} :
theorem free_group.red.church_rosser {α : Type u} {L₁ L₂ L₃ : list × bool)} :

Church-Rosser theorem for word reduction: If w1 w2 w3 are words such that w1 reduces to w2 and w3 respectively, then there is a word w4 such that w2 and w3 reduce to w4 respectively. This is also known as Newman's diamond lemma.

theorem free_add_group.red.church_rosser {α : Type u} {L₁ L₂ L₃ : list × bool)} :

Church-Rosser theorem for word reduction: If w1 w2 w3 are words such that w1 reduces to w2 and w3 respectively, then there is a word w4 such that w2 and w3 reduce to w4 respectively. This is also known as Newman's diamond lemma.

theorem free_add_group.red.cons_cons {α : Type u} {L₁ L₂ : list × bool)} {p : α × bool} :
free_add_group.red L₁ L₂ free_add_group.red (p :: L₁) (p :: L₂)
theorem free_group.red.cons_cons {α : Type u} {L₁ L₂ : list × bool)} {p : α × bool} :
free_group.red L₁ L₂ free_group.red (p :: L₁) (p :: L₂)
theorem free_group.red.cons_cons_iff {α : Type u} {L₁ L₂ : list × bool)} (p : α × bool) :
free_group.red (p :: L₁) (p :: L₂) free_group.red L₁ L₂
theorem free_add_group.red.cons_cons_iff {α : Type u} {L₁ L₂ : list × bool)} (p : α × bool) :
free_add_group.red (p :: L₁) (p :: L₂) free_add_group.red L₁ L₂
theorem free_add_group.red.append_append_left_iff {α : Type u} {L₁ L₂ : list × bool)} (L : list × bool)) :
free_add_group.red (L ++ L₁) (L ++ L₂) free_add_group.red L₁ L₂
theorem free_group.red.append_append_left_iff {α : Type u} {L₁ L₂ : list × bool)} (L : list × bool)) :
free_group.red (L ++ L₁) (L ++ L₂) free_group.red L₁ L₂
theorem free_group.red.append_append {α : Type u} {L₁ L₂ L₃ L₄ : list × bool)} (h₁ : free_group.red L₁ L₃) (h₂ : free_group.red L₂ L₄) :
free_group.red (L₁ ++ L₂) (L₃ ++ L₄)
theorem free_add_group.red.append_append {α : Type u} {L₁ L₂ L₃ L₄ : list × bool)} (h₁ : free_add_group.red L₁ L₃) (h₂ : free_add_group.red L₂ L₄) :
free_add_group.red (L₁ ++ L₂) (L₃ ++ L₄)
theorem free_add_group.red.to_append_iff {α : Type u} {L L₁ L₂ : list × bool)} :
free_add_group.red L (L₁ ++ L₂) (L₃ L₄ : list × bool)), L = L₃ ++ L₄ free_add_group.red L₃ L₁ free_add_group.red L₄ L₂
theorem free_group.red.to_append_iff {α : Type u} {L L₁ L₂ : list × bool)} :
free_group.red L (L₁ ++ L₂) (L₃ L₄ : list × bool)), L = L₃ ++ L₄ free_group.red L₃ L₁ free_group.red L₄ L₂

The empty word [] only reduces to itself.

The empty word [] only reduces to itself.

theorem free_group.red.singleton_iff {α : Type u} {L₁ : list × bool)} {x : α × bool} :
free_group.red [x] L₁ L₁ = [x]

A letter only reduces to itself.

theorem free_add_group.red.singleton_iff {α : Type u} {L₁ : list × bool)} {x : α × bool} :
free_add_group.red [x] L₁ L₁ = [x]

A letter only reduces to itself.

theorem free_group.red.cons_nil_iff_singleton {α : Type u} {L : list × bool)} {x : α} {b : bool} :

If x is a letter and w is a word such that xw reduces to the empty word, then w reduces to x⁻¹

theorem free_add_group.red.cons_nil_iff_singleton {α : Type u} {L : list × bool)} {x : α} {b : bool} :

If x is a letter and w is a word such that x + w reduces to the empty word, then w reduces to -x.

theorem free_add_group.red.red_iff_irreducible {α : Type u} {L : list × bool)} {x1 : α} {b1 : bool} {x2 : α} {b2 : bool} (h : (x1, b1) (x2, b2)) :
free_add_group.red [(x1, !b1), (x2, b2)] L L = [(x1, !b1), (x2, b2)]
theorem free_group.red.red_iff_irreducible {α : Type u} {L : list × bool)} {x1 : α} {b1 : bool} {x2 : α} {b2 : bool} (h : (x1, b1) (x2, b2)) :
free_group.red [(x1, !b1), (x2, b2)] L L = [(x1, !b1), (x2, b2)]
theorem free_group.red.inv_of_red_of_ne {α : Type u} {L₁ L₂ : list × bool)} {x1 : α} {b1 : bool} {x2 : α} {b2 : bool} (H1 : (x1, b1) (x2, b2)) (H2 : free_group.red ((x1, b1) :: L₁) ((x2, b2) :: L₂)) :
free_group.red L₁ ((x1, !b1) :: (x2, b2) :: L₂)

If x and y are distinct letters and w₁ w₂ are words such that xw₁ reduces to yw₂, then w₁ reduces to x⁻¹yw₂.

theorem free_add_group.red.neg_of_red_of_ne {α : Type u} {L₁ L₂ : list × bool)} {x1 : α} {b1 : bool} {x2 : α} {b2 : bool} (H1 : (x1, b1) (x2, b2)) (H2 : free_add_group.red ((x1, b1) :: L₁) ((x2, b2) :: L₂)) :
free_add_group.red L₁ ((x1, !b1) :: (x2, b2) :: L₂)

If x and y are distinct letters and w₁ w₂ are words such that x + w₁ reduces to y + w₂, then w₁ reduces to -x + y + w₂.

theorem free_add_group.red.step.sublist {α : Type u} {L₁ L₂ : list × bool)} (H : free_add_group.red.step L₁ L₂) :
L₂ <+ L₁
theorem free_group.red.step.sublist {α : Type u} {L₁ L₂ : list × bool)} (H : free_group.red.step L₁ L₂) :
L₂ <+ L₁
@[protected]
theorem free_add_group.red.sublist {α : Type u} {L₁ L₂ : list × bool)} :
free_add_group.red L₁ L₂ L₂ <+ L₁

If w₁ w₂ are words such that w₁ reduces to w₂, then w₂ is a sublist of w₁.

@[protected]
theorem free_group.red.sublist {α : Type u} {L₁ L₂ : list × bool)} :
free_group.red L₁ L₂ L₂ <+ L₁

If w₁ w₂ are words such that w₁ reduces to w₂, then w₂ is a sublist of w₁.

theorem free_add_group.red.length_le {α : Type u} {L₁ L₂ : list × bool)} (h : free_add_group.red L₁ L₂) :
L₂.length L₁.length
theorem free_group.red.length_le {α : Type u} {L₁ L₂ : list × bool)} (h : free_group.red L₁ L₂) :
L₂.length L₁.length
theorem free_group.red.sizeof_of_step {α : Type u} {L₁ L₂ : list × bool)} :
free_group.red.step L₁ L₂ L₂.sizeof < L₁.sizeof
theorem free_add_group.red.sizeof_of_step {α : Type u} {L₁ L₂ : list × bool)} :
free_add_group.red.step L₁ L₂ L₂.sizeof < L₁.sizeof
theorem free_group.red.length {α : Type u} {L₁ L₂ : list × bool)} (h : free_group.red L₁ L₂) :
(n : ), L₁.length = L₂.length + 2 * n
theorem free_add_group.red.length {α : Type u} {L₁ L₂ : list × bool)} (h : free_add_group.red L₁ L₂) :
(n : ), L₁.length = L₂.length + 2 * n
theorem free_add_group.red.antisymm {α : Type u} {L₁ L₂ : list × bool)} (h₁₂ : free_add_group.red L₁ L₂) (h₂₁ : free_add_group.red L₂ L₁) :
L₁ = L₂
theorem free_group.red.antisymm {α : Type u} {L₁ L₂ : list × bool)} (h₁₂ : free_group.red L₁ L₂) (h₂₁ : free_group.red L₂ L₁) :
L₁ = L₂
theorem free_group.join_red_of_step {α : Type u} {L₁ L₂ : list × bool)} (h : free_group.red.step L₁ L₂) :
theorem free_add_group.join_red_of_step {α : Type u} {L₁ L₂ : list × bool)} (h : free_add_group.red.step L₁ L₂) :
def free_group (α : Type u) :

The free group over a type, i.e. the words formed by the elements of the type and their formal inverses, quotient by one step reduction.

Equations
Instances for free_group
def free_add_group (α : Type u) :

The free additive group over a type, i.e. the words formed by the elements of the type and their formal inverses, quotient by one step reduction.

Equations
Instances for free_add_group
def free_group.mk {α : Type u} (L : list × bool)) :

The canonical map from list (α × bool) to the free group on α.

Equations
def free_add_group.mk {α : Type u} (L : list × bool)) :

The canonical map from list (α × bool) to the free additive group on α.

Equations
@[simp]
@[simp]
theorem free_group.quot_mk_eq_mk {α : Type u} {L : list × bool)} :
@[simp]
theorem free_group.quot_lift_mk {α : Type u} {L : list × bool)} (β : Type v) (f : list × bool) β) (H : (L₁ L₂ : list × bool)), free_group.red.step L₁ L₂ f L₁ = f L₂) :
quot.lift f H (free_group.mk L) = f L
@[simp]
theorem free_add_group.quot_lift_mk {α : Type u} {L : list × bool)} (β : Type v) (f : list × bool) β) (H : (L₁ L₂ : list × bool)), free_add_group.red.step L₁ L₂ f L₁ = f L₂) :
quot.lift f H (free_add_group.mk L) = f L
@[simp]
theorem free_group.quot_lift_on_mk {α : Type u} {L : list × bool)} (β : Type v) (f : list × bool) β) (H : (L₁ L₂ : list × bool)), free_group.red.step L₁ L₂ f L₁ = f L₂) :
@[simp]
theorem free_add_group.quot_lift_on_mk {α : Type u} {L : list × bool)} (β : Type v) (f : list × bool) β) (H : (L₁ L₂ : list × bool)), free_add_group.red.step L₁ L₂ f L₁ = f L₂) :
@[simp]
@[simp]
theorem free_group.quot_map_mk {α : Type u} {L : list × bool)} (β : Type v) (f : list × bool) list × bool)) (H : (free_group.red.step free_group.red.step) f f) :
@[protected, instance]
def free_group.has_one {α : Type u} :
Equations
@[protected, instance]
Equations
@[protected, instance]
Equations
@[protected, instance]
Equations
@[protected, instance]
def free_group.has_mul {α : Type u} :
Equations
@[simp]
theorem free_group.mul_mk {α : Type u} {L₁ L₂ : list × bool)} :
@[simp]
theorem free_add_group.add_mk {α : Type u} {L₁ L₂ : list × bool)} :
def free_group.inv_rev {α : Type u} (w : list × bool)) :
list × bool)

Transform a word representing a free group element into a word representing its inverse.

Equations
def free_add_group.neg_rev {α : Type u} (w : list × bool)) :
list × bool)

Transform a word representing a free group element into a word representing its negative.

Equations
@[simp]
theorem free_group.inv_rev_length {α : Type u} {L₁ : list × bool)} :
@[simp]
theorem free_add_group.neg_rev_length {α : Type u} {L₁ : list × bool)} :
@[simp]
@[simp]
theorem free_group.inv_rev_inv_rev {α : Type u} {L₁ : list × bool)} :
@[protected, instance]
Equations
@[protected, instance]
def free_group.has_inv {α : Type u} :
Equations
@[simp]
theorem free_group.red.inv_rev {α : Type u} {L₁ L₂ : list × bool)} (h : free_group.red L₁ L₂) :
@[simp]
theorem free_group.red_inv_rev_iff {α : Type u} {L₁ L₂ : list × bool)} :
@[protected, instance]
def free_group.group {α : Type u} :
Equations
@[protected, instance]
Equations
def free_group.of {α : Type u} (x : α) :

of is the canonical injection from the type to the free group over that type by sending each element to the equivalence class of the letter that is the element.

Equations
def free_add_group.of {α : Type u} (x : α) :

of is the canonical injection from the type to the free group over that type by sending each element to the equivalence class of the letter that is the element.

Equations
theorem free_group.red.exact {α : Type u} {L₁ L₂ : list × bool)} :

The canonical map from the type to the additive free group is an injection.

The canonical map from the type to the free group is an injection.

def free_add_group.lift.aux {α : Type u} {β : Type v} [add_group β] (f : α β) :
list × bool) β

Given f : α → β with β an additive group, the canonical map list (α × bool) → β

Equations
def free_group.lift.aux {α : Type u} {β : Type v} [group β] (f : α β) :
list × bool) β

Given f : α → β with β a group, the canonical map list (α × bool) → β

Equations
theorem free_add_group.red.step.lift {α : Type u} {L₁ L₂ : list × bool)} {β : Type v} [add_group β] {f : α β} (H : free_add_group.red.step L₁ L₂) :
theorem free_group.red.step.lift {α : Type u} {L₁ L₂ : list × bool)} {β : Type v} [group β] {f : α β} (H : free_group.red.step L₁ L₂) :
@[simp]
theorem free_group.lift_symm_apply {α : Type u} {β : Type v} [group β] (g : free_group α →* β) (ᾰ : α) :
def free_group.lift {α : Type u} {β : Type v} [group β] :
β) (free_group α →* β)

If β is a group, then any function from α to β extends uniquely to a group homomorphism from the free group over α to β

Equations
@[simp]
theorem free_add_group.lift_symm_apply {α : Type u} {β : Type v} [add_group β] (g : free_add_group α →+ β) (ᾰ : α) :
def free_add_group.lift {α : Type u} {β : Type v} [add_group β] :
β) (free_add_group α →+ β)

If β is an additive group, then any function from α to β extends uniquely to an additive group homomorphism from the free additive group over α to β

Equations
@[simp]
theorem free_add_group.lift.mk {α : Type u} {L : list × bool)} {β : Type v} [add_group β] {f : α β} :
(free_add_group.lift f) (free_add_group.mk L) = (list.map (λ (x : α × bool), cond x.snd (f x.fst) (-f x.fst)) L).sum
@[simp]
theorem free_group.lift.mk {α : Type u} {L : list × bool)} {β : Type v} [group β] {f : α β} :
(free_group.lift f) (free_group.mk L) = (list.map (λ (x : α × bool), cond x.snd (f x.fst) (f x.fst)⁻¹) L).prod
@[simp]
theorem free_group.lift.of {α : Type u} {β : Type v} [group β] {f : α β} {x : α} :
@[simp]
theorem free_add_group.lift.of {α : Type u} {β : Type v} [add_group β] {f : α β} {x : α} :
theorem free_add_group.lift.unique {α : Type u} {β : Type v} [add_group β] {f : α β} (g : free_add_group α →+ β) (hg : (x : α), g (free_add_group.of x) = f x) {x : free_add_group α} :
theorem free_group.lift.unique {α : Type u} {β : Type v} [group β] {f : α β} (g : free_group α →* β) (hg : (x : α), g (free_group.of x) = f x) {x : free_group α} :
@[ext]
theorem free_group.ext_hom {α : Type u} {G : Type u_1} [group G] (f g : free_group α →* G) (h : (a : α), f (free_group.of a) = g (free_group.of a)) :
f = g

Two homomorphisms out of a free group are equal if they are equal on generators.

See note [partially-applied ext lemmas].

@[ext]
theorem free_add_group.ext_hom {α : Type u} {G : Type u_1} [add_group G] (f g : free_add_group α →+ G) (h : (a : α), f (free_add_group.of a) = g (free_add_group.of a)) :
f = g

Two homomorphisms out of a free additive group are equal if they are equal on generators.

See note [partially-applied ext lemmas].

theorem free_group.lift.range_le {α : Type u} {β : Type v} [group β] {f : α β} {s : subgroup β} (H : set.range f s) :
theorem free_add_group.lift.range_le {α : Type u} {β : Type v} [add_group β] {f : α β} {s : add_subgroup β} (H : set.range f s) :
def free_group.map {α : Type u} {β : Type v} (f : α β) :

Any function from α to β extends uniquely to a group homomorphism from the free group over α to the free group over β.

Equations
def free_add_group.map {α : Type u} {β : Type v} (f : α β) :

Any function from α to β extends uniquely to an additive group homomorphism from the additive free group over α to the additive free group over β.

Equations
@[simp]
theorem free_group.map.mk {α : Type u} {L : list × bool)} {β : Type v} {f : α β} :
(free_group.map f) (free_group.mk L) = free_group.mk (list.map (λ (x : α × bool), (f x.fst, x.snd)) L)
@[simp]
theorem free_add_group.map.mk {α : Type u} {L : list × bool)} {β : Type v} {f : α β} :
@[simp]
theorem free_add_group.map.id {α : Type u} (x : free_add_group α) :
@[simp]
theorem free_group.map.id {α : Type u} (x : free_group α) :
@[simp]
theorem free_group.map.id' {α : Type u} (x : free_group α) :
(free_group.map (λ (z : α), z)) x = x
@[simp]
theorem free_add_group.map.id' {α : Type u} (x : free_add_group α) :
(free_add_group.map (λ (z : α), z)) x = x
theorem free_group.map.comp {α : Type u} {β : Type v} {γ : Type w} (f : α β) (g : β γ) (x : free_group α) :
theorem free_add_group.map.comp {α : Type u} {β : Type v} {γ : Type w} (f : α β) (g : β γ) (x : free_add_group α) :
@[simp]
theorem free_add_group.map.of {α : Type u} {β : Type v} {f : α β} {x : α} :
@[simp]
theorem free_group.map.of {α : Type u} {β : Type v} {f : α β} {x : α} :
theorem free_group.map.unique {α : Type u} {β : Type v} {f : α β} (g : free_group α →* free_group β) (hg : (x : α), g (free_group.of x) = free_group.of (f x)) {x : free_group α} :
theorem free_add_group.map.unique {α : Type u} {β : Type v} {f : α β} (g : free_add_group α →+ free_add_group β) (hg : (x : α), g (free_add_group.of x) = free_add_group.of (f x)) {x : free_add_group α} :
theorem free_group.map_eq_lift {α : Type u} {β : Type v} {f : α β} {x : free_group α} :
@[simp]
theorem free_group.free_group_congr_apply {α : Type u_1} {β : Type u_2} (e : α β) (ᾰ : free_group α) :
@[simp]
def free_group.free_group_congr {α : Type u_1} {β : Type u_2} (e : α β) :

Equivalent types give rise to multiplicatively equivalent free groups.

The converse can be found in group_theory.free_abelian_group_finsupp, as equiv.of_free_group_equiv

Equations
def free_add_group.free_add_group_congr {α : Type u_1} {β : Type u_2} (e : α β) :

Equivalent types give rise to additively equivalent additive free groups.

Equations
def free_group.prod {α : Type u} [group α] :

If α is a group, then any function from α to α extends uniquely to a homomorphism from the free group over α to α. This is the multiplicative version of free_group.sum.

Equations
def free_add_group.sum {α : Type u} [add_group α] :

If α is an additive group, then any function from α to α extends uniquely to an additive homomorphism from the additive free group over α to α.

Equations
@[simp]
theorem free_group.prod_mk {α : Type u} {L : list × bool)} [group α] :
@[simp]
theorem free_add_group.sum_mk {α : Type u} {L : list × bool)} [add_group α] :
@[simp]
@[simp]
theorem free_group.prod.of {α : Type u} [group α] {x : α} :
theorem free_group.prod.unique {α : Type u} [group α] (g : free_group α →* α) (hg : (x : α), g (free_group.of x) = x) {x : free_group α} :
theorem free_add_group.sum.unique {α : Type u} [add_group α] (g : free_add_group α →+ α) (hg : (x : α), g (free_add_group.of x) = x) {x : free_add_group α} :
theorem free_group.lift_eq_prod_map {α : Type u} {β : Type v} [group β] {f : α β} {x : free_group α} :
def free_group.sum {α : Type u} [add_group α] (x : free_group α) :
α

If α is a group, then any function from α to α extends uniquely to a homomorphism from the free group over α to α. This is the additive version of prod.

Equations
@[simp]
theorem free_group.sum_mk {α : Type u} {L : list × bool)} [add_group α] :
(free_group.mk L).sum = (list.map (λ (x : α × bool), cond x.snd x.fst (-x.fst)) L).sum
@[simp]
theorem free_group.sum.of {α : Type u} [add_group α] {x : α} :
@[simp]
theorem free_group.sum.map_mul {α : Type u} [add_group α] {x y : free_group α} :
(x * y).sum = x.sum + y.sum
@[simp]
theorem free_group.sum.map_one {α : Type u} [add_group α] :
1.sum = 0
@[simp]
theorem free_group.sum.map_inv {α : Type u} [add_group α] {x : free_group α} :

The bijection between the additive free group on the empty type, and a type with one element.

Equations

The bijection between the free group on the empty type, and a type with one element.

Equations

The bijection between the free group on a singleton, and the integers.

Equations
@[protected, instance]
Equations
@[protected]
theorem free_group.induction_on {α : Type u} {C : free_group α Prop} (z : free_group α) (C1 : C 1) (Cp : (x : α), C (has_pure.pure x)) (Ci : (x : α), C (has_pure.pure x) C (has_pure.pure x)⁻¹) (Cm : (x y : free_group α), C x C y C (x * y)) :
C z
@[protected]
theorem free_add_group.induction_on {α : Type u} {C : free_add_group α Prop} (z : free_add_group α) (C1 : C 0) (Cp : (x : α), C (has_pure.pure x)) (Ci : (x : α), C (has_pure.pure x) C (-has_pure.pure x)) (Cm : (x y : free_add_group α), C x C y C (x + y)) :
C z
@[simp]
theorem free_group.map_pure {α β : Type u} (f : α β) (x : α) :
@[simp]
theorem free_add_group.map_pure {α β : Type u} (f : α β) (x : α) :
@[simp]
theorem free_add_group.map_zero {α β : Type u} (f : α β) :
f <$> 0 = 0
@[simp]
theorem free_group.map_one {α β : Type u} (f : α β) :
f <$> 1 = 1
@[simp]
theorem free_add_group.map_add {α β : Type u} (f : α β) (x y : free_add_group α) :
f <$> (x + y) = f <$> x + f <$> y
@[simp]
theorem free_group.map_mul {α β : Type u} (f : α β) (x y : free_group α) :
f <$> (x * y) = f <$> x * f <$> y
@[simp]
theorem free_add_group.map_neg {α β : Type u} (f : α β) (x : free_add_group α) :
f <$> -x = -f <$> x
@[simp]
theorem free_group.map_inv {α β : Type u} (f : α β) (x : free_group α) :
f <$> x⁻¹ = (f <$> x)⁻¹
@[simp]
theorem free_group.pure_bind {α β : Type u} (f : α free_group β) (x : α) :
@[simp]
theorem free_add_group.pure_bind {α β : Type u} (f : α free_add_group β) (x : α) :
@[simp]
theorem free_group.one_bind {α β : Type u} (f : α free_group β) :
1 >>= f = 1
@[simp]
theorem free_add_group.zero_bind {α β : Type u} (f : α free_add_group β) :
0 >>= f = 0
@[simp]
theorem free_group.mul_bind {α β : Type u} (f : α free_group β) (x y : free_group α) :
x * y >>= f = (x >>= f) * (y >>= f)
@[simp]
theorem free_add_group.add_bind {α β : Type u} (f : α free_add_group β) (x y : free_add_group α) :
x + y >>= f = (x >>= f) + (y >>= f)
@[simp]
theorem free_add_group.neg_bind {α β : Type u} (f : α free_add_group β) (x : free_add_group α) :
-x >>= f = -(x >>= f)
@[simp]
theorem free_group.inv_bind {α β : Type u} (f : α free_group β) (x : free_group α) :
x⁻¹ >>= f = (x >>= f)⁻¹
def free_group.reduce {α : Type u} [decidable_eq α] (L : list × bool)) :
list × bool)

The maximal reduction of a word. It is computable iff α has decidable equality.

Equations
def free_add_group.reduce {α : Type u} [decidable_eq α] (L : list × bool)) :
list × bool)

The maximal reduction of a word. It is computable iff α has decidable equality.

Equations
@[simp]
theorem free_add_group.reduce.cons {α : Type u} {L : list × bool)} [decidable_eq α] (x : α × bool) :
free_add_group.reduce (x :: L) = (free_add_group.reduce L).cases_on [x] (λ (hd : α × bool) (tl : list × bool)), ite (x.fst = hd.fst x.snd = !hd.snd) tl (x :: hd :: tl))
@[simp]
theorem free_group.reduce.cons {α : Type u} {L : list × bool)} [decidable_eq α] (x : α × bool) :
free_group.reduce (x :: L) = (free_group.reduce L).cases_on [x] (λ (hd : α × bool) (tl : list × bool)), ite (x.fst = hd.fst x.snd = !hd.snd) tl (x :: hd :: tl))

The first theorem that characterises the function reduce: a word reduces to its maximal reduction.

The first theorem that characterises the function reduce: a word reduces to its maximal reduction.

theorem free_add_group.reduce.not {α : Type u} [decidable_eq α] {p : Prop} {L₁ L₂ L₃ : list × bool)} {x : α} {b : bool} :
free_add_group.reduce L₁ = L₂ ++ (x, b) :: (x, !b) :: L₃ p
theorem free_group.reduce.not {α : Type u} [decidable_eq α] {p : Prop} {L₁ L₂ L₃ : list × bool)} {x : α} {b : bool} :
free_group.reduce L₁ = L₂ ++ (x, b) :: (x, !b) :: L₃ p
theorem free_add_group.reduce.min {α : Type u} {L₁ L₂ : list × bool)} [decidable_eq α] (H : free_add_group.red (free_add_group.reduce L₁) L₂) :

The second theorem that characterises the function reduce: the maximal reduction of a word only reduces to itself.

theorem free_group.reduce.min {α : Type u} {L₁ L₂ : list × bool)} [decidable_eq α] (H : free_group.red (free_group.reduce L₁) L₂) :

The second theorem that characterises the function reduce: the maximal reduction of a word only reduces to itself.

@[simp]

reduce is idempotent, i.e. the maximal reduction of the maximal reduction of a word is the maximal reduction of the word.

@[simp]

reduce is idempotent, i.e. the maximal reduction of the maximal reduction of a word is the maximal reduction of the word.

theorem free_group.reduce.step.eq {α : Type u} {L₁ L₂ : list × bool)} [decidable_eq α] (H : free_group.red.step L₁ L₂) :
theorem free_add_group.reduce.eq_of_red {α : Type u} {L₁ L₂ : list × bool)} [decidable_eq α] (H : free_add_group.red L₁ L₂) :

If a word reduces to another word, then they have a common maximal reduction.

theorem free_group.reduce.eq_of_red {α : Type u} {L₁ L₂ : list × bool)} [decidable_eq α] (H : free_group.red L₁ L₂) :

If a word reduces to another word, then they have a common maximal reduction.

theorem free_group.red.reduce_eq {α : Type u} {L₁ L₂ : list × bool)} [decidable_eq α] (H : free_group.red L₁ L₂) :

Alias of free_group.reduce.eq_of_red.

theorem free_add_group.red.reduce_right {α : Type u} {L₁ L₂ : list × bool)} [decidable_eq α] (h : free_add_group.red L₁ L₂) :
theorem free_group.red.reduce_right {α : Type u} {L₁ L₂ : list × bool)} [decidable_eq α] (h : free_group.red L₁ L₂) :
theorem free_add_group.red.reduce_left {α : Type u} {L₁ L₂ : list × bool)} [decidable_eq α] (h : free_add_group.red L₁ L₂) :
theorem free_group.red.reduce_left {α : Type u} {L₁ L₂ : list × bool)} [decidable_eq α] (h : free_group.red L₁ L₂) :
theorem free_group.reduce.sound {α : Type u} {L₁ L₂ : list × bool)} [decidable_eq α] (H : free_group.mk L₁ = free_group.mk L₂) :

If two words correspond to the same element in the free group, then they have a common maximal reduction. This is the proof that the function that sends an element of the free group to its maximal reduction is well-defined.

If two words correspond to the same element in the additive free group, then they have a common maximal reduction. This is the proof that the function that sends an element of the free group to its maximal reduction is well-defined.

If two words have a common maximal reduction, then they correspond to the same element in the additive free group.

theorem free_group.reduce.exact {α : Type u} {L₁ L₂ : list × bool)} [decidable_eq α] (H : free_group.reduce L₁ = free_group.reduce L₂) :

If two words have a common maximal reduction, then they correspond to the same element in the free group.

A word and its maximal reduction correspond to the same element of the free group.

A word and its maximal reduction correspond to the same element of the additive free group.

theorem free_group.reduce.rev {α : Type u} {L₁ L₂ : list × bool)} [decidable_eq α] (H : free_group.red L₁ L₂) :

If words w₁ w₂ are such that w₁ reduces to w₂, then w₂ reduces to the maximal reduction of w₁.

theorem free_add_group.reduce.rev {α : Type u} {L₁ L₂ : list × bool)} [decidable_eq α] (H : free_add_group.red L₁ L₂) :

If words w₁ w₂ are such that w₁ reduces to w₂, then w₂ reduces to the maximal reduction of w₁.

The function that sends an element of the additive free group to its maximal reduction.

Equations
def free_group.to_word {α : Type u} [decidable_eq α] :

The function that sends an element of the free group to its maximal reduction.

Equations
@[simp]
theorem free_group.to_word_inj {α : Type u} [decidable_eq α] {x y : free_group α} :
@[simp]
theorem free_add_group.to_word_inj {α : Type u} [decidable_eq α] {x y : free_add_group α} :
@[simp]
@[simp]
theorem free_group.to_word_mk {α : Type u} {L₁ : list × bool)} [decidable_eq α] :
@[simp]
@[simp]
theorem free_group.to_word_eq_nil_iff {α : Type u} [decidable_eq α] {x : free_group α} :
def free_group.reduce.church_rosser {α : Type u} {L₁ L₂ L₃ : list × bool)} [decidable_eq α] (H12 : free_group.red L₁ L₂) (H13 : free_group.red L₁ L₃) :
{L₄ // free_group.red L₂ L₄ free_group.red L₃ L₄}

Constructive Church-Rosser theorem (compare church_rosser).

Equations
def free_add_group.reduce.church_rosser {α : Type u} {L₁ L₂ L₃ : list × bool)} [decidable_eq α] (H12 : free_add_group.red L₁ L₂) (H13 : free_add_group.red L₁ L₃) :
{L₄ // free_add_group.red L₂ L₄ free_add_group.red L₃ L₄}

Constructive Church-Rosser theorem (compare church_rosser).

Equations
@[protected, instance]
Equations
@[protected, instance]
Equations
@[protected, instance]
Equations
def free_group.red.enum {α : Type u} [decidable_eq α] (L₁ : list × bool)) :
list (list × bool))

A list containing every word that w₁ reduces to.

Equations
theorem free_group.red.enum.sound {α : Type u} {L₁ L₂ : list × bool)} [decidable_eq α] (H : L₂ free_group.red.enum L₁) :
free_group.red L₁ L₂
theorem free_group.red.enum.complete {α : Type u} {L₁ L₂ : list × bool)} [decidable_eq α] (H : free_group.red L₁ L₂) :
@[protected, instance]
def free_group.subtype.fintype {α : Type u} {L₁ : list × bool)} [decidable_eq α] :
fintype {L₂ // free_group.red L₁ L₂}
Equations
def free_add_group.norm {α : Type u} [decidable_eq α] (x : free_add_group α) :

The length of reduced words provides a norm on an additive free group.

Equations
def free_group.norm {α : Type u} [decidable_eq α] (x : free_group α) :

The length of reduced words provides a norm on a free group.

Equations
@[simp]
theorem free_group.norm_inv_eq {α : Type u} [decidable_eq α] {x : free_group α} :
@[simp]
theorem free_add_group.norm_neg_eq {α : Type u} [decidable_eq α] {x : free_add_group α} :
(-x).norm = x.norm
@[simp]
theorem free_add_group.norm_eq_zero {α : Type u} [decidable_eq α] {x : free_add_group α} :
x.norm = 0 x = 0
@[simp]
theorem free_group.norm_eq_zero {α : Type u} [decidable_eq α] {x : free_group α} :
x.norm = 0 x = 1
@[simp]
theorem free_group.norm_one {α : Type u} [decidable_eq α] :
1.norm = 0
@[simp]
theorem free_add_group.norm_zero {α : Type u} [decidable_eq α] :
0.norm = 0
theorem free_group.norm_mk_le {α : Type u} {L₁ : list × bool)} [decidable_eq α] :
theorem free_add_group.norm_mk_le {α : Type u} {L₁ : list × bool)} [decidable_eq α] :
theorem free_add_group.norm_add_le {α : Type u} [decidable_eq α] (x y : free_add_group α) :
(x + y).norm x.norm + y.norm
theorem free_group.norm_mul_le {α : Type u} [decidable_eq α] (x y : free_group α) :
(x * y).norm x.norm + y.norm