equal
deleted
inserted
replaced
418 text {* TODO: move to NthRoot *} |
418 text {* TODO: move to NthRoot *} |
419 lemma sqrt_add_le_add_sqrt: |
419 lemma sqrt_add_le_add_sqrt: |
420 assumes x: "0 \<le> x" and y: "0 \<le> y" |
420 assumes x: "0 \<le> x" and y: "0 \<le> y" |
421 shows "sqrt (x + y) \<le> sqrt x + sqrt y" |
421 shows "sqrt (x + y) \<le> sqrt x + sqrt y" |
422 apply (rule power2_le_imp_le) |
422 apply (rule power2_le_imp_le) |
423 apply (simp add: real_sum_squared_expand x y) |
423 apply (simp add: power2_sum x y) |
424 apply (simp add: mult_nonneg_nonneg x y) |
424 apply (simp add: mult_nonneg_nonneg x y) |
425 apply (simp add: x y) |
425 apply (simp add: x y) |
426 done |
426 done |
427 |
427 |
428 subsection {* A generic notion of "hull" (convex, affine, conic hull and closure). *} |
428 subsection {* A generic notion of "hull" (convex, affine, conic hull and closure). *} |