mathlib3 documentation

group_theory.submonoid.operations

Operations on submonoids #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

In this file we define various operations on submonoids and monoid_homs.

Main definitions #

Conversion between multiplicative and additive definitions #

(Commutative) monoid structure on a submonoid #

Group actions by submonoids #

Operations on submonoids #

Monoid homomorphisms between submonoid #

Operations on monoid_homs #

Tags #

submonoid, range, product, map, comap

Conversion to/from additive/multiplicative #

Submonoids of monoid M are isomorphic to additive submonoids of additive M.

Equations
@[reducible]

Additive submonoids of an additive monoid additive M are isomorphic to submonoids of M.

Additive submonoids of an additive monoid A are isomorphic to multiplicative submonoids of multiplicative A.

Equations
@[reducible]

Submonoids of a monoid multiplicative A are isomorphic to additive submonoids of A.

comap and map #

def submonoid.comap {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (f : F) (S : submonoid N) :

The preimage of a submonoid along a monoid homomorphism is a submonoid.

Equations
def add_submonoid.comap {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] (f : F) (S : add_submonoid N) :

The preimage of an add_submonoid along an add_monoid homomorphism is an add_submonoid.

Equations
@[simp]
theorem submonoid.coe_comap {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (S : submonoid N) (f : F) :
@[simp]
theorem add_submonoid.coe_comap {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] (S : add_submonoid N) (f : F) :
@[simp]
theorem submonoid.mem_comap {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {S : submonoid N} {f : F} {x : M} :
@[simp]
theorem add_submonoid.mem_comap {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] {S : add_submonoid N} {f : F} {x : M} :
theorem add_submonoid.comap_comap {M : Type u_1} {N : Type u_2} {P : Type u_3} [add_zero_class M] [add_zero_class N] [add_zero_class P] (S : add_submonoid P) (g : N →+ P) (f : M →+ N) :
theorem submonoid.comap_comap {M : Type u_1} {N : Type u_2} {P : Type u_3} [mul_one_class M] [mul_one_class N] [mul_one_class P] (S : submonoid P) (g : N →* P) (f : M →* N) :
@[simp]
theorem submonoid.comap_id {P : Type u_3} [mul_one_class P] (S : submonoid P) :
def submonoid.map {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (f : F) (S : submonoid M) :

The image of a submonoid along a monoid homomorphism is a submonoid.

Equations
def add_submonoid.map {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] (f : F) (S : add_submonoid M) :

The image of an add_submonoid along an add_monoid homomorphism is an add_submonoid.

Equations
@[simp]
theorem submonoid.coe_map {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (f : F) (S : submonoid M) :
@[simp]
theorem add_submonoid.coe_map {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] (f : F) (S : add_submonoid M) :
@[simp]
theorem add_submonoid.mem_map {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] {f : F} {S : add_submonoid M} {y : N} :
y add_submonoid.map f S (x : M) (H : x S), f x = y
@[simp]
theorem submonoid.mem_map {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {f : F} {S : submonoid M} {y : N} :
y submonoid.map f S (x : M) (H : x S), f x = y
theorem submonoid.mem_map_of_mem {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (f : F) {S : submonoid M} {x : M} (hx : x S) :
theorem add_submonoid.mem_map_of_mem {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] (f : F) {S : add_submonoid M} {x : M} (hx : x S) :
theorem add_submonoid.apply_coe_mem_map {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] (f : F) (S : add_submonoid M) (x : S) :
theorem submonoid.apply_coe_mem_map {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (f : F) (S : submonoid M) (x : S) :
theorem submonoid.map_map {M : Type u_1} {N : Type u_2} {P : Type u_3} [mul_one_class M] [mul_one_class N] [mul_one_class P] (S : submonoid M) (g : N →* P) (f : M →* N) :
theorem add_submonoid.map_map {M : Type u_1} {N : Type u_2} {P : Type u_3} [add_zero_class M] [add_zero_class N] [add_zero_class P] (S : add_submonoid M) (g : N →+ P) (f : M →+ N) :
theorem add_submonoid.mem_map_iff_mem {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] {f : F} (hf : function.injective f) {S : add_submonoid M} {x : M} :
theorem submonoid.mem_map_iff_mem {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {f : F} (hf : function.injective f) {S : submonoid M} {x : M} :
theorem add_submonoid.map_le_iff_le_comap {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] {f : F} {S : add_submonoid M} {T : add_submonoid N} :
theorem submonoid.map_le_iff_le_comap {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {f : F} {S : submonoid M} {T : submonoid N} :
theorem submonoid.gc_map_comap {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (f : F) :
theorem submonoid.map_le_of_le_comap {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (S : submonoid M) {F : Type u_4} [mc : monoid_hom_class F M N] {T : submonoid N} {f : F} :
theorem add_submonoid.map_le_of_le_comap {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] (S : add_submonoid M) {F : Type u_4} [mc : add_monoid_hom_class F M N] {T : add_submonoid N} {f : F} :
theorem submonoid.le_comap_of_map_le {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (S : submonoid M) {F : Type u_4} [mc : monoid_hom_class F M N] {T : submonoid N} {f : F} :
theorem add_submonoid.le_comap_of_map_le {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] (S : add_submonoid M) {F : Type u_4} [mc : add_monoid_hom_class F M N] {T : add_submonoid N} {f : F} :
theorem submonoid.le_comap_map {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (S : submonoid M) {F : Type u_4} [mc : monoid_hom_class F M N] {f : F} :
theorem add_submonoid.le_comap_map {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] (S : add_submonoid M) {F : Type u_4} [mc : add_monoid_hom_class F M N] {f : F} :
theorem add_submonoid.map_comap_le {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] {S : add_submonoid N} {f : F} :
theorem submonoid.map_comap_le {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {S : submonoid N} {f : F} :
theorem add_submonoid.monotone_map {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] {f : F} :
theorem submonoid.monotone_map {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {f : F} :
theorem add_submonoid.monotone_comap {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] {f : F} :
theorem submonoid.monotone_comap {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {f : F} :
@[simp]
theorem submonoid.map_comap_map {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (S : submonoid M) {F : Type u_4} [mc : monoid_hom_class F M N] {f : F} :
@[simp]
theorem submonoid.comap_map_comap {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {S : submonoid N} {f : F} :
theorem submonoid.map_sup {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (S T : submonoid M) (f : F) :
theorem add_submonoid.map_sup {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] (S T : add_submonoid M) (f : F) :
theorem submonoid.map_supr {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {ι : Sort u_3} (f : F) (s : ι submonoid M) :
submonoid.map f (supr s) = (i : ι), submonoid.map f (s i)
theorem add_submonoid.map_supr {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] {ι : Sort u_3} (f : F) (s : ι add_submonoid M) :
theorem submonoid.comap_inf {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (S T : submonoid N) (f : F) :
theorem add_submonoid.comap_inf {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] (S T : add_submonoid N) (f : F) :
theorem submonoid.comap_infi {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {ι : Sort u_3} (f : F) (s : ι submonoid N) :
submonoid.comap f (infi s) = (i : ι), submonoid.comap f (s i)
theorem add_submonoid.comap_infi {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] {ι : Sort u_3} (f : F) (s : ι add_submonoid N) :
@[simp]
theorem submonoid.map_bot {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (f : F) :
@[simp]
theorem add_submonoid.map_bot {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] (f : F) :
@[simp]
theorem add_submonoid.comap_top {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] (f : F) :
@[simp]
theorem submonoid.comap_top {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (f : F) :
@[simp]
theorem submonoid.map_id {M : Type u_1} [mul_one_class M] (S : submonoid M) :

map f and comap f form a galois_coinsertion when f is injective.

Equations

map f and comap f form a galois_coinsertion when f is injective.

Equations
theorem submonoid.comap_map_eq_of_injective {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {f : F} (hf : function.injective f) (S : submonoid M) :
theorem submonoid.comap_inf_map_of_injective {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {f : F} (hf : function.injective f) (S T : submonoid M) :
theorem submonoid.comap_infi_map_of_injective {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {ι : Type u_5} {f : F} (hf : function.injective f) (S : ι submonoid M) :
submonoid.comap f ( (i : ι), submonoid.map f (S i)) = infi S
theorem add_submonoid.comap_infi_map_of_injective {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] {ι : Type u_5} {f : F} (hf : function.injective f) (S : ι add_submonoid M) :
theorem submonoid.comap_sup_map_of_injective {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {f : F} (hf : function.injective f) (S T : submonoid M) :
theorem submonoid.comap_supr_map_of_injective {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {ι : Type u_5} {f : F} (hf : function.injective f) (S : ι submonoid M) :
submonoid.comap f ( (i : ι), submonoid.map f (S i)) = supr S
theorem add_submonoid.comap_supr_map_of_injective {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] {ι : Type u_5} {f : F} (hf : function.injective f) (S : ι add_submonoid M) :
theorem submonoid.map_le_map_iff_of_injective {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {f : F} (hf : function.injective f) {S T : submonoid M} :
def submonoid.gi_map_comap {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {f : F} (hf : function.surjective f) :

map f and comap f form a galois_insertion when f is surjective.

Equations

map f and comap f form a galois_insertion when f is surjective.

Equations
theorem submonoid.map_comap_eq_of_surjective {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {f : F} (hf : function.surjective f) (S : submonoid N) :
theorem submonoid.map_inf_comap_of_surjective {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {f : F} (hf : function.surjective f) (S T : submonoid N) :
theorem add_submonoid.map_infi_comap_of_surjective {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] {ι : Type u_5} {f : F} (hf : function.surjective f) (S : ι add_submonoid N) :
theorem submonoid.map_infi_comap_of_surjective {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {ι : Type u_5} {f : F} (hf : function.surjective f) (S : ι submonoid N) :
submonoid.map f ( (i : ι), submonoid.comap f (S i)) = infi S
theorem submonoid.map_sup_comap_of_surjective {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {f : F} (hf : function.surjective f) (S T : submonoid N) :
theorem submonoid.map_supr_comap_of_surjective {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {ι : Type u_5} {f : F} (hf : function.surjective f) (S : ι submonoid N) :
submonoid.map f ( (i : ι), submonoid.comap f (S i)) = supr S
theorem add_submonoid.map_supr_comap_of_surjective {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] {ι : Type u_5} {f : F} (hf : function.surjective f) (S : ι add_submonoid N) :
theorem submonoid.comap_le_comap_iff_of_surjective {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {f : F} (hf : function.surjective f) {S T : submonoid N} :
@[protected, instance]
def one_mem_class.has_one {A : Type u_4} {M₁ : Type u_5} [set_like A M₁] [has_one M₁] [hA : one_mem_class A M₁] (S' : A) :

A submonoid of a monoid inherits a 1.

Equations
@[protected, instance]
def zero_mem_class.has_zero {A : Type u_4} {M₁ : Type u_5} [set_like A M₁] [has_zero M₁] [hA : zero_mem_class A M₁] (S' : A) :

An add_submonoid of an add_monoid inherits a zero.

Equations
@[simp, norm_cast]
theorem zero_mem_class.coe_zero {A : Type u_4} {M₁ : Type u_5} [set_like A M₁] [has_zero M₁] [hA : zero_mem_class A M₁] (S' : A) :
0 = 0
@[simp, norm_cast]
theorem one_mem_class.coe_one {A : Type u_4} {M₁ : Type u_5} [set_like A M₁] [has_one M₁] [hA : one_mem_class A M₁] (S' : A) :
1 = 1
@[simp, norm_cast]
theorem zero_mem_class.coe_eq_zero {A : Type u_4} {M₁ : Type u_5} [set_like A M₁] [has_zero M₁] [hA : zero_mem_class A M₁] {S' : A} {x : S'} :
x = 0 x = 0
@[simp, norm_cast]
theorem one_mem_class.coe_eq_one {A : Type u_4} {M₁ : Type u_5} [set_like A M₁] [has_one M₁] [hA : one_mem_class A M₁] {S' : A} {x : S'} :
x = 1 x = 1
theorem zero_mem_class.zero_def {A : Type u_4} {M₁ : Type u_5} [set_like A M₁] [has_zero M₁] [hA : zero_mem_class A M₁] (S' : A) :
0 = 0, _⟩
theorem one_mem_class.one_def {A : Type u_4} {M₁ : Type u_5} [set_like A M₁] [has_one M₁] [hA : one_mem_class A M₁] (S' : A) :
1 = 1, _⟩
@[protected, instance]
def add_submonoid_class.has_nsmul {M : Type u_1} [add_monoid M] {A : Type u_2} [set_like A M] [add_submonoid_class A M] (S : A) :

An add_submonoid of an add_monoid inherits a scalar multiplication.

Equations
@[protected, instance]
def submonoid_class.has_pow {M : Type u_1} [monoid M] {A : Type u_2} [set_like A M] [submonoid_class A M] (S : A) :

A submonoid of a monoid inherits a power operator.

Equations
@[simp, norm_cast]
theorem add_submonoid_class.coe_nsmul {M : Type u_1} [add_monoid M] {A : Type u_2} [set_like A M] [add_submonoid_class A M] {S : A} (x : S) (n : ) :
(n x) = n x
@[simp, norm_cast]
theorem submonoid_class.coe_pow {M : Type u_1} [monoid M] {A : Type u_2} [set_like A M] [submonoid_class A M] {S : A} (x : S) (n : ) :
(x ^ n) = x ^ n
@[simp]
theorem add_submonoid_class.mk_nsmul {M : Type u_1} [add_monoid M] {A : Type u_2} [set_like A M] [add_submonoid_class A M] {S : A} (x : M) (hx : x S) (n : ) :
n x, hx⟩ = n x, _⟩
@[simp]
theorem submonoid_class.mk_pow {M : Type u_1} [monoid M] {A : Type u_2} [set_like A M] [submonoid_class A M] {S : A} (x : M) (hx : x S) (n : ) :
x, hx⟩ ^ n = x ^ n, _⟩
@[protected, instance]

An add_submonoid of an unital additive magma inherits an unital additive magma structure.

Equations
@[protected, instance]

A submonoid of a unital magma inherits a unital magma structure.

Equations
@[protected, instance]
def submonoid_class.to_monoid {M : Type u_1} [monoid M] {A : Type u_2} [set_like A M] [submonoid_class A M] (S : A) :

A submonoid of a monoid inherits a monoid structure.

Equations
@[protected, instance]
def add_submonoid_class.to_add_monoid {M : Type u_1} [add_monoid M] {A : Type u_2} [set_like A M] [add_submonoid_class A M] (S : A) :

An add_submonoid of an add_monoid inherits an add_monoid structure.

Equations
@[protected, instance]
def submonoid_class.to_comm_monoid {M : Type u_1} [comm_monoid M] {A : Type u_2} [set_like A M] [submonoid_class A M] (S : A) :

A submonoid of a comm_monoid is a comm_monoid.

Equations
def submonoid_class.subtype {M : Type u_1} [mul_one_class M] {A : Type u_4} [set_like A M] [hA : submonoid_class A M] (S' : A) :
S' →* M

The natural monoid hom from a submonoid of monoid M to M.

Equations
def add_submonoid_class.subtype {M : Type u_1} [add_zero_class M] {A : Type u_4} [set_like A M] [hA : add_submonoid_class A M] (S' : A) :
S' →+ M

The natural monoid hom from an add_submonoid of add_monoid M to M.

Equations
@[simp]
theorem add_submonoid_class.coe_subtype {M : Type u_1} [add_zero_class M] {A : Type u_4} [set_like A M] [hA : add_submonoid_class A M] (S' : A) :
@[simp]
theorem submonoid_class.coe_subtype {M : Type u_1} [mul_one_class M] {A : Type u_4} [set_like A M] [hA : submonoid_class A M] (S' : A) :
@[protected, instance]
def submonoid.has_mul {M : Type u_1} [mul_one_class M] (S : submonoid M) :

A submonoid of a monoid inherits a multiplication.

Equations
@[protected, instance]

An add_submonoid of an add_monoid inherits an addition.

Equations
@[protected, instance]
def submonoid.has_one {M : Type u_1} [mul_one_class M] (S : submonoid M) :

A submonoid of a monoid inherits a 1.

Equations
@[protected, instance]

An add_submonoid of an add_monoid inherits a zero.

Equations
@[simp, norm_cast]
theorem submonoid.coe_mul {M : Type u_1} [mul_one_class M] (S : submonoid M) (x y : S) :
(x * y) = x * y
@[simp, norm_cast]
theorem add_submonoid.coe_add {M : Type u_1} [add_zero_class M] (S : add_submonoid M) (x y : S) :
(x + y) = x + y
@[simp, norm_cast]
theorem add_submonoid.coe_zero {M : Type u_1} [add_zero_class M] (S : add_submonoid M) :
0 = 0
@[simp, norm_cast]
theorem submonoid.coe_one {M : Type u_1} [mul_one_class M] (S : submonoid M) :
1 = 1
@[simp]
theorem submonoid.mk_mul_mk {M : Type u_1} [mul_one_class M] (S : submonoid M) (x y : M) (hx : x S) (hy : y S) :
x, hx⟩ * y, hy⟩ = x * y, _⟩
@[simp]
theorem add_submonoid.mk_add_mk {M : Type u_1} [add_zero_class M] (S : add_submonoid M) (x y : M) (hx : x S) (hy : y S) :
x, hx⟩ + y, hy⟩ = x + y, _⟩
theorem submonoid.mul_def {M : Type u_1} [mul_one_class M] (S : submonoid M) (x y : S) :
x * y = x * y, _⟩
theorem add_submonoid.add_def {M : Type u_1} [add_zero_class M] (S : add_submonoid M) (x y : S) :
x + y = x + y, _⟩
theorem submonoid.one_def {M : Type u_1} [mul_one_class M] (S : submonoid M) :
1 = 1, _⟩
theorem add_submonoid.zero_def {M : Type u_1} [add_zero_class M] (S : add_submonoid M) :
0 = 0, _⟩
@[protected, instance]

An add_submonoid of an unital additive magma inherits an unital additive magma structure.

Equations
@[protected, instance]

A submonoid of a unital magma inherits a unital magma structure.

Equations
@[protected]
theorem submonoid.pow_mem {M : Type u_1} [monoid M] (S : submonoid M) {x : M} (hx : x S) (n : ) :
x ^ n S
@[protected]
theorem add_submonoid.nsmul_mem {M : Type u_1} [add_monoid M] (S : add_submonoid M) {x : M} (hx : x S) (n : ) :
n x S
@[simp, norm_cast]
theorem add_submonoid.coe_nsmul {M : Type u_1} [add_monoid M] {S : add_submonoid M} (x : S) (n : ) :
(n x) = n x
@[simp, norm_cast]
theorem submonoid.coe_pow {M : Type u_1} [monoid M] {S : submonoid M} (x : S) (n : ) :
(x ^ n) = x ^ n
@[protected, instance]
def submonoid.to_monoid {M : Type u_1} [monoid M] (S : submonoid M) :

A submonoid of a monoid inherits a monoid structure.

Equations
@[protected, instance]

An add_submonoid of an add_monoid inherits an add_monoid structure.

Equations
@[protected, instance]

A submonoid of a comm_monoid is a comm_monoid.

Equations

The natural monoid hom from an add_submonoid of add_monoid M to M.

Equations
def submonoid.subtype {M : Type u_1} [mul_one_class M] (S : submonoid M) :

The natural monoid hom from a submonoid of monoid M to M.

Equations
@[simp]
@[simp]
theorem submonoid.coe_subtype {M : Type u_1} [mul_one_class M] (S : submonoid M) :

The top submonoid is isomorphic to the monoid.

Equations

The top additive submonoid is isomorphic to the additive monoid.

Equations
noncomputable def add_submonoid.equiv_map_of_injective {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] (S : add_submonoid M) (f : M →+ N) (hf : function.injective f) :

An additive subgroup is isomorphic to its image under an injective function. If you have an isomorphism, use add_equiv.add_submonoid_map for better definitional equalities.

Equations
noncomputable def submonoid.equiv_map_of_injective {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (S : submonoid M) (f : M →* N) (hf : function.injective f) :

A subgroup is isomorphic to its image under an injective function. If you have an isomorphism, use mul_equiv.submonoid_map for better definitional equalities.

Equations
@[simp]
@[simp]
theorem submonoid.coe_equiv_map_of_injective_apply {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (S : submonoid M) (f : M →* N) (hf : function.injective f) (x : S) :
def submonoid.prod {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (s : submonoid M) (t : submonoid N) :

Given submonoids s, t of monoids M, N respectively, s × t as a submonoid of M × N.

Equations
def add_submonoid.prod {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] (s : add_submonoid M) (t : add_submonoid N) :

Given add_submonoids s, t of add_monoids A, B respectively, s × t as an add_submonoid of A × B.

Equations
theorem add_submonoid.coe_prod {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] (s : add_submonoid M) (t : add_submonoid N) :
(s.prod t) = s ×ˢ t
theorem submonoid.coe_prod {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (s : submonoid M) (t : submonoid N) :
(s.prod t) = s ×ˢ t
theorem submonoid.mem_prod {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {s : submonoid M} {t : submonoid N} {p : M × N} :
p s.prod t p.fst s p.snd t
theorem add_submonoid.mem_prod {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {s : add_submonoid M} {t : add_submonoid N} {p : M × N} :
p s.prod t p.fst s p.snd t
theorem add_submonoid.prod_mono {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {s₁ s₂ : add_submonoid M} {t₁ t₂ : add_submonoid N} (hs : s₁ s₂) (ht : t₁ t₂) :
s₁.prod t₁ s₂.prod t₂
theorem submonoid.prod_mono {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {s₁ s₂ : submonoid M} {t₁ t₂ : submonoid N} (hs : s₁ s₂) (ht : t₁ t₂) :
s₁.prod t₁ s₂.prod t₂
theorem submonoid.prod_top {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (s : submonoid M) :
theorem submonoid.top_prod {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (s : submonoid N) :
@[simp]
@[simp]
theorem submonoid.top_prod_top {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] :
theorem submonoid.bot_prod_bot {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] :
def submonoid.prod_equiv {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (s : submonoid M) (t : submonoid N) :

The product of submonoids is isomorphic to their product as monoids.

Equations
def add_submonoid.prod_equiv {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] (s : add_submonoid M) (t : add_submonoid N) :

The product of additive submonoids is isomorphic to their product as additive monoids

Equations
theorem submonoid.map_inl {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (s : submonoid M) :
theorem submonoid.map_inr {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (s : submonoid N) :
@[simp]
theorem submonoid.prod_bot_sup_bot_prod {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (s : submonoid M) (t : submonoid N) :
@[simp]
theorem add_submonoid.mem_map_equiv {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {f : M ≃+ N} {K : add_submonoid M} {x : N} :
theorem submonoid.mem_map_equiv {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {f : M ≃* N} {K : submonoid M} {x : N} :
@[simp]
theorem submonoid.map_equiv_top {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (f : M ≃* N) :
theorem submonoid.le_prod_iff {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {s : submonoid M} {t : submonoid N} {u : submonoid (M × N)} :
theorem submonoid.prod_le_iff {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {s : submonoid M} {t : submonoid N} {u : submonoid (M × N)} :

For many categories (monoids, modules, rings, ...) the set-theoretic image of a morphism f is a subobject of the codomain. When this is the case, it is useful to define the range of a morphism in such a way that the underlying carrier set of the range subobject is definitionally set.range f. In particular this means that the types ↥(set.range f) and ↥f.range are interchangeable without proof obligations.

A convenient candidate definition for range which is mathematically correct is map ⊤ f, just as set.range could have been defined as f '' set.univ. However, this lacks the desired definitional convenience, in that it both does not match set.range, and that it introduces a redudant x ∈ ⊤ term which clutters proofs. In such a case one may resort to the copy pattern. A copy function converts the definitional problem for the carrier set of a subobject into a one-off propositional proof obligation which one discharges while writing the definition of the definitionally convenient range (the parameter hs in the example below).

A good example is the case of a morphism of monoids. A convenient definition for monoid_hom.mrange would be (⊤ : submonoid M).map f. However since this lacks the required definitional convenience, we first define submonoid.copy as follows:

protected def copy (S : submonoid M) (s : set M) (hs : s = S) : submonoid M :=
{ carrier  := s,
  one_mem' := hs.symm  S.one_mem',
  mul_mem' := hs.symm  S.mul_mem' }

and then finally define:

def mrange (f : M →* N) : submonoid N :=
(( : submonoid M).map f).copy (set.range f) set.image_univ.symm
def monoid_hom.mrange {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (f : F) :

The range of a monoid homomorphism is a submonoid. See Note [range copy pattern].

Equations
Instances for monoid_hom.mrange
def add_monoid_hom.mrange {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] (f : F) :

The range of an add_monoid_hom is an add_submonoid.

Equations
Instances for add_monoid_hom.mrange
@[simp]
theorem monoid_hom.coe_mrange {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (f : F) :
@[simp]
theorem add_monoid_hom.coe_mrange {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] (f : F) :
@[simp]
theorem add_monoid_hom.mem_mrange {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] {f : F} {y : N} :
@[simp]
theorem monoid_hom.mem_mrange {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] {f : F} {y : N} :
y monoid_hom.mrange f (x : M), f x = y
theorem monoid_hom.mrange_eq_map {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (f : F) :
theorem monoid_hom.map_mrange {M : Type u_1} {N : Type u_2} {P : Type u_3} [mul_one_class M] [mul_one_class N] [mul_one_class P] (g : N →* P) (f : M →* N) :

The range of a surjective add_monoid hom is the whole of the codomain.

theorem monoid_hom.mrange_top_of_surjective {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (f : F) (hf : function.surjective f) :

The range of a surjective monoid hom is the whole of the codomain.

theorem monoid_hom.mclosure_preimage_le {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (f : F) (s : set N) :
theorem add_monoid_hom.map_mclosure {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] (f : F) (s : set M) :

The image under an add_monoid hom of the add_submonoid generated by a set equals the add_submonoid generated by the image of the set.

theorem monoid_hom.map_mclosure {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (f : F) (s : set M) :

The image under a monoid hom of the submonoid generated by a set equals the submonoid generated by the image of the set.

def add_monoid_hom.restrict {M : Type u_1} [add_zero_class M] {N : Type u_2} {S : Type u_3} [add_zero_class N] [set_like S M] [add_submonoid_class S M] (f : M →+ N) (s : S) :

Restriction of an add_monoid hom to an add_submonoid of the domain.

Equations
def monoid_hom.restrict {M : Type u_1} [mul_one_class M] {N : Type u_2} {S : Type u_3} [mul_one_class N] [set_like S M] [submonoid_class S M] (f : M →* N) (s : S) :

Restriction of a monoid hom to a submonoid of the domain.

Equations
@[simp]
theorem add_monoid_hom.restrict_apply {M : Type u_1} [add_zero_class M] {N : Type u_2} {S : Type u_3} [add_zero_class N] [set_like S M] [add_submonoid_class S M] (f : M →+ N) (s : S) (x : s) :
(f.restrict s) x = f x
@[simp]
theorem monoid_hom.restrict_apply {M : Type u_1} [mul_one_class M] {N : Type u_2} {S : Type u_3} [mul_one_class N] [set_like S M] [submonoid_class S M] (f : M →* N) (s : S) (x : s) :
(f.restrict s) x = f x
@[simp]
theorem monoid_hom.restrict_mrange {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (S : submonoid M) (f : M →* N) :
@[simp]
theorem monoid_hom.cod_restrict_apply {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {S : Type u_3} [set_like S N] [submonoid_class S N] (f : M →* N) (s : S) (h : (x : M), f x s) (n : M) :
(f.cod_restrict s h) n = f n, _⟩
def add_monoid_hom.cod_restrict {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {S : Type u_3} [set_like S N] [add_submonoid_class S N] (f : M →+ N) (s : S) (h : (x : M), f x s) :

Restriction of an add_monoid hom to an add_submonoid of the codomain.

Equations
def monoid_hom.cod_restrict {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {S : Type u_3} [set_like S N] [submonoid_class S N] (f : M →* N) (s : S) (h : (x : M), f x s) :

Restriction of a monoid hom to a submonoid of the codomain.

Equations
@[simp]
theorem add_monoid_hom.cod_restrict_apply {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {S : Type u_3} [set_like S N] [add_submonoid_class S N] (f : M →+ N) (s : S) (h : (x : M), f x s) (n : M) :
(f.cod_restrict s h) n = f n, _⟩

Restriction of an add_monoid hom to its range interpreted as a submonoid.

Equations
def monoid_hom.mrange_restrict {M : Type u_1} [mul_one_class M] {N : Type u_2} [mul_one_class N] (f : M →* N) :

Restriction of a monoid hom to its range interpreted as a submonoid.

Equations
@[simp]
theorem add_monoid_hom.coe_mrange_restrict {M : Type u_1} [add_zero_class M] {N : Type u_2} [add_zero_class N] (f : M →+ N) (x : M) :
@[simp]
theorem monoid_hom.coe_mrange_restrict {M : Type u_1} [mul_one_class M] {N : Type u_2} [mul_one_class N] (f : M →* N) (x : M) :
def monoid_hom.mker {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (f : F) :

The multiplicative kernel of a monoid homomorphism is the submonoid of elements x : G such that f x = 1

Equations
def add_monoid_hom.mker {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] (f : F) :

The additive kernel of an add_monoid homomorphism is the add_submonoid of elements such that f x = 0

Equations
theorem monoid_hom.mem_mker {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (f : F) {x : M} :
theorem add_monoid_hom.mem_mker {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] (f : F) {x : M} :
theorem monoid_hom.coe_mker {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (f : F) :
theorem add_monoid_hom.coe_mker {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] (f : F) :
@[protected, instance]
def add_monoid_hom.decidable_mem_mker {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] [decidable_eq N] (f : F) :
Equations
@[protected, instance]
def monoid_hom.decidable_mem_mker {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] [decidable_eq N] (f : F) :
decidable_pred (λ (_x : M), _x monoid_hom.mker f)
Equations
theorem monoid_hom.comap_mker {M : Type u_1} {N : Type u_2} {P : Type u_3} [mul_one_class M] [mul_one_class N] [mul_one_class P] (g : N →* P) (f : M →* N) :
@[simp]
theorem add_monoid_hom.comap_bot' {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {F : Type u_4} [mc : add_monoid_hom_class F M N] (f : F) :
@[simp]
theorem monoid_hom.comap_bot' {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {F : Type u_4} [mc : monoid_hom_class F M N] (f : F) :
@[simp]
@[simp]
theorem monoid_hom.mker_one {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] :
theorem monoid_hom.prod_map_comap_prod' {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {M' : Type u_3} {N' : Type u_4} [mul_one_class M'] [mul_one_class N'] (f : M →* N) (g : M' →* N') (S : submonoid N) (S' : submonoid N') :
theorem add_monoid_hom.sum_map_comap_sum' {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {M' : Type u_3} {N' : Type u_4} [add_zero_class M'] [add_zero_class N'] (f : M →+ N) (g : M' →+ N') (S : add_submonoid N) (S' : add_submonoid N') :
theorem add_monoid_hom.mker_sum_map {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {M' : Type u_3} {N' : Type u_4} [add_zero_class M'] [add_zero_class N'] (f : M →+ N) (g : M' →+ N') :
theorem monoid_hom.mker_prod_map {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {M' : Type u_3} {N' : Type u_4} [mul_one_class M'] [mul_one_class N'] (f : M →* N) (g : M' →* N') :
@[simp]
@[simp]
@[simp]
theorem monoid_hom.submonoid_comap_apply_coe {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (f : M →* N) (N' : submonoid N) (x : (submonoid.comap f N')) :

the add_monoid_hom from the preimage of an additive submonoid to itself.

Equations
def monoid_hom.submonoid_comap {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (f : M →* N) (N' : submonoid N) :

The monoid_hom from the preimage of a submonoid to itself.

Equations
@[simp]

the add_monoid_hom from an additive submonoid to its image. See add_equiv.add_submonoid_map for a variant for add_equivs.

Equations
def monoid_hom.submonoid_map {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (f : M →* N) (M' : submonoid M) :

The monoid_hom from a submonoid to its image. See mul_equiv.submonoid_map for a variant for mul_equivs.

Equations
@[simp]
theorem monoid_hom.submonoid_map_apply_coe {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (f : M →* N) (M' : submonoid M) (x : M') :
@[simp]
theorem add_monoid_hom.add_submonoid_map_apply_coe {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] (f : M →+ N) (M' : add_submonoid M) (x : M') :
@[simp]
@[simp]
theorem submonoid.prod_eq_bot_iff {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {s : submonoid M} {t : submonoid N} :
s.prod t = s = t =
theorem add_submonoid.sum_eq_bot_iff {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {s : add_submonoid M} {t : add_submonoid N} :
s.prod t = s = t =
theorem submonoid.prod_eq_top_iff {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] {s : submonoid M} {t : submonoid N} :
s.prod t = s = t =
theorem add_submonoid.sum_eq_top_iff {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] {s : add_submonoid M} {t : add_submonoid N} :
s.prod t = s = t =
def submonoid.inclusion {M : Type u_1} [mul_one_class M] {S T : submonoid M} (h : S T) :

The monoid hom associated to an inclusion of submonoids.

Equations
def add_submonoid.inclusion {M : Type u_1} [add_zero_class M] {S T : add_submonoid M} (h : S T) :

The add_monoid hom associated to an inclusion of submonoids.

Equations
@[simp]
theorem add_submonoid.eq_top_iff' {M : Type u_1} [add_zero_class M] (S : add_submonoid M) :
S = (x : M), x S
theorem submonoid.eq_top_iff' {M : Type u_1} [mul_one_class M] (S : submonoid M) :
S = (x : M), x S
theorem submonoid.eq_bot_iff_forall {M : Type u_1} [mul_one_class M] (S : submonoid M) :
S = (x : M), x S x = 1
theorem add_submonoid.eq_bot_iff_forall {M : Type u_1} [add_zero_class M] (S : add_submonoid M) :
S = (x : M), x S x = 0
theorem submonoid.nontrivial_iff_exists_ne_one {M : Type u_1} [mul_one_class M] (S : submonoid M) :
nontrivial S (x : M) (H : x S), x 1

A submonoid is either the trivial submonoid or nontrivial.

An additive submonoid is either the trivial additive submonoid or nontrivial.

theorem submonoid.bot_or_exists_ne_one {M : Type u_1} [mul_one_class M] (S : submonoid M) :
S = (x : M) (H : x S), x 1

A submonoid is either the trivial submonoid or contains a nonzero element.

theorem add_submonoid.bot_or_exists_ne_zero {M : Type u_1} [add_zero_class M] (S : add_submonoid M) :
S = (x : M) (H : x S), x 0

An additive submonoid is either the trivial additive submonoid or contains a nonzero element.

def mul_equiv.submonoid_congr {M : Type u_1} [mul_one_class M] {S T : submonoid M} (h : S = T) :

Makes the identity isomorphism from a proof that two submonoids of a multiplicative monoid are equal.

Equations
def add_equiv.add_submonoid_congr {M : Type u_1} [add_zero_class M] {S T : add_submonoid M} (h : S = T) :

Makes the identity additive isomorphism from a proof two submonoids of an additive monoid are equal.

Equations
def mul_equiv.of_left_inverse' {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (f : M →* N) {g : N M} (h : function.left_inverse g f) :

A monoid homomorphism f : M →* N with a left-inverse g : N → M defines a multiplicative equivalence between M and f.mrange.

This is a bidirectional version of monoid_hom.mrange_restrict.

Equations
@[simp]
theorem add_equiv.of_left_inverse'_apply {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] (f : M →+ N) {g : N M} (h : function.left_inverse g f) (ᾰ : M) :
@[simp]
theorem mul_equiv.of_left_inverse'_apply {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (f : M →* N) {g : N M} (h : function.left_inverse g f) (ᾰ : M) :
@[simp]
theorem mul_equiv.of_left_inverse'_symm_apply {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (f : M →* N) {g : N M} (h : function.left_inverse g f) (ᾰ : (monoid_hom.mrange f)) :
def add_equiv.of_left_inverse' {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] (f : M →+ N) {g : N M} (h : function.left_inverse g f) :

An additive monoid homomorphism f : M →+ N with a left-inverse g : N → M defines an additive equivalence between M and f.mrange.

This is a bidirectional version of add_monoid_hom.mrange_restrict.

Equations
@[simp]
theorem add_equiv.of_left_inverse'_symm_apply {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] (f : M →+ N) {g : N M} (h : function.left_inverse g f) (ᾰ : (add_monoid_hom.mrange f)) :

An add_equiv φ between two additive monoids M and N induces an add_equiv between a submonoid S ≤ M and the submonoid φ(S) ≤ N. See add_monoid_hom.add_submonoid_map for a variant for add_monoid_homs.

Equations
def mul_equiv.submonoid_map {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (e : M ≃* N) (S : submonoid M) :

A mul_equiv φ between two monoids M and N induces a mul_equiv between a submonoid S ≤ M and the submonoid φ(S) ≤ N. See monoid_hom.submonoid_map for a variant for monoid_homs.

Equations
@[simp]
theorem mul_equiv.coe_submonoid_map_apply {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (e : M ≃* N) (S : submonoid M) (g : S) :
@[simp]
theorem add_equiv.coe_add_submonoid_map_apply {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] (e : M ≃+ N) (S : add_submonoid M) (g : S) :
@[simp]
theorem mul_equiv.submonoid_map_symm_apply {M : Type u_1} {N : Type u_2} [mul_one_class M] [mul_one_class N] (e : M ≃* N) (S : submonoid M) (g : (submonoid.map e S)) :
((e.submonoid_map S).symm) g = (e.symm) g, _⟩
@[simp]
theorem add_equiv.add_submonoid_map_symm_apply {M : Type u_1} {N : Type u_2} [add_zero_class M] [add_zero_class N] (e : M ≃+ N) (S : add_submonoid M) (g : (add_submonoid.map e S)) :

Actions by submonoids #

These instances tranfer the action by an element m : M of a monoid M written as m • a onto the action by an element s : S of a submonoid S : submonoid M such that s • a = (s : M) • a.

These instances work particularly well in conjunction with monoid.to_mul_action, enabling s • m as an alias for ↑s * m.

@[protected, instance]
def add_submonoid.has_vadd {M' : Type u_4} {α : Type u_5} [add_zero_class M'] [has_vadd M' α] (S : add_submonoid M') :
Equations
@[protected, instance]
def submonoid.has_smul {M' : Type u_4} {α : Type u_5} [mul_one_class M'] [has_smul M' α] (S : submonoid M') :
Equations
@[protected, instance]
def add_submonoid.vadd_comm_class_left {M' : Type u_4} {α : Type u_5} {β : Type u_6} [add_zero_class M'] [has_vadd M' β] [has_vadd α β] [vadd_comm_class M' α β] (S : add_submonoid M') :
@[protected, instance]
def submonoid.smul_comm_class_left {M' : Type u_4} {α : Type u_5} {β : Type u_6} [mul_one_class M'] [has_smul M' β] [has_smul α β] [smul_comm_class M' α β] (S : submonoid M') :
@[protected, instance]
def add_submonoid.vadd_comm_class_right {M' : Type u_4} {α : Type u_5} {β : Type u_6} [add_zero_class M'] [has_vadd α β] [has_vadd M' β] [vadd_comm_class α M' β] (S : add_submonoid M') :
@[protected, instance]
def submonoid.smul_comm_class_right {M' : Type u_4} {α : Type u_5} {β : Type u_6} [mul_one_class M'] [has_smul α β] [has_smul M' β] [smul_comm_class α M' β] (S : submonoid M') :
@[protected, instance]
def submonoid.is_scalar_tower {M' : Type u_4} {α : Type u_5} {β : Type u_6} [mul_one_class M'] [has_smul α β] [has_smul M' α] [has_smul M' β] [is_scalar_tower M' α β] (S : submonoid M') :

Note that this provides is_scalar_tower S M' M' which is needed by smul_mul_assoc.

theorem submonoid.smul_def {M' : Type u_4} {α : Type u_5} [mul_one_class M'] [has_smul M' α] {S : submonoid M'} (g : S) (m : α) :
g m = g m
theorem add_submonoid.vadd_def {M' : Type u_4} {α : Type u_5} [add_zero_class M'] [has_vadd M' α] {S : add_submonoid M'} (g : S) (m : α) :
g +ᵥ m = g +ᵥ m
@[protected, instance]
def submonoid.has_faithful_smul {M' : Type u_4} {α : Type u_5} [mul_one_class M'] [has_smul M' α] [has_faithful_smul M' α] (S : submonoid M') :
@[protected, instance]
def submonoid.mul_action {M' : Type u_4} {α : Type u_5} [monoid M'] [mul_action M' α] (S : submonoid M') :

The action by a submonoid is the action by the underlying monoid.

Equations
@[protected, instance]
def add_submonoid.add_action {M' : Type u_4} {α : Type u_5} [add_monoid M'] [add_action M' α] (S : add_submonoid M') :

The additive action by an add_submonoid is the action by the underlying add_monoid.

Equations
@[protected, instance]
def submonoid.distrib_mul_action {M' : Type u_4} {α : Type u_5} [monoid M'] [add_monoid α] [distrib_mul_action M' α] (S : submonoid M') :

The action by a submonoid is the action by the underlying monoid.

Equations
@[protected, instance]

The action by a submonoid is the action by the underlying monoid.

Equations