Skip to content

Commit 8e985cd

Browse files
committed
chore(Algebra/Order/Nonneg/Basic): remove duplicate Nonneg.pow_nonneg (#24997)
This lemma already exists in the root namespace, so it is a duplicate.
1 parent e262afd commit 8e985cd

File tree

1 file changed

+2
-3
lines changed

1 file changed

+2
-3
lines changed

Mathlib/Algebra/Order/Nonneg/Basic.lean

Lines changed: 2 additions & 3 deletions
Original file line numberDiff line numberDiff line change
@@ -177,9 +177,6 @@ section Pow
177177

178178
variable [MonoidWithZero α] [Preorder α] [ZeroLEOneClass α] [PosMulMono α]
179179

180-
theorem pow_nonneg {a : α} (H : 0 ≤ a) : ∀ n : ℕ, 0 ≤ a ^ n := by
181-
simp [H]
182-
183180
instance pow : Pow { x : α // 0 ≤ x } ℕ where
184181
pow x n := ⟨(x : α) ^ n, pow_nonneg x.2 n⟩
185182

@@ -193,6 +190,8 @@ theorem mk_pow {x : α} (hx : 0 ≤ x) (n : ℕ) :
193190
(⟨x, hx⟩ : { x : α // 0 ≤ x }) ^ n = ⟨x ^ n, pow_nonneg hx n⟩ :=
194191
rfl
195192

193+
@[deprecated (since := "2025-05-19")] alias pow_nonneg := _root_.pow_nonneg
194+
196195
end Pow
197196

198197
section Semiring

0 commit comments

Comments
 (0)