remove outdated comment
authorhuffman
Thu, 12 Apr 2012 07:33:14 +0200
changeset 47428 45b58fec9024
parent 47427 0daa97ed1585
child 47429 ec64d94cbf9c
child 47437 4625ee486ff6
remove outdated comment
src/HOL/RealDef.thy
--- a/src/HOL/RealDef.thy	Wed Apr 11 21:40:46 2012 +0200
+++ b/src/HOL/RealDef.thy	Thu Apr 12 07:33:14 2012 +0200
@@ -1058,8 +1058,7 @@
 by simp (* solved by linordered_ring_le_cancel_factor simproc *)
 
 lemma real_mult_le_cancel_iff2 [simp]: "(0::real) < z ==> (z*x \<le> z*y) = (x\<le>y)"
-by (rule mult_le_cancel_left_pos)
-(* BH: Why doesn't "simp" prove this one, like it does the last one? *)
+by simp (* solved by linordered_ring_le_cancel_factor simproc *)
 
 
 subsection {* Embedding numbers into the Reals *}