Skip to content

Commit 04818fd

Browse files
committed
feat: a ≤ b / c → a * c ≤ b (#2027)
Match leanprover-community/mathlib3#18367
1 parent 5d55252 commit 04818fd

File tree

1 file changed

+8
-1
lines changed

1 file changed

+8
-1
lines changed

Mathlib/Algebra/Order/Field/Basic.lean

Lines changed: 8 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -3,7 +3,7 @@ Copyright (c) 2014 Robert Lewis. All rights reserved.
33
Released under Apache 2.0 license as described in the file LICENSE.
44
Authors: Robert Lewis, Leonardo de Moura, Mario Carneiro, Floris van Doorn
55
! 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
77
! Please do not edit these lines, except to modify the commit id
88
! if you have ported upstream changes.
99
-/
@@ -234,6 +234,13 @@ theorem div_le_of_nonneg_of_le_mul (hb : 0 ≤ b) (hc : 0 ≤ c) (h : a ≤ c *
234234
rwa [div_le_iff hb']
235235
#align div_le_of_nonneg_of_le_mul div_le_of_nonneg_of_le_mul
236236

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+
237244
theorem div_le_one_of_le (h : a ≤ b) (hb : 0 ≤ b) : a / b ≤ 1 :=
238245
div_le_of_nonneg_of_le_mul hb zero_le_one <| by rwa [one_mul]
239246
#align div_le_one_of_le div_le_one_of_le

0 commit comments

Comments
 (0)