diff -r 5bc338cee4a0 -r dd675800469d src/HOL/Probability/Probability_Mass_Function.thy --- a/src/HOL/Probability/Probability_Mass_Function.thy Wed Oct 09 23:00:52 2019 +0200 +++ b/src/HOL/Probability/Probability_Mass_Function.thy Wed Oct 09 14:51:54 2019 +0000 @@ -1785,7 +1785,7 @@ assumes "A \ {}" "finite A" "\x. x \ A \ finite (set_pmf (f x))" shows "measure_pmf.expectation (pmf_of_set A \ f) h = (\a\A. measure_pmf.expectation (f a) h /\<^sub>R real (card A))" - using assms by (subst pmf_expectation_bind[of A]) (auto simp: divide_simps) + using assms by (subst pmf_expectation_bind[of A]) (auto simp: field_split_simps) lemma map_pmf_of_set: assumes "finite A" "A \ {}" @@ -1995,7 +1995,7 @@ by (simp add: indicator_def) show "pmf (binomial_pmf (Suc n) p) k = pmf ?rhs k" by (cases k; cases "k > n") - (insert assms, auto simp: pmf_bind measure_pmf_single A divide_simps algebra_simps + (insert assms, auto simp: pmf_bind measure_pmf_single A field_split_simps algebra_simps not_less less_eq_Suc_le [symmetric] power_diff') qed