Skip to content

Commit 178cf0f

Browse files
committed
feat: port RingTheory.HahnSeries (#4261)
1 parent 9594d4a commit 178cf0f

File tree

4 files changed

+1893
-10
lines changed

4 files changed

+1893
-10
lines changed

Mathlib.lean

Lines changed: 1 addition & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -1937,6 +1937,7 @@ import Mathlib.RingTheory.GradedAlgebra.Basic
19371937
import Mathlib.RingTheory.GradedAlgebra.HomogeneousIdeal
19381938
import Mathlib.RingTheory.GradedAlgebra.HomogeneousLocalization
19391939
import Mathlib.RingTheory.GradedAlgebra.Radical
1940+
import Mathlib.RingTheory.HahnSeries
19401941
import Mathlib.RingTheory.Henselian
19411942
import Mathlib.RingTheory.Ideal.AssociatedPrime
19421943
import Mathlib.RingTheory.Ideal.Basic

Mathlib/RingTheory/DiscreteValuationRing/Basic.lean

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -433,7 +433,7 @@ theorem addVal_uniformizer {ϖ : R} (hϖ : Irreducible ϖ) : addVal R ϖ = 1 :=
433433
using addVal_def ϖ 11
434434
#align discrete_valuation_ring.add_val_uniformizer DiscreteValuationRing.addVal_uniformizer
435435

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

0 commit comments

Comments
 (0)