src/HOL/NthRoot.thy
changeset 49962 a8cc904a6820
parent 49753 a344f1a21211
child 51478 270b21f3ae0a
--- a/src/HOL/NthRoot.thy	Fri Oct 19 10:46:42 2012 +0200
+++ b/src/HOL/NthRoot.thy	Fri Oct 19 15:12:52 2012 +0200
@@ -598,7 +598,7 @@
   "sqrt ((a + c)\<twosuperior> + (b + d)\<twosuperior>) \<le> sqrt (a\<twosuperior> + b\<twosuperior>) + sqrt (c\<twosuperior> + d\<twosuperior>)"
 apply (rule power2_le_imp_le, simp)
 apply (simp add: power2_sum)
-apply (simp only: mult_assoc right_distrib [symmetric])
+apply (simp only: mult_assoc distrib_left [symmetric])
 apply (rule mult_left_mono)
 apply (rule power2_le_imp_le)
 apply (simp add: power2_sum power_mult_distrib)