amending 689997a8a582
authorimmler
Thu, 17 Jan 2019 17:50:01 -0500
changeset 69684 94284d4dab98
parent 69683 8b3458ca0762
child 69686 aeceb14f387a
amending 689997a8a582
src/HOL/Analysis/Finite_Cartesian_Product.thy
--- a/src/HOL/Analysis/Finite_Cartesian_Product.thy	Thu Jan 17 16:38:00 2019 -0500
+++ b/src/HOL/Analysis/Finite_Cartesian_Product.thy	Thu Jan 17 17:50:01 2019 -0500
@@ -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)