src/HOL/Probability/Distributions.thy
changeset 53077 a1b3784f8129
parent 53015 a1119cf551e8
child 56371 fb9ae0727548
equal deleted inserted replaced
53076:47c9aff07725 53077:a1b3784f8129
   370     (\<integral> x. (x / measure lborel {a .. b}) * indicator {a .. b} x \<partial>lborel)"
   370     (\<integral> x. (x / measure lborel {a .. b}) * indicator {a .. b} x \<partial>lborel)"
   371     by (intro integral_cong) auto
   371     by (intro integral_cong) auto
   372   also have "(\<integral> x. (x / measure lborel {a .. b}) * indicator {a .. b} x \<partial>lborel) = (a + b) / 2"
   372   also have "(\<integral> x. (x / measure lborel {a .. b}) * indicator {a .. b} x \<partial>lborel) = (a + b) / 2"
   373   proof (subst integral_FTC_atLeastAtMost)
   373   proof (subst integral_FTC_atLeastAtMost)
   374     fix x
   374     fix x
   375     show "DERIV (\<lambda>x. x ^ 2 / (2 * measure lborel {a..b})) x :> x / measure lborel {a..b}"
   375     show "DERIV (\<lambda>x. x\<^sup>2 / (2 * measure lborel {a..b})) x :> x / measure lborel {a..b}"
   376       using uniform_distributed_params[OF D]
   376       using uniform_distributed_params[OF D]
   377       by (auto intro!: DERIV_intros)
   377       by (auto intro!: DERIV_intros)
   378     show "isCont (\<lambda>x. x / Sigma_Algebra.measure lborel {a..b}) x"
   378     show "isCont (\<lambda>x. x / Sigma_Algebra.measure lborel {a..b}) x"
   379       using uniform_distributed_params[OF D]
   379       using uniform_distributed_params[OF D]
   380       by (auto intro!: isCont_divide)
   380       by (auto intro!: isCont_divide)