src/HOL/RealDef.thy
changeset 44349 f057535311c5
parent 44348 40101794c52f
child 44350 63cddfbc5a09
--- a/src/HOL/RealDef.thy	Sat Aug 20 13:07:00 2011 -0700
+++ b/src/HOL/RealDef.thy	Sat Aug 20 15:54:26 2011 -0700
@@ -1553,11 +1553,6 @@
 
 subsection{* Simprules combining x+y and 0: ARE THEY NEEDED?*}
 
-text{*Needed in this non-standard form by Hyperreal/Transcendental*}
-lemma real_0_le_divide_iff:
-     "((0::real) \<le> x/y) = ((x \<le> 0 | 0 \<le> y) & (0 \<le> x | y \<le> 0))"
-by (auto simp add: zero_le_divide_iff)
-
 lemma real_add_minus_iff [simp]: "(x + - a = (0::real)) = (x=a)" 
 by arith