Skip to content

Commit

Permalink
feat(ring_theory/hahn_series): Loosen definition of additive valuation (
Browse files Browse the repository at this point in the history
#17057)

The definitions and theorems realted to the additive valuation of Hahn series don't actually require the value group to be a group; just a cancellative monoid, as in the rest of the file.

This came about while I was thinking about Bhargava's recent proof of van der Waerden's theorem and I wondered how hard proving, say, the irreducibility theorem would be in mathlib.
  • Loading branch information
khwilson committed Oct 19, 2022
1 parent 91b3301 commit cb8faf7
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions src/ring_theory/hahn_series.lean
Expand Up @@ -1159,7 +1159,7 @@ end algebra

section valuation

variables (Γ R) [linear_ordered_add_comm_group Γ] [ring R] [is_domain R]
variables (Γ R) [linear_ordered_cancel_add_comm_monoid Γ] [ring R] [is_domain R]

/-- The additive valuation on `hahn_series Γ R`, returning the smallest index at which
a Hahn Series has a nonzero coefficient, or `⊤` for the 0 series. -/
Expand Down Expand Up @@ -1208,7 +1208,7 @@ end
end valuation

lemma is_pwo_Union_support_powers
[linear_ordered_add_comm_group Γ] [ring R] [is_domain R]
[linear_ordered_cancel_add_comm_monoid Γ] [ring R] [is_domain R]
{x : hahn_series Γ R} (hx : 0 < add_val Γ R x) :
(⋃ n : ℕ, (x ^ n).support).is_pwo :=
begin
Expand Down Expand Up @@ -1531,7 +1531,7 @@ end emb_domain

section powers

variables [linear_ordered_add_comm_group Γ] [comm_ring R] [is_domain R]
variables [linear_ordered_cancel_add_comm_monoid Γ] [comm_ring R] [is_domain R]

/-- The powers of an element of positive valuation form a summable family. -/
def powers (x : hahn_series Γ R) (hx : 0 < add_val Γ R x) :
Expand Down

0 comments on commit cb8faf7

Please sign in to comment.