Skip to content

Commit

Permalink
feat(algebra/ordered_ring): a + 1 ≤ 2 * a (#7995)
Browse files Browse the repository at this point in the history
Prove one lemma, useful for the Liouville PR #4301.  The placement of the lemma will change, once the `ordered` refactor will get to  `ordered_ring`.
  • Loading branch information
adomani committed Jun 20, 2021
1 parent fae00c7 commit 767901a
Showing 1 changed file with 6 additions and 0 deletions.
6 changes: 6 additions & 0 deletions src/algebra/ordered_ring.lean
Expand Up @@ -16,6 +16,12 @@ set_option old_structure_cmd true
universe u
variable {α : Type u}

lemma add_one_le_two_mul [preorder α] [semiring α] [covariant_class α α (+) (≤)]
{a : α} (a1 : 1 ≤ a) :
a + 12 * a :=
calc a + 1 ≤ a + a : add_le_add_left a1 a
... = 2 * a : (two_mul _).symm

/-- An `ordered_semiring α` is a semiring `α` with a partial order such that
multiplication with a positive number and addition are monotone. -/
@[protect_proj]
Expand Down

0 comments on commit 767901a

Please sign in to comment.