Finiteness conditions in commutative algebra #
THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.
In this file we define several notions of finiteness that are common in commutative algebra.
Main declarations #
module.finite
,algebra.finite
,ring_hom.finite
,alg_hom.finite
all of these express that some object is finitely generated as module over some base ring.algebra.finite_type
,ring_hom.finite_type
,alg_hom.finite_type
all of these express that some object is finitely generated as algebra over some base ring.algebra.finite_presentation
,ring_hom.finite_presentation
,alg_hom.finite_presentation
all of these express that some object is finitely presented as algebra over some base ring.
An algebra over a commutative semiring is finite_presentation
if it is the quotient of a
polynomial ring in n
variables by a finitely generated ideal.
Equations
- algebra.finite_presentation R A = ∃ (n : ℕ) (f : mv_polynomial (fin n) R →ₐ[R] A), function.surjective ⇑f ∧ (ring_hom.ker f.to_ring_hom).fg
An algebra over a Noetherian ring is finitely generated if and only if it is finitely presented.
The ring of polynomials in finitely many variables is finitely presented.
R
is finitely presented as R
-algebra.
R[X]
is finitely presented as R
-algebra.
The quotient of a finitely presented algebra by a finitely generated ideal is finitely presented.
If f : A →ₐ[R] B
is surjective with finitely generated kernel and A
is finitely presented,
then so is B
.
An algebra is finitely presented if and only if it is a quotient of a polynomial ring whose variables are indexed by a fintype by a finitely generated ideal.
If A
is a finitely presented R
-algebra, then mv_polynomial (fin n) A
is finitely presented
as R
-algebra.
If A
is an R
-algebra and S
is an A
-algebra, both finitely presented, then S
is
finitely presented as R
-algebra.
This is used to prove the strictly stronger ker_fg_of_surjective
. Use it instead.
If f : A →ₐ[R] B
is a sujection between finitely-presented R
-algebras, then the kernel of
f
is finitely generated.
An algebra morphism A →ₐ[R] B
is of finite_presentation
if it is of finite presentation as
ring morphism. In other words, if B
is finitely presented as A
-algebra.