The SubMulAction of the stabilizer of a point on the complement of that point #
When a group G
acts on a type α
, the stabilizer of a point a : α
acts naturally on the complement of that point.
Such actions (as the similar one for the fixator of a set acting on the complement
of that set, defined in Mathlib.GroupTheory.GroupAction.SubMulAction.OfFixingSubgroup
)
are useful to study the multiple transitivity of the group G
,
since n
-transitivity of G
on α
is equivalent to n - 1
-transitivity
of stabilizer G a
on the complement of a
.
We define equivariant maps that relate various of these sub_mul_actions and permit to manipulate them in a relatively smooth way.
SubMulAction.ofStabilizer a
: the action ofstabilizer G a
on{a}ᶜ
SubMulAction.Enat_card_ofStabilizer_eq_add_one
,SubMulAction.nat_card_ofStabilizer_eq
compute the cardinality of thecarrier
of that action.
Consider a b : α
and g : G
such that hg : g • b = a
.
SubMulAction.conjMap hg
is the equivariant map fromSubMulAction.ofStabilizer G a
toSubMulAction.ofStabilizer G b
.SubMulAction.ofStabilizer.isPretransitive_iff_conj hg
shows that this actions are equivalently pretransitive orSubMulAction.ofStabilizer.isMultiplyPretransitive_iff_conj hg
shows that this actions are equivalentlyn
-pretransitive for alln : ℕ
.SubMulAction.ofStabilizer.append
: givenx : Fin n ↪ ofStabilizer G a
, appenda
to obtainy : Fin n.succ ↪ α
SubMulAction.ofStabilizer.isMultiplyPretransitive_iff
: is the action ofG
onα
is pretransitive, then it isn.succ
pretransitive if and only if the action ofstabilizer G a
onofStabilizer G a
isn
-pretransitive.
Action of the stabilizer of a point on the complement.
Instances For
Action of the stabilizer of a point on the complement.
Instances For
Conjugation induces an equivariant map between the SubAddAction of the stabilizer of a point and that of its translate.
Equations
- SubAddAction.ofStabilizer.conjMap hg = { toFun := fun (x : ↥(SubAddAction.ofStabilizer G a)) => ⟨g +ᵥ ↑x, ⋯⟩, map_vadd' := ⋯ }
Instances For
Conjugation induces an equivariant map between the SubMulAction of the stabilizer of a point and that of its translate.
Equations
- SubMulAction.ofStabilizer.conjMap hg = { toFun := fun (x : ↥(SubMulAction.ofStabilizer G a)) => ⟨g • ↑x, ⋯⟩, map_smul' := ⋯ }
Instances For
Append a
to x : Fin n ↪ ofStabilizer G a
to get an element of Fin n.succ ↪ α
.
Equations
- SubMulAction.ofStabilizer.snoc x = Fin.Embedding.snoc (x.trans (Function.Embedding.subtype fun (x : α) => x ∈ SubMulAction.ofStabilizer G a)) ⋯
Instances For
Append a
to x : Fin n ↪ ofStabilizer G a
to get an element of Fin n.succ ↪ α
.
Equations
- SubAddAction.ofStabilizer.snoc x = Fin.Embedding.snoc (x.trans (Function.Embedding.subtype fun (x : α) => x ∈ SubAddAction.ofStabilizer G a)) ⋯