Documentation

Mathlib.RingTheory.JacobsonIdeal

Jacobson radical #

The Jacobson radical of a ring R is defined to be the intersection of all maximal ideals of R. This is similar to how the nilradical is equal to the intersection of all prime ideals of R.

We can extend the idea of the nilradical to ideals of R, by letting the radical of an ideal I be the intersection of prime ideals containing I. Under this extension, the original nilradical is the radical of the zero ideal . Here we define the Jacobson radical of an ideal I in a similar way, as the intersection of maximal ideals containing I.

Main definitions #

Let R be a commutative ring, and I be an ideal of R

Main statements #

Tags #

Jacobson, Jacobson radical, Local Ideal

def Ideal.jacobson {R : Type u} [Ring R] (I : Ideal R) :

The Jacobson radical of I is the infimum of all maximal (left) ideals containing I.

Equations
Instances For
    theorem Ideal.le_jacobson {R : Type u} [Ring R] {I : Ideal R} :
    @[simp]
    theorem Ideal.jacobson_eq_top_iff {R : Type u} [Ring R] {I : Ideal R} :
    theorem Ideal.jacobson_eq_bot {R : Type u} [Ring R] {I : Ideal R} :
    Equations
    • =
    theorem Ideal.mem_jacobson_iff {R : Type u} [Ring R] {I : Ideal R} {x : R} :
    x Ideal.jacobson I ∀ (y : R), ∃ (z : R), z * y * x + z - 1 I
    theorem Ideal.exists_mul_sub_mem_of_sub_one_mem_jacobson {R : Type u} [Ring R] {I : Ideal R} (r : R) (h : r - 1 Ideal.jacobson I) :
    ∃ (s : R), s * r - 1 I
    theorem Ideal.eq_jacobson_iff_sInf_maximal {R : Type u} [Ring R] {I : Ideal R} :
    Ideal.jacobson I = I ∃ (M : Set (Ideal R)), (JM, Ideal.IsMaximal J J = ) I = sInf M

    An ideal equals its Jacobson radical iff it is the intersection of a set of maximal ideals. Allowing the set to include ⊤ is equivalent, and is included only to simplify some proofs.

    theorem Ideal.eq_jacobson_iff_sInf_maximal' {R : Type u} [Ring R] {I : Ideal R} :
    Ideal.jacobson I = I ∃ (M : Set (Ideal R)), (JM, ∀ (K : Ideal R), J < KK = ) I = sInf M
    theorem Ideal.eq_jacobson_iff_not_mem {R : Type u} [Ring R] {I : Ideal R} :
    Ideal.jacobson I = I xI, ∃ (M : Ideal R), (I M Ideal.IsMaximal M) xM

    An ideal I equals its Jacobson radical if and only if every element outside I also lies outside of a maximal ideal containing I.

    theorem Ideal.map_jacobson_of_surjective {R : Type u} {S : Type v} [Ring R] [Ring S] {I : Ideal R} {f : R →+* S} (hf : Function.Surjective f) :
    theorem Ideal.map_jacobson_of_bijective {R : Type u} {S : Type v} [Ring R] [Ring S] {I : Ideal R} {f : R →+* S} (hf : Function.Bijective f) :
    theorem Ideal.comap_jacobson {R : Type u} {S : Type v} [Ring R] [Ring S] {f : R →+* S} {K : Ideal S} :
    theorem Ideal.jacobson_mono {R : Type u} [Ring R] {I : Ideal R} {J : Ideal R} :
    theorem Ideal.mem_jacobson_bot {R : Type u} [CommRing R] {x : R} :
    x Ideal.jacobson ∀ (y : R), IsUnit (x * y + 1)

    An ideal I of R is equal to its Jacobson radical if and only if the Jacobson radical of the quotient ring R/I is the zero ideal

    The standard radical and Jacobson radical of an ideal I of R are equal if and only if the nilradical and Jacobson radical of the quotient ring R/I coincide

    class Ideal.IsLocal {R : Type u} [CommRing R] (I : Ideal R) :

    An ideal I is local iff its Jacobson radical is maximal.

    Instances
      theorem Ideal.IsLocal.le_jacobson {R : Type u} [CommRing R] {I : Ideal R} {J : Ideal R} (hi : Ideal.IsLocal I) (hij : I J) (hj : J ) :
      theorem Ideal.IsLocal.mem_jacobson_or_exists_inv {R : Type u} [CommRing R] {I : Ideal R} (hi : Ideal.IsLocal I) (x : R) :
      x Ideal.jacobson I ∃ (y : R), y * x - 1 I