File tree Expand file tree Collapse file tree 1 file changed +10
-1
lines changed
Mathlib/RingTheory/Valuation Expand file tree Collapse file tree 1 file changed +10
-1
lines changed Original file line number Diff line number Diff line change @@ -552,11 +552,20 @@ lemma isEquiv {Γ₁ Γ₂ : Type*}
552552 simp_rw [← Valuation.Compatible.rel_iff_le]
553553
554554@[simp]
555- lemma valuation_posSubmonoid_ne_zero_of_compatible {Γ : Type *} [LinearOrderedCommMonoidWithZero Γ]
555+ lemma _root_.Valuation.apply_posSubmonoid_ne_zero {Γ : Type *} [LinearOrderedCommMonoidWithZero Γ]
556556 (v : Valuation R Γ) [v.Compatible] (x : posSubmonoid R) :
557557 v (x : R) ≠ 0 := by
558558 simp [(isEquiv v (valuation R)).ne_zero, valuation_posSubmonoid_ne_zero]
559559
560+ @[deprecated (since := "2025-08-06")]
561+ alias valuation_posSubmonoid_ne_zero_of_compatible := _root_.Valuation.apply_posSubmonoid_ne_zero
562+
563+ @[simp]
564+ lemma _root_.Valuation.apply_posSubmonoid_pos {Γ : Type *} [LinearOrderedCommMonoidWithZero Γ]
565+ (v : Valuation R Γ) [v.Compatible] (x : posSubmonoid R) :
566+ 0 < v x :=
567+ zero_lt_iff.mpr <| v.apply_posSubmonoid_ne_zero x
568+
560569variable (R) in
561570/-- An alias for endowing a ring with a preorder defined as the valuative relation. -/
562571def WithPreorder := R
You can’t perform that action at this time.
0 commit comments