module Algebra.Group.Cayley {ℓ} (G : Group ℓ) where
open Group-on (G .snd) renaming (underlying-set to G-set)
Cayley’s theorem🔗
Cayley’s theorem says that any group admits a representation as a subgroup of a symmetric group, specifically the symmetric group acting on the underlying set of
First, recall that we get a family of equivalences by multiplication on the left, the principal action of on itself:
: ⌞ G ⌟ → ⌞ G ⌟ ≃ ⌞ G ⌟
Cayley = (λ y → x ⋆ y) , ⋆-equivl x Cayley x
We then show that this map is a group homomorphism from to
: is-group-hom (G .snd) (Sym G-set) Cayley
Cayley-is-hom .is-group-hom.pres-⋆ x y = ext λ e → sym associative Cayley-is-hom
Finally, we show that this map is injective; Thus,
embeds as a subgroup of
(the image of Cayley
).
: injective Cayley
Cayley-injective {x} {y} eqvs-equal =
Cayley-injective
x ≡⟨ sym idr ⟩
x ⋆ unit ≡⟨⟩.fst unit ≡⟨ happly (ap fst eqvs-equal) unit ⟩
Cayley x .fst unit ≡⟨⟩
Cayley y
y ⋆ unit ≡⟨ idr ⟩ y ∎