Lemmas about subgroups within the permutations (self-equivalences) of a type α
#
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
This file provides extra lemmas about some subgroup
s that exist within equiv.perm α
.
group_theory.subgroup
depends on group_theory.perm.basic
, so these need to be in a separate
file.
It also provides decidable instances on membership in these subgroups, since
monoid_hom.decidable_mem_range
cannot be inferred without the help of a lambda.
The presence of these instances induces a fintype
instance on the quotient_group.quotient
of
these subgroups.
Equations
- equiv.perm.sum_congr_hom.decidable_mem_range = λ (x : equiv.perm (α ⊕ β)), infer_instance
Equations
- equiv.perm.sigma_congr_right_hom.decidable_mem_range = λ (x : equiv.perm (Σ (a : α), β a)), infer_instance
Equations
Cayley's theorem: Every group G is isomorphic to a subgroup of the symmetric group acting on
G
. Note that we generalize this to an arbitrary "faithful" group action by G
. Setting H = G
recovers the usual statement of Cayley's theorem via right_cancel_monoid.to_has_faithful_smul