src/HOL/Analysis/Henstock_Kurzweil_Integration.thy
changeset 63938 f6ce08859d4c
parent 63928 d81fb5b46a5c
child 63940 0d82c4c94014
--- a/src/HOL/Analysis/Henstock_Kurzweil_Integration.thy	Wed Sep 21 16:59:51 2016 +0100
+++ b/src/HOL/Analysis/Henstock_Kurzweil_Integration.thy	Thu Sep 22 15:44:47 2016 +0100
@@ -2902,7 +2902,7 @@
   fixes f :: "'n::euclidean_space \<Rightarrow> 'm::euclidean_space"
   assumes "f integrable_on s"
   shows "integral s (\<lambda>x. f x \<bullet> k) = integral s f \<bullet> k"
-  unfolding integral_linear[OF assms(1) bounded_linear_component,unfolded o_def] ..
+  unfolding integral_linear[OF assms(1) bounded_linear_inner_left,unfolded o_def] ..
 
 lemma has_integral_setsum:
   assumes "finite t"
@@ -3090,7 +3090,7 @@
   shows "(f has_integral y) A \<longleftrightarrow> (\<forall>b\<in>Basis. ((\<lambda>x. f x \<bullet> b) has_integral (y \<bullet> b)) A)"
 proof safe
   fix b :: 'b assume "(f has_integral y) A"
-  from has_integral_linear[OF this(1) bounded_linear_component, of b]
+  from has_integral_linear[OF this(1) bounded_linear_inner_left, of b]
     show "((\<lambda>x. f x \<bullet> b) has_integral (y \<bullet> b)) A" by (simp add: o_def)
 next
   assume "(\<forall>b\<in>Basis. ((\<lambda>x. f x \<bullet> b) has_integral (y \<bullet> b)) A)"
@@ -3148,7 +3148,7 @@
 
 lemma integrable_component:
   "f integrable_on A \<Longrightarrow> (\<lambda>x. f x \<bullet> (y :: 'b :: euclidean_space)) integrable_on A"
-  by (drule integrable_linear[OF _ bounded_linear_component[of y]]) (simp add: o_def)
+  by (drule integrable_linear[OF _ bounded_linear_inner_left[of y]]) (simp add: o_def)