Skip to content

Commit

Permalink
feat(algebra/archimedean): order_dual α is archimedean (#8476)
Browse files Browse the repository at this point in the history
  • Loading branch information
urkud committed Jul 31, 2021
1 parent 339a122 commit b3943dc
Showing 1 changed file with 5 additions and 0 deletions.
5 changes: 5 additions & 0 deletions src/algebra/archimedean.lean
Expand Up @@ -35,6 +35,11 @@ such that `0 < y` there exists a natural number `n` such that `x ≤ n • y`. -
class archimedean (α) [ordered_add_comm_monoid α] : Prop :=
(arch : ∀ (x : α) {y}, 0 < y → ∃ n : ℕ, x ≤ n • y)

instance order_dual.archimedean [ordered_add_comm_group α] [archimedean α] :
archimedean (order_dual α) :=
⟨λ x y hy, let ⟨n, hn⟩ := archimedean.arch (-x : α) (neg_pos.2 hy) in
⟨n, by rwa [neg_nsmul, neg_le_neg_iff] at hn⟩⟩

namespace linear_ordered_add_comm_group
variables [linear_ordered_add_comm_group α] [archimedean α]

Expand Down

0 comments on commit b3943dc

Please sign in to comment.