Skip to content

Commit

Permalink
feat(algebra/archimedean): pow_unbounded_of_gt_one (#50)
Browse files Browse the repository at this point in the history
  • Loading branch information
ChrisHughes24 authored and johoelzl committed Feb 19, 2018
1 parent 500dcc9 commit 3c25d94
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions algebra/archimedean.lean
Original file line number Diff line number Diff line change
Expand Up @@ -107,6 +107,14 @@ let ⟨n, h⟩ := archimedean.arch x zero_lt_one in
section linear_ordered_ring
variables [linear_ordered_ring α] [archimedean α]

lemma pow_unbounded_of_gt_one (x : α) {y : α}
(hy1 : 1 < y) : ∃ n : ℕ, x < monoid.pow y n :=
have hy0 : 0 < y - 1 := sub_pos_of_lt hy1,
let ⟨n, h⟩ := archimedean.arch x hy0 in
⟨n, calc x ≤ (y - 1) • n : h
... < 1 + (y - 1) • n : by rw add_comm; exact lt_add_one _
... ≤ monoid.pow y n : pow_ge_one_add_sub_mul (le_of_lt hy1) _⟩

theorem exists_int_gt (x : α) : ∃ n : ℤ, x < n :=
let ⟨n, h⟩ := exists_nat_gt x in ⟨n, by simp [h]⟩

Expand Down

0 comments on commit 3c25d94

Please sign in to comment.