Skip to content

Commit

Permalink
feat(group_theory/free_product): is_free_group_free_product_of_is_fre…
Browse files Browse the repository at this point in the history
…e_group (#12125)
  • Loading branch information
nomeata committed Feb 21, 2022
1 parent 7c6678a commit 2f33463
Showing 1 changed file with 16 additions and 0 deletions.
16 changes: 16 additions & 0 deletions src/group_theory/free_product.lean
Expand Up @@ -5,6 +5,7 @@ Authors: David Wärn
-/
import algebra.free_monoid
import group_theory.congruence
import group_theory.is_free_group
import data.list.chain
/-!
# The free product of groups or monoids
Expand Down Expand Up @@ -327,4 +328,19 @@ instance : decidable_eq (free_product M) := word.equiv.decidable_eq

end word

/-- The free product of free groups is itself a free group -/
@[simps]
instance {ι : Type*} (G : ι → Type*) [∀ i, group (G i)] [hG : ∀ i, is_free_group (G i)] :
is_free_group (free_product G) :=
{ generators := Σ i, is_free_group.generators (G i),
of := λ x, free_product.of (is_free_group.of x.2),
unique_lift' :=
begin
introsI X _ f,
refine ⟨free_product.lift (λ i, is_free_group.lift (λ x, f ⟨i, x⟩)), _ ⟩,
split,
{ simp, },
{ intros g hfg, ext i x, simpa using hfg ⟨i, x⟩, }
end, }

end free_product

0 comments on commit 2f33463

Please sign in to comment.