src/HOL/OrderedGroup.thy
changeset 23389 aaca6a8e5414
parent 23181 f52b555f8141
child 23477 f4b83f03cac9
--- a/src/HOL/OrderedGroup.thy	Thu Jun 14 18:33:29 2007 +0200
+++ b/src/HOL/OrderedGroup.thy	Thu Jun 14 18:33:31 2007 +0200
@@ -377,10 +377,10 @@
 subsection {* Ordering Rules for Unary Minus *}
 
 lemma le_imp_neg_le:
-      assumes "a \<le> (b::'a::{pordered_ab_semigroup_add_imp_le, ab_group_add})" shows "-b \<le> -a"
+  assumes "a \<le> (b::'a::{pordered_ab_semigroup_add_imp_le, ab_group_add})" shows "-b \<le> -a"
 proof -
   have "-a+a \<le> -a+b"
-    by (rule add_left_mono) 
+    using `a \<le> b` by (rule add_left_mono) 
   hence "0 \<le> -a+b"
     by simp
   hence "0 + (-b) \<le> (-a + b) + (-b)"