mathlib documentation

algebra.​group_action_hom

algebra.​group_action_hom

Equivariant homomorphisms

Main definitions

Notations

@[nolint]
structure mul_action_hom (M : Type u_1) [monoid M] (X : Type u_2) [mul_action M X] (Y : Type u_3) [mul_action M Y] :
Type (max u_2 u_3)

Equivariant functions.

@[instance]
def mul_action_hom.​has_coe_to_fun (M : Type u_1) [monoid M] (X : Type u_2) [mul_action M X] (Y : Type u_3) [mul_action M Y] :

Equations
@[simp]
theorem mul_action_hom.​map_smul {M : Type u_1} [monoid M] {X : Type u_2} [mul_action M X] {Y : Type u_3} [mul_action M Y] (f : X →[M] Y) (m : M) (x : X) :
f (m x) = m f x

@[ext]
theorem mul_action_hom.​ext {M : Type u_1} [monoid M] {X : Type u_2} [mul_action M X] {Y : Type u_3} [mul_action M Y] {f g : X →[M] Y} :
(∀ (x : X), f x = g x)f = g

theorem mul_action_hom.​ext_iff {M : Type u_1} [monoid M] {X : Type u_2} [mul_action M X] {Y : Type u_3} [mul_action M Y] {f g : X →[M] Y} :
f = g ∀ (x : X), f x = g x

def mul_action_hom.​id (M : Type u_1) [monoid M] {X : Type u_2} [mul_action M X] :
X →[M] X

The identity map as an equivariant map.

Equations
@[simp]
theorem mul_action_hom.​id_apply (M : Type u_1) [monoid M] {X : Type u_2} [mul_action M X] (x : X) :

def mul_action_hom.​comp {M : Type u_1} [monoid M] {X : Type u_2} [mul_action M X] {Y : Type u_3} [mul_action M Y] {Z : Type u_4} [mul_action M Z] :
(Y →[M] Z)(X →[M] Y)(X →[M] Z)

Composition of two equivariant maps.

Equations
@[simp]
theorem mul_action_hom.​comp_apply {M : Type u_1} [monoid M] {X : Type u_2} [mul_action M X] {Y : Type u_3} [mul_action M Y] {Z : Type u_4} [mul_action M Z] (g : Y →[M] Z) (f : X →[M] Y) (x : X) :
(g.comp f) x = g (f x)

@[simp]
theorem mul_action_hom.​id_comp {M : Type u_1} [monoid M] {X : Type u_2} [mul_action M X] {Y : Type u_3} [mul_action M Y] (f : X →[M] Y) :

@[simp]
theorem mul_action_hom.​comp_id {M : Type u_1} [monoid M] {X : Type u_2} [mul_action M X] {Y : Type u_3} [mul_action M Y] (f : X →[M] Y) :

The canonical map to the left cosets.

Equations
@[simp]
theorem mul_action_hom.​to_quotient_apply {G : Type u_15} [group G] (H : subgroup G) (g : G) :

@[nolint]
structure distrib_mul_action_hom (M : Type u_1) [monoid M] (A : Type u_5) [add_monoid A] [distrib_mul_action M A] (B : Type u_7) [add_monoid B] [distrib_mul_action M B] :
Type (max u_5 u_7)

Equivariant additive monoid homomorphisms.

def distrib_mul_action_hom.​to_mul_action_hom {M : Type u_1} [monoid M] {A : Type u_5} [add_monoid A] [distrib_mul_action M A] {B : Type u_7} [add_monoid B] [distrib_mul_action M B] :
(A →+[M] B)(A →[M] B)

Reinterpret an equivariant additive monoid homomorphism as an equivariant function.

def distrib_mul_action_hom.​to_add_monoid_hom {M : Type u_1} [monoid M] {A : Type u_5} [add_monoid A] [distrib_mul_action M A] {B : Type u_7} [add_monoid B] [distrib_mul_action M B] :
(A →+[M] B)A →+ B

Reinterpret an equivariant additive monoid homomorphism as an additive monoid homomorphism.

@[instance]
def distrib_mul_action_hom.​has_coe (M : Type u_1) [monoid M] (A : Type u_5) [add_monoid A] [distrib_mul_action M A] (B : Type u_7) [add_monoid B] [distrib_mul_action M B] :
has_coe (A →+[M] B) (A →+ B)

Equations
@[instance]
def distrib_mul_action_hom.​has_coe' (M : Type u_1) [monoid M] (A : Type u_5) [add_monoid A] [distrib_mul_action M A] (B : Type u_7) [add_monoid B] [distrib_mul_action M B] :
has_coe (A →+[M] B) (A →[M] B)

Equations
@[instance]
def distrib_mul_action_hom.​has_coe_to_fun (M : Type u_1) [monoid M] (A : Type u_5) [add_monoid A] [distrib_mul_action M A] (B : Type u_7) [add_monoid B] [distrib_mul_action M B] :

Equations
theorem distrib_mul_action_hom.​coe_fn_coe {M : Type u_1} [monoid M] {A : Type u_5} [add_monoid A] [distrib_mul_action M A] {B : Type u_7} [add_monoid B] [distrib_mul_action M B] (f : A →+[M] B) :

theorem distrib_mul_action_hom.​coe_fn_coe' {M : Type u_1} [monoid M] {A : Type u_5} [add_monoid A] [distrib_mul_action M A] {B : Type u_7} [add_monoid B] [distrib_mul_action M B] (f : A →+[M] B) :

@[ext]
theorem distrib_mul_action_hom.​ext {M : Type u_1} [monoid M] {A : Type u_5} [add_monoid A] [distrib_mul_action M A] {B : Type u_7} [add_monoid B] [distrib_mul_action M B] {f g : A →+[M] B} :
(∀ (x : A), f x = g x)f = g

theorem distrib_mul_action_hom.​ext_iff {M : Type u_1} [monoid M] {A : Type u_5} [add_monoid A] [distrib_mul_action M A] {B : Type u_7} [add_monoid B] [distrib_mul_action M B] {f g : A →+[M] B} :
f = g ∀ (x : A), f x = g x

@[simp]
theorem distrib_mul_action_hom.​map_zero {M : Type u_1} [monoid M] {A : Type u_5} [add_monoid A] [distrib_mul_action M A] {B : Type u_7} [add_monoid B] [distrib_mul_action M B] (f : A →+[M] B) :
f 0 = 0

@[simp]
theorem distrib_mul_action_hom.​map_add {M : Type u_1} [monoid M] {A : Type u_5} [add_monoid A] [distrib_mul_action M A] {B : Type u_7} [add_monoid B] [distrib_mul_action M B] (f : A →+[M] B) (x y : A) :
f (x + y) = f x + f y

@[simp]
theorem distrib_mul_action_hom.​map_neg {M : Type u_1} [monoid M] (A' : Type u_6) [add_group A'] [distrib_mul_action M A'] (B' : Type u_8) [add_group B'] [distrib_mul_action M B'] (f : A' →+[M] B') (x : A') :
f (-x) = -f x

@[simp]
theorem distrib_mul_action_hom.​map_sub {M : Type u_1} [monoid M] (A' : Type u_6) [add_group A'] [distrib_mul_action M A'] (B' : Type u_8) [add_group B'] [distrib_mul_action M B'] (f : A' →+[M] B') (x y : A') :
f (x - y) = f x - f y

@[simp]
theorem distrib_mul_action_hom.​map_smul {M : Type u_1} [monoid M] {A : Type u_5} [add_monoid A] [distrib_mul_action M A] {B : Type u_7} [add_monoid B] [distrib_mul_action M B] (f : A →+[M] B) (m : M) (x : A) :
f (m x) = m f x

def distrib_mul_action_hom.​id (M : Type u_1) [monoid M] {A : Type u_5} [add_monoid A] [distrib_mul_action M A] :
A →+[M] A

The identity map as an equivariant additive monoid homomorphism.

Equations
@[simp]
theorem distrib_mul_action_hom.​id_apply (M : Type u_1) [monoid M] {A : Type u_5} [add_monoid A] [distrib_mul_action M A] (x : A) :

def distrib_mul_action_hom.​comp {M : Type u_1} [monoid M] {A : Type u_5} [add_monoid A] [distrib_mul_action M A] {B : Type u_7} [add_monoid B] [distrib_mul_action M B] {C : Type u_9} [add_monoid C] [distrib_mul_action M C] :
(B →+[M] C)(A →+[M] B)(A →+[M] C)

Composition of two equivariant additive monoid homomorphisms.

Equations
@[simp]
theorem distrib_mul_action_hom.​comp_apply {M : Type u_1} [monoid M] {A : Type u_5} [add_monoid A] [distrib_mul_action M A] {B : Type u_7} [add_monoid B] [distrib_mul_action M B] {C : Type u_9} [add_monoid C] [distrib_mul_action M C] (g : B →+[M] C) (f : A →+[M] B) (x : A) :
(g.comp f) x = g (f x)

@[simp]
theorem distrib_mul_action_hom.​id_comp {M : Type u_1} [monoid M] {A : Type u_5} [add_monoid A] [distrib_mul_action M A] {B : Type u_7} [add_monoid B] [distrib_mul_action M B] (f : A →+[M] B) :

@[simp]
theorem distrib_mul_action_hom.​comp_id {M : Type u_1} [monoid M] {A : Type u_5} [add_monoid A] [distrib_mul_action M A] {B : Type u_7} [add_monoid B] [distrib_mul_action M B] (f : A →+[M] B) :

def mul_semiring_action_hom.​to_distrib_mul_action_hom {M : Type u_1} [monoid M] {R : Type u_10} [semiring R] [mul_semiring_action M R] {S : Type u_12} [semiring S] [mul_semiring_action M S] :
(R →+*[M] S)(R →+[M] S)

Reinterpret an equivariant ring homomorphism as an equivariant additive monoid homomorphism.

@[nolint]
structure mul_semiring_action_hom (M : Type u_1) [monoid M] (R : Type u_10) [semiring R] [mul_semiring_action M R] (S : Type u_12) [semiring S] [mul_semiring_action M S] :
Type (max u_10 u_12)

Equivariant ring homomorphisms.

def mul_semiring_action_hom.​to_ring_hom {M : Type u_1} [monoid M] {R : Type u_10} [semiring R] [mul_semiring_action M R] {S : Type u_12} [semiring S] [mul_semiring_action M S] :
(R →+*[M] S)R →+* S

Reinterpret an equivariant ring homomorphism as a ring homomorphism.

@[instance]
def mul_semiring_action_hom.​has_coe (M : Type u_1) [monoid M] (R : Type u_10) [semiring R] [mul_semiring_action M R] (S : Type u_12) [semiring S] [mul_semiring_action M S] :
has_coe (R →+*[M] S) (R →+* S)

Equations
@[instance]
def mul_semiring_action_hom.​has_coe' (M : Type u_1) [monoid M] (R : Type u_10) [semiring R] [mul_semiring_action M R] (S : Type u_12) [semiring S] [mul_semiring_action M S] :
has_coe (R →+*[M] S) (R →+[M] S)

Equations
@[instance]
def mul_semiring_action_hom.​has_coe_to_fun (M : Type u_1) [monoid M] (R : Type u_10) [semiring R] [mul_semiring_action M R] (S : Type u_12) [semiring S] [mul_semiring_action M S] :

Equations
theorem mul_semiring_action_hom.​coe_fn_coe {M : Type u_1} [monoid M] {R : Type u_10} [semiring R] [mul_semiring_action M R] {S : Type u_12} [semiring S] [mul_semiring_action M S] (f : R →+*[M] S) :

theorem mul_semiring_action_hom.​coe_fn_coe' {M : Type u_1} [monoid M] {R : Type u_10} [semiring R] [mul_semiring_action M R] {S : Type u_12} [semiring S] [mul_semiring_action M S] (f : R →+*[M] S) :

@[ext]
theorem mul_semiring_action_hom.​ext {M : Type u_1} [monoid M] {R : Type u_10} [semiring R] [mul_semiring_action M R] {S : Type u_12} [semiring S] [mul_semiring_action M S] {f g : R →+*[M] S} :
(∀ (x : R), f x = g x)f = g

theorem mul_semiring_action_hom.​ext_iff {M : Type u_1} [monoid M] {R : Type u_10} [semiring R] [mul_semiring_action M R] {S : Type u_12} [semiring S] [mul_semiring_action M S] {f g : R →+*[M] S} :
f = g ∀ (x : R), f x = g x

@[simp]
theorem mul_semiring_action_hom.​map_zero {M : Type u_1} [monoid M] {R : Type u_10} [semiring R] [mul_semiring_action M R] {S : Type u_12} [semiring S] [mul_semiring_action M S] (f : R →+*[M] S) :
f 0 = 0

@[simp]
theorem mul_semiring_action_hom.​map_add {M : Type u_1} [monoid M] {R : Type u_10} [semiring R] [mul_semiring_action M R] {S : Type u_12} [semiring S] [mul_semiring_action M S] (f : R →+*[M] S) (x y : R) :
f (x + y) = f x + f y

@[simp]
theorem mul_semiring_action_hom.​map_neg {M : Type u_1} [monoid M] (R' : Type u_11) [ring R'] [mul_semiring_action M R'] (S' : Type u_13) [ring S'] [mul_semiring_action M S'] (f : R' →+*[M] S') (x : R') :
f (-x) = -f x

@[simp]
theorem mul_semiring_action_hom.​map_sub {M : Type u_1} [monoid M] (R' : Type u_11) [ring R'] [mul_semiring_action M R'] (S' : Type u_13) [ring S'] [mul_semiring_action M S'] (f : R' →+*[M] S') (x y : R') :
f (x - y) = f x - f y

@[simp]
theorem mul_semiring_action_hom.​map_one {M : Type u_1} [monoid M] {R : Type u_10} [semiring R] [mul_semiring_action M R] {S : Type u_12} [semiring S] [mul_semiring_action M S] (f : R →+*[M] S) :
f 1 = 1

@[simp]
theorem mul_semiring_action_hom.​map_mul {M : Type u_1} [monoid M] {R : Type u_10} [semiring R] [mul_semiring_action M R] {S : Type u_12} [semiring S] [mul_semiring_action M S] (f : R →+*[M] S) (x y : R) :
f (x * y) = f x * f y

@[simp]
theorem mul_semiring_action_hom.​map_smul {M : Type u_1} [monoid M] {R : Type u_10} [semiring R] [mul_semiring_action M R] {S : Type u_12} [semiring S] [mul_semiring_action M S] (f : R →+*[M] S) (m : M) (x : R) :
f (m x) = m f x

def mul_semiring_action_hom.​id (M : Type u_1) [monoid M] {R : Type u_10} [semiring R] [mul_semiring_action M R] :
R →+*[M] R

The identity map as an equivariant ring homomorphism.

Equations
@[simp]
theorem mul_semiring_action_hom.​id_apply (M : Type u_1) [monoid M] {R : Type u_10} [semiring R] [mul_semiring_action M R] (x : R) :

def mul_semiring_action_hom.​comp {M : Type u_1} [monoid M] {R : Type u_10} [semiring R] [mul_semiring_action M R] {S : Type u_12} [semiring S] [mul_semiring_action M S] {T : Type u_14} [semiring T] [mul_semiring_action M T] :
(S →+*[M] T)(R →+*[M] S)(R →+*[M] T)

Composition of two equivariant additive monoid homomorphisms.

Equations
@[simp]
theorem mul_semiring_action_hom.​comp_apply {M : Type u_1} [monoid M] {R : Type u_10} [semiring R] [mul_semiring_action M R] {S : Type u_12} [semiring S] [mul_semiring_action M S] {T : Type u_14} [semiring T] [mul_semiring_action M T] (g : S →+*[M] T) (f : R →+*[M] S) (x : R) :
(g.comp f) x = g (f x)

@[simp]
theorem mul_semiring_action_hom.​id_comp {M : Type u_1} [monoid M] {R : Type u_10} [semiring R] [mul_semiring_action M R] {S : Type u_12} [semiring S] [mul_semiring_action M S] (f : R →+*[M] S) :

@[simp]
theorem mul_semiring_action_hom.​comp_id {M : Type u_1} [monoid M] {R : Type u_10} [semiring R] [mul_semiring_action M R] {S : Type u_12} [semiring S] [mul_semiring_action M S] (f : R →+*[M] S) :

def mul_semiring_action_hom.​polynomial {M : Type u_1} [monoid M] {P : Type u_16} [comm_semiring P] [mul_semiring_action M P] {Q : Type u_17} [comm_semiring Q] [mul_semiring_action M Q] :

An equivariant map induces an equivariant map on polynomials.

Equations
@[simp]
theorem mul_semiring_action_hom.​coe_polynomial {M : Type u_1} [monoid M] {P : Type u_16} [comm_semiring P] [mul_semiring_action M P] {Q : Type u_17} [comm_semiring Q] [mul_semiring_action M Q] (g : P →+*[M] Q) :

def is_invariant_subring.​subtype_hom (M : Type u_1) [monoid M] {R' : Type u_11} [ring R'] [mul_semiring_action M R'] (U : set R') [is_subring U] [is_invariant_subring M U] :

The canonical inclusion from an invariant subring.

Equations
@[simp]
theorem is_invariant_subring.​coe_subtype_hom (M : Type u_1) [monoid M] {R' : Type u_11} [ring R'] [mul_semiring_action M R'] (U : set R') [is_subring U] [is_invariant_subring M U] :