mathlib3 documentation

ring_theory.dedekind_domain.basic

Dedekind domains #

THIS FILE IS SYNCHRONIZED WITH MATHLIB4. Any changes to this file require a corresponding PR to mathlib4.

This file defines the notion of a Dedekind domain (or Dedekind ring), as a Noetherian integrally closed commutative ring of Krull dimension at most one.

Main definitions #

Implementation notes #

The definitions that involve a field of fractions choose a canonical field of fractions, but are independent of that choice. The ..._iff lemmas express this independence.

Often, definitions assume that Dedekind domains are not fields. We found it more practical to add a (h : ¬ is_field A) assumption whenever this is explicitly needed.

References #

Tags #

dedekind domain, dedekind ring

def ring.dimension_le_one (R : Type u_1) [comm_ring R] :
Prop

A ring R has Krull dimension at most one if all nonzero prime ideals are maximal.

Equations
theorem ring.dimension_le_one.not_lt_lt {R : Type u_1} [comm_ring R] (h : ring.dimension_le_one R) (p₀ p₁ p₂ : ideal R) [hp₁ : p₁.is_prime] [hp₂ : p₂.is_prime] :
¬(p₀ < p₁ p₁ < p₂)
theorem ring.dimension_le_one.eq_bot_of_lt {R : Type u_1} [comm_ring R] (h : ring.dimension_le_one R) (p P : ideal R) [hp : p.is_prime] [hP : P.is_prime] (hpP : p < P) :
p =
@[class]
structure is_dedekind_domain (A : Type u_2) [comm_ring A] [is_domain A] :
Prop

A Dedekind domain is an integral domain that is Noetherian, integrally closed, and has Krull dimension at most one.

This is definition 3.2 of [Neu99].

The integral closure condition is independent of the choice of field of fractions: use is_dedekind_domain_iff to prove is_dedekind_domain for a given fraction_map.

This is the default implementation, but there are equivalent definitions, is_dedekind_domain_dvr and is_dedekind_domain_inv. TODO: Prove that these are actually equivalent definitions.

Instances of this typeclass

An integral domain is a Dedekind domain iff and only if it is Noetherian, has dimension ≤ 1, and is integrally closed in a given fraction field. In particular, this definition does not depend on the choice of this fraction field.