Skip to content

Commit a8d2931

Browse files
committed
chore: rename valuation_posSubmonoid_ne_zero_of_compatible (#28040)
and sneak one more lemma in
1 parent f77f5d6 commit a8d2931

File tree

1 file changed

+10
-1
lines changed

1 file changed

+10
-1
lines changed

Mathlib/RingTheory/Valuation/ValuativeRel.lean

Lines changed: 10 additions & 1 deletion
Original file line numberDiff line numberDiff 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+
560569
variable (R) in
561570
/-- An alias for endowing a ring with a preorder defined as the valuative relation. -/
562571
def WithPreorder := R

0 commit comments

Comments
 (0)