Documentation

Mathlib.GroupTheory.Perm.Option

Permutations of Option α #

@[simp]
theorem Equiv.optionCongr_one {α : Type u_1} :
@[simp]
theorem Equiv.optionCongr_swap {α : Type u_1} [DecidableEq α] (x y : α) :
optionCongr (swap x y) = swap (some x) (some y)
@[simp]
theorem Equiv.optionCongr_sign {α : Type u_1} [DecidableEq α] [Fintype α] (e : Perm α) :

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

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