Exploration 5: Permutation groups
November 16, 2023.Questions:
- TODO
Recall that a permutation of a set is a reordering of elements and is usually written like . Given an arbitrary set , the permutations on the set are written .
This notation is called cycle notation; is a cycle. More complex permutations are composed of cycles: the permutation maps and . Ordering matters: the rightmost permutation is performed first.
The identity permutation (which does nothing to the set) can be written as a length cycle, like .
Composing permutations
Consider the permutation . This first swaps and , and then swaps and . Since the net effect is the same as the cycle , we consider them to be the same permutation. That is, the set is a single-element set.
Permutations can be used to represent groups. Here’s how:
- If is finite, there is a bijection from to the set via renaming.
- We can imagine transforming every to be a permutation in . Such a permutation would start from , go to via the bijection, apply , and go back to via the bijection.
- Then .
- We need to find an injective homomorphism
between a finite group
and
.
If we can, then
.
- by injectivity, so , so is some permutation group, so we are done.
- Define (left-product with ). Since this map is invertible (by left-product with ), it results in a permutation of elements, i.e. an element of .
- is a homomorphism, since applying left product of then left product of is the same as applying left product of .
- is obviously one-to-one from its definition, i.e. given two maps and , if they are equal we must have .
- Then is an injective homomorphism, so we are done.
The implication of Cayley’s theorem is: to study the groups of order , we need only study the symmetric group .
Motivating example: . Proof. For every , .
This proof is simple but required knowledge of cyclic groups, namely that every can be represented as g^k for some . But using only the fact that is finite, we can ignore everything about cyclic groups and use Cayley’s theorem to reduce the proof to one about permutation groups.
Proof. Since is finite, by Cayley’s theorem it is isomorphic to a permutation group . We know that . Taking the image of this theorem via the isomorphism gives us .
What kinds of problems can we reduce to permutation group problems? Any problem involving finite groups! This may not always be a good move, since the permutation group can have up to elements (a lot). But in general, we can now use theorems about permutation groups in any problem about finite groups.
In this section, we show how we can use groups to permute sets.
Given a group and a set , define the product as the left action of on . It takes an element and maps an element of to another element of .
The idea behind these group actions is that each element of permutes the elements of in some way, so that the product of two permutations (two elements of ) is like doing one permutation after the other, with being the identity permutation.
For example, let’s have act on elements of the set . The table might look like this:
1 2 3
(1) | 1 2 3
(1 2) | 2 1 3
(1 3) | 3 2 1
(2 3) | 1 3 2
(1 2 3) | 2 3 1
(1 3 2) | 3 1 2
Here I picked an ordering of the elements in the set and arbitrarily named the permutations of .
Every (finite) group action is just a natural group action of permutation groups
In the abstract, where each element actually gets permuted to is immaterial – a group action just needs to behave like a permutation (identity, composition, inverses).
Let’s expand on this. Given an arbitrary group acting on an arbitrary set (both finite), we can use the table representation above (with elements of as rows and elements of as columns) to show that the action of on naturally turns out to be permutations, if successive group actions are to follow the composition and inverse laws.
TODO mention cayley tables somewhere with the following facts
- if the cayley table is symmetric about the main diagonal, then the group is abelian
- TODO
Example and . We can let the action be anything (even trivial, fixing all of X) but let’s explore our choices. Draw the empty Cayley table, knowing that must be identity:
e g g²
e | e g g²
a |
b |
c |
Each row must contain a permutation of . This is a natural consequence of the inverse law: every permutation must be reversible, so you can’t lose information by dropping one of those elements after a permutation.
In our example, since each element in is self-inverse (order ), we can only treat them as permutations looking like this:
1 2 3
() | 1 2 3
(1 2) | 2 1 3
(1 3) | 3 2 1
(2 3) | 1 3 2
after bijectively mapping each element of to a natural number, and mapping each to one of . (I picked the mapping arbitrarily here.)
We only need to define the action on some set of generators of , then the other rows can be derived by composition. Thus, the process for defining a group action works in general like this:
- Map each element to a natural number
- Map each generating element to a permutation with the same order as
which falls out naturally because must follow the composition and inverse laws.
In this section, we visit the properties of group actions.
Recall the natural group action of acting on elements of the set .
1 2 3
(1) | 1 2 3
(1 2) | 2 1 3
(1 3) | 3 2 1
(2 3) | 1 3 2
(1 2 3) | 2 3 1
(1 3 2) | 3 1 2
The permutations fix , the permutations fix , and {(1),(1~2)} fixes . Call these sets , , — they are the stabilizers of , , respectively. Concretely, the stabilizer of an element is all the elements of that fix .
The orbit of (denoted , sometimes ) is the set of all elements can get mapped to. Here, each of , , is able to reach all of , , , so for all , the orbit . Since everything in can reach everything in , there is only one orbit. When an action can take every element to every element like this, and therefore there is one orbit, we call it transitive.
For a non-transitive example, consider the action of on the power set of :
{} {1} {2} {3} {1,2} {1,3} {2,3} {1,2,3}
(1) | {} {1} {2} {3} {1,2} {1,3} {2,3} {1,2,3}
(1 2) | {} {2} {1} {3} {1,2} {2,3} {1,3} {1,2,3}
(1 3) | {} {3} {2} {1} {2,3} {1,3} {1,2} {1,2,3}
(2 3) | {} {1} {3} {2} {1,3} {1,2} {2,3} {1,2,3}
(1 2 3) | {} {2} {3} {1} {2,3} {1,2} {1,3} {1,2,3}
(1 3 2) | {} {3} {1} {2} {1,3} {2,3} {1,2} {1,2,3}
You can see that maps only to , etc. In this example, the orbits of each element in consists of all the sets with the same number of elements.
- Define the relation on where whenever are in the same orbit. Since it just checks set inclusion, trivially satisfies the properties of an equivalence relation.
- Since is an equivalence relation, it partitions into equivalence classes.
Corollary: Elements of act on by permuting each orbit separately.
When for every pair , it is the same as saying that every can reach every via , i.e. the action is transitive.
- Since the group action is transitive, let for some fixed . Then: shows that left-multiplication by is a map between arbitrary orbits and . It is a bijection since the inverse is left-multiplication by .
- Since there is a bijection between arbitrary orbits they must all have the same cardinality.
The stabilizer of some (denoted ) is a subgroup of composed of every that permutes that to itself. Similarly, the normalizer of a subgroup (denoted ) is the subgroup of composed of every that permutes to itself.
- ()
- If a subgroup acts transitively on it means it sends every element of to every element of . That is, for every .
- Fix some and some , giving us an element . Since the group action is transitive, we may write for some . Since this we have for arbitrary , so . Since this is true for every , we know that .
- ()
- To prove acts transitively on , we need only prove for arbitrary .
- Since the group action is transitive, . But we are given , so .
- Intuitively this makes sense – if a subgroup contains a stabilizer for then it fixes , and therefore doesn’t take to every other element of .
- Note that when . So if acts transitively on but contains any stabilizer for some , then you can show : the only possible acting transitively on is itself.
- Fix some . To find the size of the orbit , we note that
- Define an equivalence relation where iff . Then whenever are in the same equivalence class under . This means each equivalence class corresponds to a distinct element that maps to, i.e. an element of its orbit . Then the number of equivalence classes is the number of elements in the orbit, .
- This equivalence relation is the same as used in the proof of Lagrange’s theorem, so reusing the same argument in that proof, the equivalence classes all have the same size which divides . Therefore the number of equivalence classes is .
- Therefore, number of equivalence classes .
In this section, we study two possible actions of groups on themselves.
Consider a group acting on itself: .
An action of on is transitive iff for every , for some . In this case both , so we can let to make the above equation always true.
- An element is in the stabilizer of iff .
- In this case, is an element in , so we right-multiply by the inverse to get .
- Then the only stabilizer of any is the identity element, so all stabilizers are trivial.
Now consider a finite group acting on itself by conjugation: . This is different from the left-multiplication definition of group action we had earlier. In fact, a group action doesn’t have to be finite or necessarily permute the elements – it just needs to be faithful, meaning there is only one identity in , and it needs to follow the group laws. An action is faithful if the intersection of all the stabilizers for is identity .
- For a conjugation group action of on itself, an element is in the intersection of all stabilizers iff for every element , . In other words, commutes with every element .
- So if the center is trivial, the intersection of all stabilizers is trivial, so the action is faithful.
The orbits of a conjugation group action of on itself are, for each element , all the elements for . But this is exactly the definition of the conjugacy classes of .
A centralizer of (denoted ) is the subgroup of that commutes with .
For a conjugation group action, an element is in the stabilizer of iff , i.e. commutes with . But this is exactly the definition of the centralizer of .
- (): if is a conjugate of then for some . But if either or is in the center (say ), then . Since when either is in the center, elements in the center end up in singleton conjugacy classes.
- (): if is in a singleton conjugacy class, for all , which means for all , so is in the center.
A group action is transitive if there is only one orbit. But since identity is always central and therefore has a singleton orbit, there are orbits outside the identity orbit, so long as the group is not trivial.
We can define at the class equation of a group action. For a group action of on , given each as a representative of each non-singleton orbit , and the number of fixpoints (singleton orbits), we have
Here’s how we arrive at the class equation:
- If you take the union of all orbits, you get the set .
- Orbits are disjoint, so you can split into the set of singleton orbits (fixpoints) and all non-singleton orbits to get .
- By orbit-stabilizer theorem, we know .
- Therefore, .
In particular, if the group action in question is the conjugation action of a group on itself, we can recover the original class equation of a group:
misc notes
Class Equation Let G be a finite group and G ~ G by conjugation: y - x := yxy~! » the orbits are the conjugacy classes » the stabilizers are centralizers Gx = {y in G | yxy^-1} = Z_G(x) » the singleton orbits are the elements of the center Z(G)={z in G | zg=gz forall g in G} Class Eqn: If xᵢ are representatives all non-central conjugacy classes in G then |G| = |Z(G)| + ∑ᵢ [G: Z_G(xᵢ)]
Consider an arbitrary part of a cycle in — in other words, . But then shows that the corresponding part of the cycle in is .
Corollary: Permutations of the same cycle type are in the same conjugacy class. Permutations of different cycle types are in different conjugacy classes.
- Consider the conjugation action on . By the orbit-stabilizer theorem, we have for an arbitrary permutation in .
- The stabilizer
may or may not contain odd permutations.
- If it contains no odd permutations, then it is completely contained in , and so we have halving the orbit (the conjugacy class) of .
- If it contains some odd permutation, then note that . Is it the case that this implies is half of ? In that case, we have , meaning the orbit (the conjugacy class) stays the same.
- Therefore, conjugacy classes in may or may not split into conjugacy classes in .
- consists of even permutations (formed by an even number of transpositions.) Such permutations are either a -cycle , a -cycle , or a product of two disjoint -cycles .
- To count the conjugacy classes in
,
we first count these permutations’ conjugacy classes in
,
since in
permutations
of the same cycle type are conjugate to each other.
- -cycles: two ways to arrange three elements, of which you have choices.
- -cycles: for each of choices of five elements, rotations of the cycle lead to the same cycle, so there are
- Cycle type : There are choices for each -cycle, and order doesn’t matter, so there are of these.
- Identity: The identity element is always in its own conjugacy class.
- This accounts for all of the permutations of . Now in some conjugacy classes may split into two, because we now lack odd permutations to conjugate by. Let’s assume that the class sizes split into . (In reality, the size class of -cycles doesn’t split.)
- Normal subgroups are unions of conjugacy classes that include the identity permutation. Given that the sizes of the non-identity conjugacy classes are at worst , the possible normal subgroup orders are .
- By Lagrange’s theorem, the order of a subgroup must divide the order of the group. Since , the only possible subgroup orders are its divisors .
- The only common orders of the above two lists are order (the trivial group) and ( itself). So they are the only normal subgroups, and thus is simple.
Exploration 4: Homomorphisms