Skip to content

Commit

Permalink
chore(ring_theory/hahn_series): remove redundant instances (#14045)
Browse files Browse the repository at this point in the history
Both of these instances can be proved `by apply_instance`
  • Loading branch information
ocfnash committed May 9, 2022
1 parent c43486e commit 5397ac0
Showing 1 changed file with 1 addition and 13 deletions.
14 changes: 1 addition & 13 deletions src/ring_theory/hahn_series.lean
Expand Up @@ -1179,19 +1179,7 @@ end algebra

section valuation

variables [linear_ordered_add_comm_group Γ] [ring R] [is_domain R]

instance : linear_ordered_comm_group (multiplicative Γ) :=
{ .. (infer_instance : linear_order (multiplicative Γ)),
.. (infer_instance : ordered_comm_group (multiplicative Γ)) }

instance : linear_ordered_comm_group_with_zero (with_zero (multiplicative Γ)) :=
{ zero_le_one := with_zero.zero_le 1,
.. (with_zero.ordered_comm_monoid),
.. (infer_instance : linear_order (with_zero (multiplicative Γ))),
.. (infer_instance : comm_group_with_zero (with_zero (multiplicative Γ))) }

variables (Γ) (R)
variables (Γ R) [linear_ordered_add_comm_group Γ] [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

0 comments on commit 5397ac0

Please sign in to comment.