Non-unital Subalgebras over Commutative Semirings #
In this file we define NonUnitalSubalgebra
s and the usual operations on them (map
, comap
).
TODO #
- once we have scalar actions by semigroups (as opposed to monoids), implement the action of a non-unital subalgebra on the larger algebra.
Embedding of a non-unital subalgebra into the non-unital algebra.
Instances For
A non-unital subalgebra is a sub(semi)ring that is also a submodule.
Instances For
Reinterpret a NonUnitalSubalgebra
as a Submodule
.
Instances For
Copy of a non-unital subalgebra with a new carrier
equal to the old one.
Useful to fix definitional equalities.
Instances For
A non-unital subalgebra over a ring is also a Subring
.
Instances For
NonUnitalSubalgebra
s inherit structure from their NonUnitalSubsemiring
/ Semiring
coercions.
The forgetful map from NonUnitalSubalgebra
to Submodule
as an OrderEmbedding
Instances For
The forgetful map from NonUnitalSubalgebra
to NonUnitalSubsemiring
as an
OrderEmbedding
Instances For
The forgetful map from NonUnitalSubalgebra
to NonUnitalSubsemiring
as an
OrderEmbedding
Instances For
NonUnitalSubalgebra
s inherit structure from their Submodule
coercions. #
Linear equivalence between S : Submodule R A
and S
. Though these types are equal,
we define it as a LinearEquiv
to avoid type equalities.
Instances For
Transport a non-unital subalgebra via an algebra homomorphism.
Instances For
Preimage of a non-unital subalgebra under an algebra homomorphism.
Instances For
A submodule closed under multiplication is a non-unital subalgebra.
Instances For
Range of an NonUnitalAlgHom
as a non-unital subalgebra.
Instances For
Restrict the codomain of a non-unital algebra homomorphism.
Instances For
Restrict the codomain of an NonUnitalAlgHom
f
to f.range
.
This is the bundled version of Set.rangeFactorization
.
Instances For
The equalizer of two non-unital R
-algebra homomorphisms
Instances For
The range of a morphism of algebras is a fintype, if the domain is a fintype.
Note that this instance can cause a diamond with Subtype.fintype
if B
is also a fintype.
The minimal non-unital subalgebra that includes s
.
Instances For
If some predicate holds for all x ∈ (s : Set A)
and this predicate is closed under the
algebraMap
, addition, multiplication and star operations, then it holds for a ∈ adjoin R s
.
The difference with NonUnitalAlgebra.adjoin_induction
is that this acts on the subtype.
Galois insertion between adjoin
and Subtype.val
.
Instances For
NonUnitalAlgHom
to ⊤ : NonUnitalSubalgebra R A
.
Instances For
The map S → T
when S
is a non-unital subalgebra contained in the non-unital subalgebra T
.
This is the non-unital subalgebra version of Submodule.ofLe
, or Subring.inclusion
Instances For
The product of two non-unital subalgebras is a non-unital subalgebra.
Instances For
Define an algebra homomorphism on a directed supremum of non-unital subalgebras by defining it on each non-unital subalgebra, and proving that it agrees on the intersection of non-unital subalgebras.
Instances For
The center of a non-unital algebra is the set of elements which commute with every element. They form a non-unital subalgebra.
Instances For
The centralizer of a set as a non-unital subalgebra.
Instances For
A non-unital subsemiring is a non-unital ℕ
-subalgebra.
Instances For
A non-unital subring is a non-unitalsubalgebra.