src/HOL/Analysis/Change_Of_Vars.thy
changeset 75462 7448423e5dba
parent 73933 fa92bc604c59
child 78475 a5f6d2fc1b1f
equal deleted inserted replaced
75461:4c3bc0d2568f 75462:7448423e5dba
  3386 proof -
  3386 proof -
  3387   have "(\<lambda>x. \<bar>g' x\<bar> *\<^sub>R vec (f(g x)) :: real ^ 1) absolutely_integrable_on S \<and>
  3387   have "(\<lambda>x. \<bar>g' x\<bar> *\<^sub>R vec (f(g x)) :: real ^ 1) absolutely_integrable_on S \<and>
  3388            integral S (\<lambda>x. \<bar>g' x\<bar> *\<^sub>R vec (f(g x))) = (vec b :: real ^ 1)
  3388            integral S (\<lambda>x. \<bar>g' x\<bar> *\<^sub>R vec (f(g x))) = (vec b :: real ^ 1)
  3389          \<longleftrightarrow> (\<lambda>x. vec (f x) :: real ^ 1) absolutely_integrable_on (g ` S) \<and>
  3389          \<longleftrightarrow> (\<lambda>x. vec (f x) :: real ^ 1) absolutely_integrable_on (g ` S) \<and>
  3390            integral (g ` S) (\<lambda>x. vec (f x)) = (vec b :: real ^ 1)"
  3390            integral (g ` S) (\<lambda>x. vec (f x)) = (vec b :: real ^ 1)"
  3391     using assms unfolding has_field_derivative_iff_has_vector_derivative
  3391     using assms unfolding has_real_derivative_iff_has_vector_derivative
  3392     by (intro has_absolute_integral_change_of_variables_1 assms) auto
  3392     by (intro has_absolute_integral_change_of_variables_1 assms) auto
  3393   thus ?thesis
  3393   thus ?thesis
  3394     by (simp add: absolutely_integrable_on_1_iff integral_on_1_eq)
  3394     by (simp add: absolutely_integrable_on_1_iff integral_on_1_eq)
  3395 qed
  3395 qed
  3396 
  3396