src/HOL/Analysis/Finite_Cartesian_Product.thy
changeset 69668 14a8cac10eac
parent 69663 41ff40bf1530
child 69669 de2f0a24b0f0
--- a/src/HOL/Analysis/Finite_Cartesian_Product.thy	Wed Jan 16 15:53:12 2019 +0100
+++ b/src/HOL/Analysis/Finite_Cartesian_Product.thy	Wed Jan 16 16:18:53 2019 +0100
@@ -626,7 +626,7 @@
 lemma%unimportant norm_le_l1_cart: "norm x \<le> sum(\<lambda>i. \<bar>x$i\<bar>) UNIV"
   by (simp add: norm_vec_def L2_set_le_sum)
 
-lemma%unimportant bounded_linear_vec_nth: "bounded_linear (\<lambda>x. x $ i)"
+lemma%unimportant bounded_linear_vec_nth[intro]: "bounded_linear (\<lambda>x. x $ i)"
 apply standard
 apply (rule vector_add_component)
 apply (rule vector_scaleR_component)