Isomorphisms between free groups come from equivalences of their generators #
This file proves that an isomorphism e : G ≃* H
between free groups G
and H
is induced by an
equivalence of generators.
TODO #
We currently construct the equivalence of generators, but don't show that it induces the isomorphism of groups.
A
is a basis of the ℤ-module FreeAbelianGroup A
.
Equations
- FreeAbelianGroup.basis α = { repr := (FreeAbelianGroup.equivFinsupp α).toIntLinearEquiv }
Instances For
def
Equiv.ofFreeAbelianGroupLinearEquiv
{α : Type u_1}
{β : Type u_2}
(e : FreeAbelianGroup α ≃ₗ[ℤ] FreeAbelianGroup β)
:
Isomorphic free abelian groups (as modules) have equivalent bases.
Equations
Instances For
def
Equiv.ofFreeAbelianGroupEquiv
{α : Type u_1}
{β : Type u_2}
(e : FreeAbelianGroup α ≃+ FreeAbelianGroup β)
:
Isomorphic free abelian groups (as additive groups) have equivalent bases.
Instances For
Isomorphic free groups have equivalent bases.
Equations
Instances For
def
Equiv.ofIsFreeGroupEquiv
{G : Type u_3}
{H : Type u_4}
[Group G]
[Group H]
[IsFreeGroup G]
[IsFreeGroup H]
(e : G ≃* H)
:
Isomorphic free groups have equivalent bases (IsFreeGroup
variant).