Skip to content

Commit

Permalink
fix(ring_theory/discrete_valuation_ring): docstring typos (#5085)
Browse files Browse the repository at this point in the history
Clarify one docstring and fix two others.
  • Loading branch information
kbuzzard committed Nov 23, 2020
1 parent e8c8ce9 commit 270fc31
Showing 1 changed file with 6 additions and 5 deletions.
11 changes: 6 additions & 5 deletions src/ring_theory/discrete_valuation_ring.lean
Original file line number Diff line number Diff line change
Expand Up @@ -45,7 +45,8 @@ universe u

open ideal local_ring

/-- An integral domain is a discrete valuation ring if it's a local PID which is not a field -/
/-- An integral domain is a *discrete valuation ring* (DVR) if it's a local PID which
is not a field. -/
class discrete_valuation_ring (R : Type u) [integral_domain R]
extends is_principal_ideal_ring R, local_ring R : Prop :=
(not_a_field' : maximal_ideal R ≠ ⊥)
Expand Down Expand Up @@ -169,10 +170,10 @@ begin
exact (hϖ.not_unit (is_unit_of_mul_is_unit_left H0)).elim } }
end

/-- Implementation detail: an integral domain in which there is a unit `p`
/-- An integral domain in which there is an irreducible element `p`
such that every nonzero element is associated to a power of `p` is a unique factorization domain.
See `discrete_valuation_ring.of_has_unit_mul_pow_irreducible_factorization`. -/
theorem ufd : unique_factorization_monoid R :=
theorem to_unique_factorization_monoid : unique_factorization_monoid R :=
let p := classical.some hR in
let spec := classical.some_spec hR in
unique_factorization_monoid.of_exists_prime_factors $ λ x hx,
Expand Down Expand Up @@ -286,15 +287,15 @@ begin
end

/--
An integral domain in which there is a unit `p`
An integral domain in which there is an irreducible element `p`
such that every nonzero element is associated to a power of `p`
is a discrete valuation ring.
-/
lemma of_has_unit_mul_pow_irreducible_factorization {R : Type u} [integral_domain R]
(hR : has_unit_mul_pow_irreducible_factorization R) :
discrete_valuation_ring R :=
begin
letI : unique_factorization_monoid R := hR.ufd,
letI : unique_factorization_monoid R := hR.to_unique_factorization_monoid,
apply of_ufd_of_unique_irreducible _ hR.unique_irreducible,
unfreezingI { obtain ⟨p, hp, H⟩ := hR, exact ⟨p, hp⟩, },
end
Expand Down

0 comments on commit 270fc31

Please sign in to comment.