diff -r 9bb2856cc845 -r 0556204bc230 src/HOL/Probability/Distributions.thy --- a/src/HOL/Probability/Distributions.thy Thu Apr 03 17:16:02 2014 +0200 +++ b/src/HOL/Probability/Distributions.thy Thu Apr 03 17:56:08 2014 +0200 @@ -52,7 +52,7 @@ let ?F = "\x. - exp (- x * l)" have deriv: "\x. DERIV ?F x :> ?f x" "\x. 0 \ l * exp (- x * l)" - by (auto intro!: DERIV_intros simp: zero_le_mult_iff) + by (auto intro!: derivative_eq_intros simp: zero_le_mult_iff) have "emeasure ?D (space ?D) = (\\<^sup>+ x. ereal (?f x) * indicator {0..} x \lborel)" by (auto simp: emeasure_density exponential_density_def @@ -178,12 +178,12 @@ proof (rule integral_FTC_atLeastAtMost) fix x assume "0 \ x" "x \ b" show "DERIV (\x. x * exp (-x)) x :> exp (-x) - x * exp (-x)" - by (auto intro!: DERIV_intros) + by (auto intro!: derivative_eq_intros) show "isCont (\x. exp (- x) - x * exp (- x)) x " by (intro continuous_intros) qed fact also have "(\x. (exp (-x)) * indicator {0 .. b} x \lborel) = - exp (- b) - - exp (- 0)" - by (rule integral_FTC_atLeastAtMost) (auto intro!: DERIV_intros) + by (rule integral_FTC_atLeastAtMost) (auto intro!: derivative_eq_intros) finally show "1 - (inverse (exp b) + b / exp b) = integral\<^sup>L lborel (?f b)" by (auto simp: field_simps exp_minus inverse_eq_divide) qed @@ -374,7 +374,7 @@ fix x show "DERIV (\x. x\<^sup>2 / (2 * measure lborel {a..b})) x :> x / measure lborel {a..b}" using uniform_distributed_params[OF D] - by (auto intro!: DERIV_intros) + by (auto intro!: derivative_eq_intros) show "isCont (\x. x / Sigma_Algebra.measure lborel {a..b}) x" using uniform_distributed_params[OF D] by (auto intro!: isCont_divide)