mathlib documentation

ring_theory.​jacobson_ideal

ring_theory.​jacobson_ideal

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} [comm_ring R] :
ideal Rideal R

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

Equations
theorem ideal.​le_jacobson {R : Type u} [comm_ring R] {I : ideal R} :

theorem ideal.​radical_le_jacobson {R : Type u} [comm_ring R] {I : ideal R} :

theorem ideal.​eq_radical_of_eq_jacobson {R : Type u} [comm_ring R] {I : ideal R} :
I.jacobson = II.radical = I

@[simp]
theorem ideal.​jacobson_top {R : Type u} [comm_ring R] :

@[simp]
theorem ideal.​jacobson_eq_top_iff {R : Type u} [comm_ring R] {I : ideal R} :

theorem ideal.​jacobson_eq_bot {R : Type u} [comm_ring R] {I : ideal R} :
I.jacobson = I =

theorem ideal.​jacobson_eq_self_of_is_maximal {R : Type u} [comm_ring R] {I : ideal R} [H : I.is_maximal] :

@[instance]
def ideal.​jacobson.​is_maximal {R : Type u} [comm_ring R] {I : ideal R} [H : I.is_maximal] :

Equations
theorem ideal.​mem_jacobson_iff {R : Type u} [comm_ring R] {I : ideal R} {x : R} :
x I.jacobson ∀ (y : R), ∃ (z : R), x * y * z + z - 1 I

theorem ideal.​eq_jacobson_iff_Inf_maximal {R : Type u} [comm_ring R] {I : ideal R} :
I.jacobson = I ∃ (M : set (ideal R)), (∀ (J : ideal R), J MJ.is_maximal J = ) I = has_Inf.Inf 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_Inf_maximal' {R : Type u} [comm_ring R] {I : ideal R} :
I.jacobson = I ∃ (M : set (ideal R)), (∀ (J : ideal R), J M∀ (K : ideal R), J < KK = ) I = has_Inf.Inf M

theorem ideal.​eq_jacobson_iff_not_mem {R : Type u} [comm_ring R] {I : ideal R} :
I.jacobson = I ∀ (x : R), x I(∃ (M : ideal R), (I M M.is_maximal) x M)

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} [comm_ring R] {S : Type v} [comm_ring S] {f : R →+* S} (hf : function.surjective f) {I : ideal R} :

theorem ideal.​comap_jacobson_of_surjective {R : Type u} [comm_ring R] {S : Type v} [comm_ring S] {f : R →+* S} (hf : function.surjective f) {K : ideal S} :

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

theorem ideal.​jacobson_mono {R : Type u} [comm_ring R] {I J : ideal R} :
I JI.jacobson J.jacobson

@[class]
def ideal.​is_local {R : Type u} [comm_ring R] :
ideal R → Prop

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

Equations
theorem ideal.​is_local.​le_jacobson {R : Type u} [comm_ring R] {I J : ideal R} :
I.is_localI JJ J I.jacobson

theorem ideal.​is_local.​mem_jacobson_or_exists_inv {R : Type u} [comm_ring R] {I : ideal R} (hi : I.is_local) (x : R) :
x I.jacobson ∃ (y : R), y * x - 1 I