Skip to content

Commit

Permalink
feat(algebra/group_power/order): add pow_lt_self_of_lt_one (#17162)
Browse files Browse the repository at this point in the history
  • Loading branch information
urkud committed Oct 26, 2022
1 parent 5155be4 commit 5118ae3
Showing 1 changed file with 4 additions and 0 deletions.
4 changes: 4 additions & 0 deletions src/algebra/group_power/order.lean
Expand Up @@ -294,6 +294,10 @@ lemma pow_lt_pow_iff_of_lt_one (h₀ : 0 < a) (h₁ : a < 1) : a ^ m < a ^ n ↔
lemma pow_lt_pow_of_lt_one (h : 0 < a) (ha : a < 1) {i j : ℕ} (hij : i < j) : a ^ j < a ^ i :=
(pow_lt_pow_iff_of_lt_one h ha).2 hij

lemma pow_lt_self_of_lt_one (h₀ : 0 < a) (h₁ : a < 1) (hn : 1 < n) : a ^ n < a :=
calc a ^ n < a ^ 1 : pow_lt_pow_of_lt_one h₀ h₁ hn
... = a : pow_one _

lemma sq_pos_of_pos (ha : 0 < a) : 0 < a ^ 2 := by { rw sq, exact mul_pos ha ha }

end strict_ordered_semiring
Expand Down

0 comments on commit 5118ae3

Please sign in to comment.