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

Commit 767901a

Browse files
committed
feat(algebra/ordered_ring): a + 1 ≤ 2 * a (#7995)
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`.
1 parent fae00c7 commit 767901a

File tree

1 file changed

+6
-0
lines changed

1 file changed

+6
-0
lines changed

src/algebra/ordered_ring.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -16,6 +16,12 @@ set_option old_structure_cmd true
1616
universe u
1717
variable {α : Type u}
1818

19+
lemma add_one_le_two_mul [preorder α] [semiring α] [covariant_class α α (+) (≤)]
20+
{a : α} (a1 : 1 ≤ a) :
21+
a + 12 * a :=
22+
calc a + 1 ≤ a + a : add_le_add_left a1 a
23+
... = 2 * a : (two_mul _).symm
24+
1925
/-- An `ordered_semiring α` is a semiring `α` with a partial order such that
2026
multiplication with a positive number and addition are monotone. -/
2127
@[protect_proj]

0 commit comments

Comments
 (0)