We read every piece of feedback, and take your input very seriously.
To see all available qualifiers, see our documentation.
There was an error while loading. Please reload this page.
Nonneg.pow_nonneg
1 parent e262afd commit 8e985cdCopy full SHA for 8e985cd
Mathlib/Algebra/Order/Nonneg/Basic.lean
@@ -177,9 +177,6 @@ section Pow
177
178
variable [MonoidWithZero α] [Preorder α] [ZeroLEOneClass α] [PosMulMono α]
179
180
-theorem pow_nonneg {a : α} (H : 0 ≤ a) : ∀ n : ℕ, 0 ≤ a ^ n := by
181
- simp [H]
182
-
183
instance pow : Pow { x : α // 0 ≤ x } ℕ where
184
pow x n := ⟨(x : α) ^ n, pow_nonneg x.2 n⟩
185
@@ -193,6 +190,8 @@ theorem mk_pow {x : α} (hx : 0 ≤ x) (n : ℕ) :
193
190
(⟨x, hx⟩ : { x : α // 0 ≤ x }) ^ n = ⟨x ^ n, pow_nonneg hx n⟩ :=
194
191
rfl
195
192
+@[deprecated (since := "2025-05-19")] alias pow_nonneg := _root_.pow_nonneg
+
196
end Pow
197
198
section Semiring
0 commit comments