mathlib documentation

group_theory.perm.sign

def equiv.perm.subtype_perm {α : Type u} (f : equiv.perm α) {p : α → Prop} (h : ∀ (x : α), p x p (f x)) :
equiv.perm {x // p x}

Equations
@[simp]
theorem equiv.perm.subtype_perm_one {α : Type u} (p : α → Prop) (h : ∀ (x : α), p x p (1 x)) :

def equiv.perm.of_subtype {α : Type u} {p : α → Prop} [decidable_pred p] :

Equations
theorem equiv.perm.eq_inv_iff_eq {α : Type u} {f : equiv.perm α} {x y : α} :
x = f⁻¹ y f x = y

theorem equiv.perm.inv_eq_iff_eq {α : Type u} {f : equiv.perm α} {x y : α} :
f⁻¹ x = y x = f y

def equiv.perm.disjoint {α : Type u} (f g : equiv.perm α) :
Prop

Two permutations f and g are disjoint if their supports are disjoint, i.e., every element is fixed either by f, or by g.

Equations
theorem equiv.perm.disjoint.symm {α : Type u} {f g : equiv.perm α} (a : f.disjoint g) :

theorem equiv.perm.disjoint_comm {α : Type u} {f g : equiv.perm α} :

theorem equiv.perm.disjoint_mul_comm {α : Type u} {f g : equiv.perm α} (h : f.disjoint g) :
f * g = g * f

@[simp]
theorem equiv.perm.disjoint_one_left {α : Type u} (f : equiv.perm α) :

@[simp]
theorem equiv.perm.disjoint_one_right {α : Type u} (f : equiv.perm α) :

theorem equiv.perm.disjoint_mul_left {α : Type u} {f g h : equiv.perm α} (H1 : f.disjoint h) (H2 : g.disjoint h) :
(f * g).disjoint h

theorem equiv.perm.disjoint_mul_right {α : Type u} {f g h : equiv.perm α} (H1 : f.disjoint g) (H2 : f.disjoint h) :
f.disjoint (g * h)

theorem equiv.perm.disjoint_prod_right {α : Type u} {f : equiv.perm α} (l : list (equiv.perm α)) (h : ∀ (g : equiv.perm α), g lf.disjoint g) :

theorem equiv.perm.disjoint_prod_perm {α : Type u} {l₁ l₂ : list (equiv.perm α)} (hl : list.pairwise equiv.perm.disjoint l₁) (hp : l₁ ~ l₂) :
l₁.prod = l₂.prod

theorem equiv.perm.of_subtype_subtype_perm {α : Type u} {f : equiv.perm α} {p : α → Prop} [decidable_pred p] (h₁ : ∀ (x : α), p x p (f x)) (h₂ : ∀ (x : α), f x xp x) :

theorem equiv.perm.of_subtype_apply_of_not_mem {α : Type u} {p : α → Prop} [decidable_pred p] (f : equiv.perm (subtype p)) {x : α} (hx : ¬p x) :

theorem equiv.perm.mem_iff_of_subtype_apply_mem {α : Type u} {p : α → Prop} [decidable_pred p] (f : equiv.perm (subtype p)) (x : α) :

@[simp]
theorem equiv.perm.subtype_perm_of_subtype {α : Type u} {p : α → Prop} [decidable_pred p] (f : equiv.perm (subtype p)) :

theorem equiv.perm.pow_apply_eq_self_of_apply_eq_self {α : Type u} {f : equiv.perm α} {x : α} (hfx : f x = x) (n : ) :
(f ^ n) x = x

theorem equiv.perm.gpow_apply_eq_self_of_apply_eq_self {α : Type u} {f : equiv.perm α} {x : α} (hfx : f x = x) (n : ) :
(f ^ n) x = x

theorem equiv.perm.pow_apply_eq_of_apply_apply_eq_self {α : Type u} {f : equiv.perm α} {x : α} (hffx : f (f x) = x) (n : ) :
(f ^ n) x = x (f ^ n) x = f x

theorem equiv.perm.gpow_apply_eq_of_apply_apply_eq_self {α : Type u} {f : equiv.perm α} {x : α} (hffx : f (f x) = x) (i : ) :
(f ^ i) x = x (f ^ i) x = f x

def equiv.perm.support {α : Type u} [decidable_eq α] [fintype α] (f : equiv.perm α) :

Equations
@[simp]
theorem equiv.perm.mem_support {α : Type u} [decidable_eq α] [fintype α] {f : equiv.perm α} {x : α} :
x f.support f x x

def equiv.perm.is_swap {α : Type u} [decidable_eq α] (f : equiv.perm α) :
Prop

Equations
theorem equiv.perm.swap_mul_eq_mul_swap {α : Type u} [decidable_eq α] (f : equiv.perm α) (x y : α) :
(equiv.swap x y) * f = f * equiv.swap (f⁻¹ x) (f⁻¹ y)

theorem equiv.perm.mul_swap_eq_swap_mul {α : Type u} [decidable_eq α] (f : equiv.perm α) (x y : α) :
f * equiv.swap x y = (equiv.swap (f x) (f y)) * f

@[simp]
theorem equiv.perm.swap_mul_self_mul {α : Type u} [decidable_eq α] (i j : α) (σ : equiv.perm α) :
(equiv.swap i j) * (equiv.swap i j) * σ = σ

Multiplying a permutation with swap i j twice gives the original permutation.

This specialization of swap_mul_self is useful when using cosets of permutations.

theorem equiv.perm.swap_mul_eq_iff {α : Type u} [decidable_eq α] {i j : α} {σ : equiv.perm α} :
(equiv.swap i j) * σ = σ i = j

theorem equiv.perm.is_swap_of_subtype {α : Type u} [decidable_eq α] {p : α → Prop} [decidable_pred p] {f : equiv.perm (subtype p)} (h : f.is_swap) :

theorem equiv.perm.ne_and_ne_of_swap_mul_apply_ne_self {α : Type u} [decidable_eq α] {f : equiv.perm α} {x y : α} (hy : ((equiv.swap x (f x)) * f) y y) :
f y y y x

theorem equiv.perm.support_swap_mul_eq {α : Type u} [decidable_eq α] [fintype α] {f : equiv.perm α} {x : α} (hffx : f (f x) x) :
((equiv.swap x (f x)) * f).support = f.support.erase x

theorem equiv.perm.card_support_swap_mul {α : Type u} [decidable_eq α] [fintype α] {f : equiv.perm α} {x : α} (hx : f x x) :

def equiv.perm.swap_factors_aux {α : Type u} [decidable_eq α] (l : list α) (f : equiv.perm α) (a : ∀ {x : α}, f x xx l) :
{l // l.prod = f ∀ (g : equiv.perm α), g l → g.is_swap}

Equations
def equiv.perm.swap_factors {α : Type u} [decidable_eq α] [fintype α] [decidable_linear_order α] (f : equiv.perm α) :
{l // l.prod = f ∀ (g : equiv.perm α), g l → g.is_swap}

swap_factors represents a permutation as a product of a list of transpositions. The representation is non unique and depends on the linear order structure. For types without linear order trunc_swap_factors can be used

Equations
def equiv.perm.trunc_swap_factors {α : Type u} [decidable_eq α] [fintype α] (f : equiv.perm α) :
trunc {l // l.prod = f ∀ (g : equiv.perm α), g l → g.is_swap}

Equations
theorem equiv.perm.swap_induction_on {α : Type u} [decidable_eq α] [fintype α] {P : equiv.perm α → Prop} (f : equiv.perm α) (a : P 1) (a_1 : ∀ (f : equiv.perm α) (x y : α), x yP fP ((equiv.swap x y) * f)) :
P f

theorem equiv.perm.swap_mul_swap_mul_swap {α : Type u} [decidable_eq α] {x y z : α} (hwz : x y) (hxz : x z) :

theorem equiv.perm.is_conj_swap {α : Type u} [decidable_eq α] {w x y z : α} (hwx : w x) (hyz : y z) :

def equiv.perm.fin_pairs_lt (n : ) :
finset (Σ (a : fin n), fin n)

set of all pairs (⟨a, b⟩ : Σ a : fin n, fin n) such that b < a

Equations
theorem equiv.perm.mem_fin_pairs_lt {n : } {a : Σ (a : fin n), fin n} :

def equiv.perm.sign_aux {n : } (a : equiv.perm (fin n)) :

Equations
@[simp]
theorem equiv.perm.sign_aux_one (n : ) :

def equiv.perm.sign_bij_aux {n : } (f : equiv.perm (fin n)) (a : Σ (a : fin n), fin n) :
Σ (a : fin n), fin n

Equations
theorem equiv.perm.sign_bij_aux_inj {n : } {f : equiv.perm (fin n)} (a b : Σ (a : fin n), fin n) (a_1 : a equiv.perm.fin_pairs_lt n) (a_2 : b equiv.perm.fin_pairs_lt n) (a_3 : f.sign_bij_aux a = f.sign_bij_aux b) :
a = b

theorem equiv.perm.sign_bij_aux_surj {n : } {f : equiv.perm (fin n)} (a : Σ (a : fin n), fin n) (H : a equiv.perm.fin_pairs_lt n) :
∃ (b : Σ (a : fin n), fin n) (H : b equiv.perm.fin_pairs_lt n), a = f.sign_bij_aux b

@[simp]

theorem equiv.perm.sign_aux_mul {n : } (f g : equiv.perm (fin n)) :

theorem equiv.perm.sign_aux_swap {n : } {x y : fin n} (hxy : x y) :

def equiv.perm.sign_aux2 {α : Type u} [decidable_eq α] (a : list α) (a_1 : equiv.perm α) :

Equations
theorem equiv.perm.sign_aux_eq_sign_aux2 {α : Type u} [decidable_eq α] {n : } (l : list α) (f : equiv.perm α) (e : α fin n) (h : ∀ (x : α), f x xx l) :

def equiv.perm.sign_aux3 {α : Type u} [decidable_eq α] [fintype α] (f : equiv.perm α) {s : multiset α} (a : ∀ (x : α), x s) :

Equations
theorem equiv.perm.sign_aux3_mul_and_swap {α : Type u} [decidable_eq α] [fintype α] (f g : equiv.perm α) (s : multiset α) (hs : ∀ (x : α), x s) :
(f * g).sign_aux3 hs = (f.sign_aux3 hs) * g.sign_aux3 hs ∀ (x y : α), x y(equiv.swap x y).sign_aux3 hs = -1

def equiv.perm.sign {α : Type u} [decidable_eq α] [fintype α] :

sign of a permutation returns the signature or parity of a permutation, 1 for even permutations, -1 for odd permutations. It is the unique surjective group homomorphism from perm α to the group with two elements.

Equations
@[simp]

@[simp]
theorem equiv.perm.sign_one {α : Type u} [decidable_eq α] [fintype α] :

@[simp]
theorem equiv.perm.sign_refl {α : Type u} [decidable_eq α] [fintype α] :

@[simp]

theorem equiv.perm.sign_swap {α : Type u} [decidable_eq α] [fintype α] {x y : α} (h : x y) :

@[simp]
theorem equiv.perm.sign_swap' {α : Type u} [decidable_eq α] [fintype α] {x y : α} :
equiv.perm.sign (equiv.swap x y) = ite (x = y) 1 (-1)

theorem equiv.perm.sign_eq_of_is_swap {α : Type u} [decidable_eq α] [fintype α] {f : equiv.perm α} (h : f.is_swap) :

theorem equiv.perm.sign_aux3_symm_trans_trans {α : Type u} {β : Type v} [decidable_eq α] [fintype α] [decidable_eq β] [fintype β] (f : equiv.perm α) (e : α β) {s : multiset α} {t : multiset β} (hs : ∀ (x : α), x s) (ht : ∀ (x : β), x t) :

theorem equiv.perm.sign_symm_trans_trans {α : Type u} {β : Type v} [decidable_eq α] [fintype α] [decidable_eq β] [fintype β] (f : equiv.perm α) (e : α β) :

theorem equiv.perm.sign_prod_list_swap {α : Type u} [decidable_eq α] [fintype α] {l : list (equiv.perm α)} (hl : ∀ (g : equiv.perm α), g l → g.is_swap) :

theorem equiv.perm.sign_subtype_perm {α : Type u} [decidable_eq α] [fintype α] (f : equiv.perm α) {p : α → Prop} [decidable_pred p] (h₁ : ∀ (x : α), p x p (f x)) (h₂ : ∀ (x : α), f x xp x) :

theorem equiv.perm.sign_eq_sign_of_equiv {α : Type u} {β : Type v} [decidable_eq α] [fintype α] [decidable_eq β] [fintype β] (f : equiv.perm α) (g : equiv.perm β) (e : α β) (h : ∀ (x : α), e (f x) = g (e x)) :

theorem equiv.perm.sign_bij {α : Type u} {β : Type v} [decidable_eq α] [fintype α] [decidable_eq β] [fintype β] {f : equiv.perm α} {g : equiv.perm β} (i : Π (x : α), f x x → β) (h : ∀ (x : α) (hx : f x x) (hx' : f (f x) f x), i (f x) hx' = g (i x hx)) (hi : ∀ (x₁ x₂ : α) (hx₁ : f x₁ x₁) (hx₂ : f x₂ x₂), i x₁ hx₁ = i x₂ hx₂x₁ = x₂) (hg : ∀ (y : β), g y y(∃ (x : α) (hx : f x x), i x hx = y)) :

def equiv.perm.is_cycle {β : Type v} (f : equiv.perm β) :
Prop

Equations
theorem equiv.perm.is_cycle_swap {α : Type u} [decidable_eq α] [fintype α] {x y : α} (hxy : x y) :

theorem equiv.perm.is_cycle_inv {β : Type v} {f : equiv.perm β} (hf : f.is_cycle) :

theorem equiv.perm.exists_gpow_eq_of_is_cycle {β : Type v} {f : equiv.perm β} (hf : f.is_cycle) {x y : β} (hx : f x x) (hy : f y y) :
∃ (i : ), (f ^ i) x = y

theorem equiv.perm.is_cycle_swap_mul_aux₁ {α : Type u} [decidable_eq α] [fintype α] (n : ) {b x : α} {f : equiv.perm α} (hb : ((equiv.swap x (f x)) * f) b b) (h : (f ^ n) (f x) = b) :
∃ (i : ), (((equiv.swap x (f x)) * f) ^ i) (f x) = b

theorem equiv.perm.is_cycle_swap_mul_aux₂ {α : Type u} [decidable_eq α] [fintype α] (n : ) {b x : α} {f : equiv.perm α} (hb : ((equiv.swap x (f x)) * f) b b) (h : (f ^ n) (f x) = b) :
∃ (i : ), (((equiv.swap x (f x)) * f) ^ i) (f x) = b

theorem equiv.perm.eq_swap_of_is_cycle_of_apply_apply_eq_self {α : Type u} [decidable_eq α] [fintype α] {f : equiv.perm α} (hf : f.is_cycle) {x : α} (hfx : f x x) (hffx : f (f x) = x) :
f = equiv.swap x (f x)

theorem equiv.perm.is_cycle_swap_mul {α : Type u} [decidable_eq α] [fintype α] {f : equiv.perm α} (hf : f.is_cycle) {x : α} (hx : f x x) (hffx : f (f x) x) :
((equiv.swap x (f x)) * f).is_cycle

@[simp]
theorem equiv.perm.support_swap {α : Type u} [decidable_eq α] [_inst_2 _inst_3 : fintype α] {x y : α} (hxy : x y) :
(equiv.swap x y).support = {x, y}

theorem equiv.perm.card_support_swap {α : Type u} [decidable_eq α] [_inst_2 _inst_3 : fintype α] {x y : α} (hxy : x y) :

theorem equiv.perm.sign_cycle {α : Type u} [decidable_eq α] [_inst_2 _inst_3 : fintype α] {f : equiv.perm α} (hf : f.is_cycle) :