Fix for simplified divide_mono theorem
authorpaulson <lp15@cam.ac.uk>
Mon, 29 Jul 2024 10:24:54 +0100
changeset 80622 0c4d17ef855d
parent 80621 6c369fec315a
child 80623 424b90ba7b6f
Fix for simplified divide_mono theorem
src/HOL/Fields.thy
--- a/src/HOL/Fields.thy	Mon Jul 29 10:13:52 2024 +0100
+++ b/src/HOL/Fields.thy	Mon Jul 29 10:24:54 2024 +0100
@@ -1156,7 +1156,7 @@
 lemma divide_right_mono_neg: "a \<le> b \<Longrightarrow> c \<le> 0 \<Longrightarrow> b / c \<le> a / c"
   by (auto dest: divide_right_mono [of _ _ "- c"])
 
-lemma divide_left_mono_neg: "a \<le> b \<Longrightarrow> c \<le> 0 \<Longrightarrow> 0 < a * b \<Longrightarrow> c / a \<le> c / b"
+lemma divide_left_mono_neg: "a \<le> b \<Longrightarrow> c \<le> 0 \<Longrightarrow> 0 < a \<Longrightarrow> c / a \<le> c / b"
   by (auto simp add: mult.commute dest: divide_left_mono [of _ _ "- c"])
 
 lemma inverse_le_iff: "inverse a \<le> inverse b \<longleftrightarrow> (0 < a * b \<longrightarrow> b \<le> a) \<and> (a * b \<le> 0 \<longrightarrow> a \<le> b)"