Documentation

Mathlib.RingTheory.Nilpotent.GeometricallyReduced

Geometrically reduced algebras #

In this file we introduce geometrically reduced algebras. For a field k, we say that a k-algebra A is geometrically reduced (IsGeometricallyReduced) if the tensor product AlgebraicClosure k ⊗[k] A is reduced.

Main results #

References #

TODO #

class Algebra.IsGeometricallyReduced (k : Type u_3) (A : Type u_4) [Field k] [Ring A] [Algebra k A] :

The k-algebra A is geometrically reduced iff its base change to AlgebraicClosure k is reduced.

Instances
    theorem Algebra.IsGeometricallyReduced.of_injective {k : Type u_1} {A : Type u_2} [Field k] [Ring A] [Algebra k A] {B : Type u_3} [Ring B] [Algebra k B] (f : A →ₐ[k] B) (hf : Function.Injective f) [IsGeometricallyReduced k B] :
    theorem Algebra.IsGeometricallyReduced.of_forall_fg {k : Type u_1} {A : Type u_2} [Field k] [Ring A] [Algebra k A] (h : ∀ (B : Subalgebra k A), B.FGIsGeometricallyReduced k B) :

    If all finitely generated subalgebras of A are geometrically reduced, then A is geometrically reduced.