File tree Expand file tree Collapse file tree 1 file changed +8
-1
lines changed
Mathlib/Algebra/Order/Field Expand file tree Collapse file tree 1 file changed +8
-1
lines changed Original file line number Diff line number Diff line change @@ -3,7 +3,7 @@ Copyright (c) 2014 Robert Lewis. All rights reserved.
3
3
Released under Apache 2.0 license as described in the file LICENSE.
4
4
Authors: Robert Lewis, Leonardo de Moura, Mario Carneiro, Floris van Doorn
5
5
! This file was ported from Lean 3 source module algebra.order.field.basic
6
- ! leanprover-community/mathlib commit f835503164c75764d4165d9e630bf27694d73ec6
6
+ ! leanprover-community/mathlib commit 5a82b0671532663333e205f422124a98bdfe673f
7
7
! Please do not edit these lines, except to modify the commit id
8
8
! if you have ported upstream changes.
9
9
-/
@@ -234,6 +234,13 @@ theorem div_le_of_nonneg_of_le_mul (hb : 0 ≤ b) (hc : 0 ≤ c) (h : a ≤ c *
234
234
rwa [div_le_iff hb']
235
235
#align div_le_of_nonneg_of_le_mul div_le_of_nonneg_of_le_mul
236
236
237
+ /-- One direction of `div_le_iff` where `c` is allowed to be `0` (but `b` must be nonnegative) -/
238
+ lemma mul_le_of_nonneg_of_le_div (hb : 0 ≤ b) (hc : 0 ≤ c) (h : a ≤ b / c) : a * c ≤ b := by
239
+ obtain rfl | hc := hc.eq_or_lt
240
+ . simpa using hb
241
+ . rwa [le_div_iff hc] at h
242
+ #align mul_le_of_nonneg_of_le_div mul_le_of_nonneg_of_le_div
243
+
237
244
theorem div_le_one_of_le (h : a ≤ b) (hb : 0 ≤ b) : a / b ≤ 1 :=
238
245
div_le_of_nonneg_of_le_mul hb zero_le_one <| by rwa [one_mul]
239
246
#align div_le_one_of_le div_le_one_of_le
You can’t perform that action at this time.
0 commit comments