Submonoids
This file defines unbundled multiplicative and additive submonoids (deprecated). For bundled form
see group_theory/submonoid
.
We some results about images and preimages of submonoids under monoid homomorphisms. These theorems use unbundled monoid homomorphisms (also deprecated).
There are also theorems about the submonoids generated by an element or a subset of a monoid, defined inductively.
Implementation notes
Unbundled submonoids will slowly be removed from mathlib.
Tags
submonoid, submonoids, is_submonoid
s
is an additive submonoid: a set containing 0 and closed under addition.
Instances
- is_add_subgroup.to_is_add_submonoid
- is_add_submonoid.inter
- is_add_submonoid.Inter
- multiples.is_add_submonoid
- univ.is_add_submonoid
- preimage.is_add_submonoid
- image.is_add_submonoid
- range.is_add_submonoid
- add_monoid.closure.is_add_submonoid
- add_submonoid.is_add_submonoid
- subalgebra.is_add_submonoid
- continuous_add_submonoid
s
is a submonoid: a set containing 1 and closed under multiplication.
Instances
- is_subgroup.to_is_submonoid
- is_subring.to_is_submonoid
- is_submonoid.inter
- is_submonoid.Inter
- powers.is_submonoid
- univ.is_submonoid
- preimage.is_submonoid
- image.is_submonoid
- range.is_submonoid
- monoid.closure.is_submonoid
- submonoid.is_submonoid
- subalgebra.is_submonoid
- Ring.sections_submonoid'
- continuous_submonoid
- field.closure.is_submonoid
The intersection of two submonoids of a monoid M
is a submonoid of M
.
Equations
- _ = _
The intersection of two add_submonoid
s of an add_monoid
M
is
an add_submonoid
of M.
The intersection of an indexed set of submonoids of a monoid M
is a submonoid of M
.
Equations
- _ = _
The intersection of an indexed set of add_submonoid
s of an add_monoid
M
is
an add_submonoid
of M
.
The union of an indexed, directed, nonempty set
of add_submonoid
s of an add_monoid
M
is an add_submonoid
of M
.
The union of an indexed, directed, nonempty set of submonoids of a monoid M
is a submonoid
of M
.
The set of natural number multiples 0, x, 2x, ...
of an element x
of an add_monoid
.
1 is in the set of natural number powers of an element of a monoid.
0 is in the set of natural number multiples of an element of an add_monoid
.
An element of a monoid is in the set of that element's natural number powers.
An element of an add_monoid
is in the set of that element's natural number multiples.
The set of natural number multiples of an element of an add_monoid
is closed under
addition.
The set of natural number powers of an element of a monoid M
is a submonoid of M
.
Equations
- _ = _
The set of natural number multiples of an element of
an add_monoid
M
is an add_submonoid
of M
.
An add_monoid
is an add_submonoid
of itself.
A monoid is a submonoid of itself.
Equations
The preimage of an add_submonoid
under an add_monoid
hom is
an add_submonoid
of the domain.
The preimage of a submonoid under a monoid hom is a submonoid of the domain.
Equations
- _ = _
The image of an add_submonoid
under an add_monoid
hom is an add_submonoid
of the codomain.
The image of a submonoid under a monoid hom is a submonoid of the codomain.
The image of a monoid hom is a submonoid of the codomain.
Equations
- _ = _
The image of an add_monoid
hom is an add_submonoid
of the codomain.
Submonoids are closed under natural powers.
An add_submonoid
is closed under multiplication by naturals.
The set of natural number powers of an element of a submonoid is a subset of the submonoid.
The set of natural number multiples of an element of an add_submonoid
is a subset of the
add_submonoid
.
The product of a list of elements of a submonoid is an element of the submonoid.
The sum of a list of elements of an add_submonoid
is an element of the
add_submonoid
.
The sum of a multiset of elements of an add_submonoid
of an add_comm_monoid
is an element of the add_submonoid
.
The product of a multiset of elements of a submonoid of a comm_monoid
is an element of
the submonoid.
The sum of elements of an add_submonoid
of an add_comm_monoid
indexed by
a finset
is an element of the add_submonoid
.
The product of elements of a submonoid of a comm_monoid
indexed by a finset
is an element
of the submonoid.
An add_submonoid
is itself an add_monoid
.
An add_submonoid
of a commutative add_monoid
is itself
a commutative add_monoid
.
Submonoids of commutative monoids are themselves commutative monoids.
Equations
- subtype.comm_monoid = {mul := monoid.mul subtype.monoid, mul_assoc := _, one := monoid.one subtype.monoid, one_mul := _, mul_one := _, mul_comm := _}
Submonoids inherit the 1 of the monoid.
An add_submonoid
inherits the 0 of the add_monoid
.
An add_submonoid
inherits the addition of the add_monoid
.
An add_submonoid
inherits the multiplication by naturals of the add_monoid
.
The natural injection from a submonoid into the monoid is a monoid hom.
Equations
The natural injection from an add_submonoid
into
the add_monoid
is an add_monoid
hom.
The natural injection from a submonoid into the monoid is a monoid hom.
Equations
The natural injection from an add_submonoid
into
the add_monoid
is an add_monoid
hom.
Given an add_monoid
hom f : γ → M
whose image is contained in
an add_submonoid
s, the induced map from γ
to s
is an add_monoid
hom.
Given a monoid hom f : γ → M
whose image is contained in a submonoid s
, the induced map
from γ
to s
is a monoid hom.
Equations
- _ = _
Given two submonoids s
and t
such that s ⊆ t
, the natural injection from s
into t
is
a monoid hom.
Equations
- _ = _
Given two add_submonoid
s s
and t
such that s ⊆ t
, the
natural injection from s
into t
is an add_monoid
hom.
- basic : ∀ {A : Type u_2} [_inst_2 : add_monoid A] (s : set A) {a : A}, a ∈ s → add_monoid.in_closure s a
- zero : ∀ {A : Type u_2} [_inst_2 : add_monoid A] (s : set A), add_monoid.in_closure s 0
- add : ∀ {A : Type u_2} [_inst_2 : add_monoid A] (s : set A) {a b : A}, add_monoid.in_closure s a → add_monoid.in_closure s b → add_monoid.in_closure s (a + b)
The inductively defined membership predicate for the submonoid generated by a subset of a monoid.
- basic : ∀ {M : Type u_1} [_inst_1 : monoid M] (s : set M) {a : M}, a ∈ s → monoid.in_closure s a
- one : ∀ {M : Type u_1} [_inst_1 : monoid M] (s : set M), monoid.in_closure s 1
- mul : ∀ {M : Type u_1} [_inst_1 : monoid M] (s : set M) {a b : M}, monoid.in_closure s a → monoid.in_closure s b → monoid.in_closure s (a * b)
The inductively defined membership predicate for the add_submonoid
generated by a subset of an
add_monoid.
The inductively defined add_submonoid
genrated by a subset of an add_monoid
.
The inductively defined submonoid generated by a subset of a monoid.
Equations
- monoid.closure s = {a : M | monoid.in_closure s a}
Equations
- _ = _
A subset of an add_monoid
is contained in the add_submonoid
it generates.
A subset of a monoid is contained in the submonoid it generates.
The add_submonoid
generated by a set is contained in any add_submonoid
that
contains the set.
The submonoid generated by a set is contained in any submonoid that contains the set.
Given subsets t
and s
of a monoid M
, if s ⊆ t
, the submonoid of M
generated by s
is
contained in the submonoid generated by t
.
Given subsets t
and s
of an add_monoid M
, if s ⊆ t
, the add_submonoid
of M
generated by s
is contained in the add_submonoid
generated by t
.
The add_submonoid
generated by an element of an add_monoid
equals the set of
natural number multiples of the element.
The submonoid generated by an element of a monoid equals the set of natural number powers of the element.
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 under the add_monoid
hom.
The image under a monoid hom of the submonoid generated by a set equals the submonoid generated by the image of the set under the monoid hom.
Given an element a
of the submonoid of a monoid M
generated by a set s
, there exists
a list of elements of s
whose product is a
.
Given an element a
of the add_submonoid
of an add_monoid M
generated by
a set s
, there exists a list of elements of s
whose sum is a
.
Given sets s, t
of a commutative add_monoid M
, x ∈ M
is in the add_submonoid
of M
generated by s ∪ t
iff there exists an element of the add_submonoid
generated by s
and an element of the add_submonoid
generated by t
whose sum is x
.
Given sets s, t
of a commutative monoid M
, x ∈ M
is in the submonoid of M
generated by
s ∪ t
iff there exists an element of the submonoid generated by s
and an element of the
submonoid generated by t
whose product is x
.
Create a bundled submonoid from a set s
and [is_submonoid s]
.
Create a bundled additive submonoid from a set s
and [is_add_submonoid s]
.
Equations
- _ = _