Skip to content
This repository was archived by the owner on Jul 24, 2024. It is now read-only.

Commit 006f84e

Browse files
committed
feat(algebra/group_power/basic): add add le_of_pow_le_pow (#5054)
add a random missing lemma
1 parent 1fbdf77 commit 006f84e

File tree

1 file changed

+3
-0
lines changed

1 file changed

+3
-0
lines changed

src/algebra/group_power/basic.lean

Lines changed: 3 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -588,6 +588,9 @@ lemma pow_le_pow_of_le_left {a b : R} (ha : 0 ≤ a) (hab : a ≤ b) : ∀ i :
588588
lemma lt_of_pow_lt_pow {a b : R} (n : ℕ) (hb : 0 ≤ b) (h : a ^ n < b ^ n) : a < b :=
589589
lt_of_not_ge $ λ hn, not_lt_of_ge (pow_le_pow_of_le_left hb hn _) h
590590

591+
lemma le_of_pow_le_pow {a b : R} (n : ℕ) (hb : 0 ≤ b) (hn : 0 < n) (h : a ^ n ≤ b ^ n) : a ≤ b :=
592+
le_of_not_lt $ λ h1, not_le_of_lt (pow_lt_pow_of_lt_left h1 hb hn) h
593+
591594
end linear_ordered_semiring
592595

593596
theorem pow_two_nonneg [linear_ordered_ring R] (a : R) : 0 ≤ a ^ 2 :=

0 commit comments

Comments
 (0)