# HG changeset patch # User paulson # Date 1531298829 -3600 # Node ID 2fae3e01a2ecb7d3c504ca5290f56f1450cfcf07 # Parent ffc3fd6c74989d79ebc1ca851a3076f71f0e58b0 patched a continuity proof diff -r ffc3fd6c7498 -r 2fae3e01a2ec src/HOL/Probability/Sinc_Integral.thy --- a/src/HOL/Probability/Sinc_Integral.thy Wed Jul 11 09:14:21 2018 +0100 +++ b/src/HOL/Probability/Sinc_Integral.thy Wed Jul 11 09:47:09 2018 +0100 @@ -80,13 +80,15 @@ using cos_gt_zero_pi[of x] by (subst tan_sec) (auto intro!: DERIV_tan simp: power_inverse) have 2: "- (pi / 2) < x \ x * 2 < pi \ isCont (\x. 1 + (tan x)\<^sup>2) x" for x using cos_gt_zero_pi[of x] by auto + have 3: "\- (pi / 2) < x; x * 2 < pi\ \ isCont (\x. inverse (1 + x\<^sup>2)) (tan x)" for x + by (rule continuous_intros | simp add: add_nonneg_eq_0_iff)+ show "LBINT x=-\..\. inverse (1 + x^2) = pi" by (subst interval_integral_substitution_nonneg[of "-pi/2" "pi/2" tan "\x. 1 + (tan x)^2"]) - (auto intro: derivative_eq_intros 1 2 filterlim_tan_at_right + (auto intro: derivative_eq_intros 1 2 3 filterlim_tan_at_right simp add: ereal_tendsto_simps filterlim_tan_at_left add_nonneg_eq_0_iff set_integrable_def) show "set_integrable lborel (einterval (-\) \) (\x. inverse (1 + x^2))" by (subst interval_integral_substitution_nonneg[of "-pi/2" "pi/2" tan "\x. 1 + (tan x)^2"]) - (auto intro: derivative_eq_intros 1 2 filterlim_tan_at_right + (auto intro: derivative_eq_intros 1 2 3 filterlim_tan_at_right simp add: ereal_tendsto_simps filterlim_tan_at_left add_nonneg_eq_0_iff set_integrable_def) qed @@ -395,11 +397,7 @@ } note aux2 = this show ?thesis using assms unfolding Si_def interval_lebesgue_integral_def set_lebesgue_integral_def sgn_real_def einterval_eq zero_ereal_def - apply auto - apply (erule aux1) - apply (rule aux2) - apply auto - done + by (auto simp: aux1 aux2) qed end