Skip to content

Commit

Permalink
feat(ring_theory/dedekind_domain/ideal): add height_one_spectrum (#12244
Browse files Browse the repository at this point in the history
)
  • Loading branch information
mariainesdff committed Feb 28, 2022
1 parent 200c254 commit 33c0a1c
Showing 1 changed file with 45 additions and 0 deletions.
45 changes: 45 additions & 0 deletions src/ring_theory/dedekind_domain/ideal.lean
Expand Up @@ -19,6 +19,7 @@ Then we prove some results on the unique factorization monoid structure of the i
every nonzero fractional ideal is invertible.
- `is_dedekind_domain_inv_iff` shows that this does note depend on the choice of field of
fractions.
- `height_one_spectrum` defines the type of nonzero prime ideals of `R`.
## Main results:
- `is_dedekind_domain_iff_is_dedekind_domain_inv`
Expand Down Expand Up @@ -742,3 +743,47 @@ begin
end

end is_dedekind_domain

section height_one_spectrum

/-!
### Height one spectrum of a Dedekind domain
If `R` is a Dedekind domain of Krull dimension 1, the maximal ideals of `R` are exactly its nonzero
prime ideals.
We define `height_one_spectrum` and provide lemmas to recover the facts that prime ideals of height
one are prime and irreducible. -/

namespace is_dedekind_domain

variables [is_domain R] [is_dedekind_domain R]

/-- The height one prime spectrum of a Dedekind domain `R` is the type of nonzero prime ideals of
`R`. Note that this equals the maximal spectrum if `R` has Krull dimension 1. -/
@[nolint has_inhabited_instance unused_arguments]
structure height_one_spectrum :=
(as_ideal : ideal R)
(is_prime : as_ideal.is_prime)
(ne_bot : as_ideal ≠ ⊥)

variables (v : height_one_spectrum R) {R}

lemma height_one_spectrum.prime (v : height_one_spectrum R) : prime v.as_ideal :=
ideal.prime_of_is_prime v.ne_bot v.is_prime

lemma height_one_spectrum.irreducible (v : height_one_spectrum R) :
irreducible v.as_ideal :=
begin
rw [unique_factorization_monoid.irreducible_iff_prime],
apply v.prime,
end

lemma height_one_spectrum.associates.irreducible (v : height_one_spectrum R) :
irreducible (associates.mk v.as_ideal) :=
begin
rw [associates.irreducible_mk _],
apply v.irreducible,
end

end is_dedekind_domain

end height_one_spectrum

0 comments on commit 33c0a1c

Please sign in to comment.