add lemma real_sqrt_sum_squares_less
authorhuffman
Tue, 29 May 2007 20:31:42 +0200
changeset 23122 3d853d6f2f7d
parent 23121 5feeb93b3ba8
child 23123 e2e370bccde1
add lemma real_sqrt_sum_squares_less
src/HOL/Hyperreal/NthRoot.thy
--- a/src/HOL/Hyperreal/NthRoot.thy	Tue May 29 18:31:30 2007 +0200
+++ b/src/HOL/Hyperreal/NthRoot.thy	Tue May 29 20:31:42 2007 +0200
@@ -536,6 +536,16 @@
 apply (simp add: add_increasing)
 done
 
+lemma real_sqrt_sum_squares_less:
+  "\<lbrakk>\<bar>x\<bar> < u / sqrt 2; \<bar>y\<bar> < u / sqrt 2\<rbrakk> \<Longrightarrow> sqrt (x\<twosuperior> + y\<twosuperior>) < u"
+apply (rule power2_less_imp_less, simp)
+apply (drule power_strict_mono [OF _ abs_ge_zero pos2])
+apply (drule power_strict_mono [OF _ abs_ge_zero pos2])
+apply (simp add: power_divide)
+apply (drule order_le_less_trans [OF abs_ge_zero])
+apply (simp add: zero_less_divide_iff)
+done
+
 text{*Needed for the infinitely close relation over the nonstandard
     complex numbers*}
 lemma lemma_sqrt_hcomplex_capprox: