src/HOL/NthRoot.thy
changeset 44349 f057535311c5
parent 44320 33439faadd67
child 49753 a344f1a21211
--- a/src/HOL/NthRoot.thy	Sat Aug 20 13:07:00 2011 -0700
+++ b/src/HOL/NthRoot.thy	Sat Aug 20 15:54:26 2011 -0700
@@ -629,7 +629,7 @@
 apply (rule_tac y = "u/sqrt 2" in order_le_less_trans)
 apply (erule_tac [2] lemma_real_divide_sqrt_less)
 apply (rule power2_le_imp_le)
-apply (auto simp add: real_0_le_divide_iff power_divide)
+apply (auto simp add: zero_le_divide_iff power_divide)
 apply (rule_tac t = "u\<twosuperior>" in real_sum_of_halves [THEN subst])
 apply (rule add_mono)
 apply (auto simp add: four_x_squared intro: power_mono)