merged
authorwenzelm
Thu, 07 Dec 2017 20:05:08 +0100
changeset 67158 a14b83897c90
parent 67156 3a9966b88a50 (diff)
parent 67157 d0657c8b7616 (current diff)
child 67159 deccbba7cfe3
merged
--- a/src/HOL/Analysis/L2_Norm.thy	Thu Dec 07 19:36:48 2017 +0100
+++ b/src/HOL/Analysis/L2_Norm.thy	Thu Dec 07 20:05:08 2017 +0100
@@ -8,7 +8,7 @@
 imports Complex_Main
 begin
 
-definition "L2_set f A = sqrt (\<Sum>i\<in>A. (f i)\<^sup>2)"
+definition %important "L2_set f A = sqrt (\<Sum>i\<in>A. (f i)\<^sup>2)"
 
 lemma L2_set_cong:
   "\<lbrakk>A = B; \<And>x. x \<in> B \<Longrightarrow> f x = g x\<rbrakk> \<Longrightarrow> L2_set f A = L2_set g B"
@@ -73,9 +73,9 @@
   unfolding L2_set_def
   by (simp add: sum_nonneg sum_nonneg_eq_0_iff)
 
-lemma L2_set_triangle_ineq:
-  shows "L2_set (\<lambda>i. f i + g i) A \<le> L2_set f A + L2_set g A"
-proof (cases "finite A")
+lemma %important L2_set_triangle_ineq:
+  "L2_set (\<lambda>i. f i + g i) A \<le> L2_set f A + L2_set g A"
+proof %unimportant (cases "finite A")
   case False
   thus ?thesis by simp
 next