Documentation

Mathlib.GroupTheory.Perm.Option

Permutations of Option α #

@[simp]
@[simp]
theorem Equiv.optionCongr_swap {α : Type u_1} [DecidableEq α] (x y : α) :
@[simp]
theorem Equiv.optionCongr_sign {α : Type u_1} [DecidableEq α] [Fintype α] (e : Equiv.Perm α) :
Equiv.Perm.sign (Equiv.optionCongr e) = Equiv.Perm.sign e
@[simp]
theorem map_equiv_removeNone {α : Type u_1} [DecidableEq α] (σ : Equiv.Perm (Option α)) :
(Equiv.removeNone σ).optionCongr = Equiv.swap none (σ none) * σ

Permutations of Option α are equivalent to fixing an Option α and permuting the remaining with a Perm α. The fixed Option α is swapped with none.

Equations
  • One or more equations did not get rendered due to their size.
Instances For
    @[simp]
    theorem Equiv.Perm.decomposeOption_apply {α : Type u_1} [DecidableEq α] (σ : Equiv.Perm (Option α)) :
    Equiv.Perm.decomposeOption σ = (σ none, Equiv.removeNone σ)
    theorem Equiv.Perm.decomposeOption_symm_sign {α : Type u_1} [DecidableEq α] [Fintype α] (e : Equiv.Perm α) :
    Equiv.Perm.sign (Equiv.Perm.decomposeOption.symm (none, e)) = Equiv.Perm.sign e

    The set of all permutations of Option α can be constructed by augmenting the set of permutations of α by each element of Option α in turn.