Zulip Chat Archive

Stream: maths

Topic: Valuation rings that are not domains


Yakov Pechersky (Oct 10 2024 at 00:36):

I am working on formalizing Kaplansky's theorem, which states that

For commutative Noetherian R, R is a PIR iff every maximal ideal is principal.

In fact, his theorem is a classification of noetherian commutative rings -- every such ring can be decomposed as a finite direct sum of integral domains and valuation rings (with DCC).
image.png

Yakov Pechersky (Oct 10 2024 at 00:37):

However, this classification is not possible to state in this manner in mathlib, since ValuationRing assumes IsDomain.

Yakov Pechersky (Oct 10 2024 at 00:39):

There are rings that satisfy the axioms of ValuationRing that cannot satisfy IsDomain, and Mathlib knows about one such example: K[X] / X^2 where K is a field. Formalized as the dual numbers over K:

import Mathlib.RingTheory.DualNumber
import Mathlib.RingTheory.Valuation.ValuationRing

open DualNumber

variable {K : Type*} [Field K]

#synth IsPrincipalIdealRing K[ε]
#synth LocalRing K[ε]
#synth IsBezout K[ε]
#check maximalIdeal_eq_span_singleton_eps -- maximal ideal is not bot; requirement for DVR
#check exists_mul_left_or_mul_right -- ∀ (a b : K[ε]), ∃ c, a * c = b ∨ b * c = a
#check ValuationRing.cond' -- ∀ (a b : A), ∃ (c : A), a * c = b ∨ b * c = a
-- but we can't have IsDomain K[ε], since ε is nilpotent
#check isNilpotent_eps

Yakov Pechersky (Oct 10 2024 at 00:42):

Can the _definition_ of ValuationRing (and possibly DVR) be loosened to not require IsDomain? A small number of theorems would also no longer require it. And it would allow me to state the classification. Otherwise, I'll have to express the classification as a direct sum of integral domains and rings-that-have-the-valuation-ring-condition-but-not-as-a-class.

Johan Commelin (Oct 10 2024 at 01:16):

Weakening valuation ring sounds fine to me. I'm less sure about DVR. Is there literature on DVRs that are not domains? Would mathlib need a DVD concept?

Yakov Pechersky (Oct 10 2024 at 01:21):

I guess for DVR, my only current argument is consistency with the VR definition

Adam Topaz (Oct 10 2024 at 01:24):

Deligne has paper(s?) on "truncated DVRs"

Ruben Van de Velde (Oct 10 2024 at 05:49):

This one? https://github.com/riccardobrasca/kaplanski4/tree/master

Cc @Riccardo Brasca

Kevin Buzzard (Oct 10 2024 at 06:00):

I think that we shouldn't deviate from the terminology used in the literature...

Damiano Testa (Oct 10 2024 at 06:03):

I agree that we should not deviate from established names: I'd rather have preDVR and DVR, rather than using DVD for what everyone else calls a DVR.

Johan Commelin (Oct 10 2024 at 06:32):

Right, but what about valuation ring?

Damiano Testa (Oct 10 2024 at 06:38):

Maybe there should be a typeclass that only assumes Mul, since this seems to be all that ValuationRing actually uses? And then we can reserve the ValuationRing name for the more restricted one?

Riccardo Brasca (Oct 10 2024 at 07:48):

Ruben Van de Velde said:

This one? https://github.com/riccardobrasca/kaplanski4/tree/master

Cc Riccardo Brasca

I am not sure what "this one" refers to, but that repo contains a proof of the fact that an integral domain is a UFD if and only if every nonzero prime ideal contains a prime element. It is not directly related to DVRs.

Yakov Pechersky (Oct 10 2024 at 11:32):

Kevin Buzzard said:

I think that we shouldn't deviate from the terminology used in the literature...

Ah, but the Kaplansky reference is part of the literature :upside_down:

Yakov Pechersky (Oct 11 2024 at 04:19):

https://github.com/leanprover-community/mathlib4/pull/17634


Last updated: May 02 2025 at 03:31 UTC