src/HOL/Probability/Sinc_Integral.thy
changeset 62390 842917225d56
parent 62087 44841d07ef1d
child 62975 1d066f6ab25d
equal deleted inserted replaced
62380:29800666e526 62390:842917225d56
   194     by auto
   194     by auto
   195   ultimately show ?thesis
   195   ultimately show ?thesis
   196     using interval_integral_FTC2[of "min 0 (x - 1)" 0 "max 0 (x + 1)" sinc x]
   196     using interval_integral_FTC2[of "min 0 (x - 1)" 0 "max 0 (x + 1)" sinc x]
   197     by (auto simp: continuous_at_imp_continuous_on isCont_sinc Si_alt_def[abs_def] zero_ereal_def
   197     by (auto simp: continuous_at_imp_continuous_on isCont_sinc Si_alt_def[abs_def] zero_ereal_def
   198                    has_field_derivative_iff_has_vector_derivative
   198                    has_field_derivative_iff_has_vector_derivative
   199              split del: split_if)
   199              split del: if_split)
   200 qed
   200 qed
   201 
   201 
   202 lemma isCont_Si: "isCont Si x"
   202 lemma isCont_Si: "isCont Si x"
   203   using DERIV_Si by (rule DERIV_isCont)
   203   using DERIV_Si by (rule DERIV_isCont)
   204 
   204 
   387     finally have "(LBINT t=ereal 0..T. sin (t * -\<theta>) / t) = (LBINT t=ereal 0..T * -\<theta>. sin t / t)"
   387     finally have "(LBINT t=ereal 0..T. sin (t * -\<theta>) / t) = (LBINT t=ereal 0..T * -\<theta>. sin t / t)"
   388       by simp
   388       by simp
   389     hence "LBINT x. indicator {0<..<T} x * sin (x * \<theta>) / x =
   389     hence "LBINT x. indicator {0<..<T} x * sin (x * \<theta>) / x =
   390        - (LBINT x. indicator {0<..<- (T * \<theta>)} x * sin x / x)"
   390        - (LBINT x. indicator {0<..<- (T * \<theta>)} x * sin x / x)"
   391       using assms `0 > \<theta>` unfolding interval_lebesgue_integral_def einterval_eq zero_ereal_def
   391       using assms `0 > \<theta>` unfolding interval_lebesgue_integral_def einterval_eq zero_ereal_def
   392         by (auto simp add: field_simps mult_le_0_iff split: split_if_asm)
   392         by (auto simp add: field_simps mult_le_0_iff split: if_split_asm)
   393   } note aux2 = this
   393   } note aux2 = this
   394   show ?thesis
   394   show ?thesis
   395     using assms unfolding Si_def interval_lebesgue_integral_def sgn_real_def einterval_eq zero_ereal_def
   395     using assms unfolding Si_def interval_lebesgue_integral_def sgn_real_def einterval_eq zero_ereal_def
   396     apply auto
   396     apply auto
   397     apply (erule aux1)
   397     apply (erule aux1)