File tree Expand file tree Collapse file tree 4 files changed +1893
-10
lines changed Expand file tree Collapse file tree 4 files changed +1893
-10
lines changed Original file line number Diff line number Diff line change @@ -1937,6 +1937,7 @@ import Mathlib.RingTheory.GradedAlgebra.Basic
1937
1937
import Mathlib.RingTheory.GradedAlgebra.HomogeneousIdeal
1938
1938
import Mathlib.RingTheory.GradedAlgebra.HomogeneousLocalization
1939
1939
import Mathlib.RingTheory.GradedAlgebra.Radical
1940
+ import Mathlib.RingTheory.HahnSeries
1940
1941
import Mathlib.RingTheory.Henselian
1941
1942
import Mathlib.RingTheory.Ideal.AssociatedPrime
1942
1943
import Mathlib.RingTheory.Ideal.Basic
Original file line number Diff line number Diff line change @@ -433,7 +433,7 @@ theorem addVal_uniformizer {ϖ : R} (hϖ : Irreducible ϖ) : addVal R ϖ = 1 :=
433
433
using addVal_def ϖ 1 hϖ 1
434
434
#align discrete_valuation_ring.add_val_uniformizer DiscreteValuationRing.addVal_uniformizer
435
435
436
- @[simp]
436
+ -- @[ simp ] Porting note: simp can prove it
437
437
theorem addVal_mul {a b : R} :
438
438
addVal R (a * b) = addVal R a + addVal R b :=
439
439
(addVal R).map_mul _ _
You can’t perform that action at this time.
0 commit comments