Skip to content

Commit

Permalink
feat: port RingTheory.HahnSeries (#4261)
Browse files Browse the repository at this point in the history
  • Loading branch information
ChrisHughes24 committed May 23, 2023
1 parent 9594d4a commit 178cf0f
Show file tree
Hide file tree
Showing 4 changed files with 1,893 additions and 10 deletions.
1 change: 1 addition & 0 deletions Mathlib.lean
Expand Up @@ -1937,6 +1937,7 @@ import Mathlib.RingTheory.GradedAlgebra.Basic
import Mathlib.RingTheory.GradedAlgebra.HomogeneousIdeal
import Mathlib.RingTheory.GradedAlgebra.HomogeneousLocalization
import Mathlib.RingTheory.GradedAlgebra.Radical
import Mathlib.RingTheory.HahnSeries
import Mathlib.RingTheory.Henselian
import Mathlib.RingTheory.Ideal.AssociatedPrime
import Mathlib.RingTheory.Ideal.Basic
Expand Down
2 changes: 1 addition & 1 deletion Mathlib/RingTheory/DiscreteValuationRing/Basic.lean
Expand Up @@ -433,7 +433,7 @@ theorem addVal_uniformizer {ϖ : R} (hϖ : Irreducible ϖ) : addVal R ϖ = 1 :=
using addVal_def ϖ 11
#align discrete_valuation_ring.add_val_uniformizer DiscreteValuationRing.addVal_uniformizer

@[simp]
--@[simp] Porting note: simp can prove it
theorem addVal_mul {a b : R} :
addVal R (a * b) = addVal R a + addVal R b :=
(addVal R).map_mul _ _
Expand Down

0 comments on commit 178cf0f

Please sign in to comment.