Nilpotent elements #
This file contains results about nilpotent elements that involve ring theory.
theorem
RingHom.ker_isRadical_iff_reduced_of_surjective
{R : Type u_1}
{S : Type u_3}
{F : Type u_4}
[CommSemiring R]
[CommRing S]
[FunLike F R S]
[RingHomClass F R S]
{f : F}
(hf : Function.Surjective ⇑f)
:
The nilradical of a commutative semiring is the ideal of nilpotent elements.
Equations
- nilradical R = Ideal.radical 0
Instances For
@[simp]
@[simp]
theorem
LinearMap.isNilpotent_mulLeft_iff
(R : Type u_1)
{A : Type v}
[CommSemiring R]
[Semiring A]
[Algebra R A]
(a : A)
:
@[simp]
theorem
LinearMap.isNilpotent_mulRight_iff
(R : Type u_1)
{A : Type v}
[CommSemiring R]
[Semiring A]
[Algebra R A]
(a : A)
:
@[simp]
theorem
LinearMap.isNilpotent_toMatrix_iff
{R : Type u_1}
[CommSemiring R]
{ι : Type u_3}
{M : Type u_4}
[Fintype ι]
[DecidableEq ι]
[AddCommMonoid M]
[Module R M]
(b : Basis ι R M)
(f : M →ₗ[R] M)
:
theorem
Module.End.isNilpotent_restrict_of_le
{R : Type u_1}
{M : Type u_3}
[Semiring R]
[AddCommMonoid M]
[Module R M]
{f : End R M}
{p q : Submodule R M}
{hp : Set.MapsTo ⇑f ↑p ↑p}
{hq : Set.MapsTo ⇑f ↑q ↑q}
(h : p ≤ q)
(hf : IsNilpotent (LinearMap.restrict f hq))
:
IsNilpotent (LinearMap.restrict f hp)
theorem
Module.End.isNilpotent.restrict
{R : Type u_1}
{M : Type u_3}
[Semiring R]
[AddCommMonoid M]
[Module R M]
{f : M →ₗ[R] M}
{p : Submodule R M}
(hf : Set.MapsTo ⇑f ↑p ↑p)
(hnil : IsNilpotent f)
:
IsNilpotent (f.restrict hf)
theorem
Module.End.IsNilpotent.mapQ
{R : Type u_1}
{M : Type v}
[Ring R]
[AddCommGroup M]
[Module R M]
{f : End R M}
{p : Submodule R M}
(hp : p ≤ Submodule.comap f p)
(hnp : IsNilpotent f)
:
IsNilpotent (p.mapQ p f hp)