Cycle factors of a permutation #
Let β
be a Fintype
and f : Equiv.Perm β
.
Equiv.Perm.cycleOf
:f.cycleOf x
is the cycle off
thatx
belongs to.Equiv.Perm.cycleFactors
:f.cycleFactors
is a list of disjoint cyclic permutations that multiply tof
.
f.cycleOf x
is the cycle of the permutation f
to which x
belongs.
Equations
- f.cycleOf x = Equiv.Perm.ofSubtype (f.subtypePerm ⋯)
Instances For
x
is in the support of f
iff Equiv.Perm.cycle_of f x
is a cycle.
Given a list l : List α
and a permutation f : Perm α
whose nonfixed points are all in l
,
recursively factors f
into cycles.
Equations
- One or more equations did not get rendered due to their size.
- Equiv.Perm.cycleFactorsAux [] f h_2 = ⟨[], ⋯⟩
Instances For
Factors a permutation f
into a list of disjoint cyclic permutations that multiply to f
.
Equations
- f.cycleFactors = Equiv.Perm.cycleFactorsAux (Finset.sort (fun (x x_1 : α) => x ≤ x_1) Finset.univ) f ⋯
Instances For
Factors a permutation f
into a list of disjoint cyclic permutations that multiply to f
,
without a linear order.
Equations
- One or more equations did not get rendered due to their size.
Instances For
Factors a permutation f
into a Finset
of disjoint cyclic permutations that multiply to f
.
Equations
- One or more equations did not get rendered due to their size.
Instances For
The product of cycle factors is equal to the original f : perm α
.
Two permutations f g : Perm α
have the same cycle factors iff they are the same.
If c is a cycle, a ∈ c.support and c is a cycle of f, then c = f.cycleOf a