Documentation

Mathlib.RingTheory.Nilpotent.Lemmas

Nilpotent elements #

This file contains results about nilpotent elements that involve ring theory.

def nilradical (R : Type u_3) [CommSemiring R] :

The nilradical of a commutative semiring is the ideal of nilpotent elements.

Equations
Instances For
    theorem mem_nilradical {R : Type u_1} [CommSemiring R] {x : R} :
    theorem nilpotent_iff_mem_prime {R : Type u_1} [CommSemiring R] {x : R} :
    IsNilpotent x ∀ (J : Ideal R), Ideal.IsPrime Jx J
    theorem nilradical_le_prime {R : Type u_1} [CommSemiring R] (J : Ideal R) [H : Ideal.IsPrime J] :
    @[simp]
    theorem nilradical_eq_zero (R : Type u_3) [CommSemiring R] [IsReduced R] :
    @[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.mapQ {R : Type u_1} {M : Type v} [Ring R] [AddCommGroup M] [Module R M] {f : Module.End R M} {p : Submodule R M} (hp : p Submodule.comap f p) (hnp : IsNilpotent f) :