Zulip Chat Archive
Stream: mathlib4
Topic: Multiply transitive group actions, and a quest for a name
Antoine Chambert-Loir (Mar 29 2025 at 09:13):
I have two questions about #23386, in which I introduce multiply transitive group actions.
So assume that G
acts on X
.
- The fact that
G
actsn
-transitively onX
is introduced as the transitivity of the group action ofG
onFin n ↪ X
. This group action exists becauseG
is a group. On the other hand, the definition could be partly generalized to actions of monoids, using a more explicit formulation. For example for 2-transitivity, this is equivalent to `∀ {a b c d : X} (_ : a ≠ b) (_ : c ≠ d), ∃ g : G, g • a = c ∧ g • b = d, which makes sense for monoids.
Question 1. Is it worthwhile to have the more general definition?
- For showing that
n
-transitivity impliesm
-transitivity whenm ≤ n
, one needs to extend an embeddingFin m ↪ X
to an embeddingFin n ↪ X
(this requires thatX
has at leastn
elements. So I prove this:
theorem _root_.Function.Embedding.giveMeAName'
{m n : ℕ} (hmn : m ≤ n) (hn : n ≤ ENat.card X) :
Function.Surjective (fun x : Fin n ↪ X ↦ (Fin.castLEEmb hmn).trans x)
but the proof is slightly lengthy. Maybe there is a simpler way.
Question 2. How should this theorem be called?
There is an unprimed version for Finite X
where ENat.card
is replaced by Nat.card
, and I also need a name for that.
Antoine Chambert-Loir (Apr 08 2025 at 07:04):
Let me revive this question — essentially in case @Eric Wieser or @Yaël Dillies have an immediate suggestion.
Johan Commelin (Apr 08 2025 at 07:20):
Minor comment: I guess the Fin 2
in (1) should be Fin n
, right?
Last updated: May 02 2025 at 03:31 UTC