src/HOL/Probability/Product_PMF.thy
changeset 75455 91c16c5ad3e9
parent 73536 5131c388a9b0
child 77434 da41823d09a7
--- a/src/HOL/Probability/Product_PMF.thy	Wed May 11 10:42:24 2022 +0200
+++ b/src/HOL/Probability/Product_PMF.thy	Tue May 17 14:10:14 2022 +0100
@@ -354,7 +354,7 @@
           Pi_pmf A dflt' (\<lambda>x. g x \<bind> (\<lambda>x. return_pmf (f x)))"
     using assms by (simp add: map_pmf_def Pi_pmf_bind)
   also have "\<dots> = Pi_pmf A dflt g \<bind> (\<lambda>h. return_pmf (\<lambda>x. if x \<in> A then f (h x) else dflt'))"
-   by (subst Pi_pmf_bind[where d' = dflt]) (auto simp: )
+   by (subst Pi_pmf_bind[where d' = dflt]) auto
   also have "\<dots> = map_pmf (\<lambda>h. f \<circ> h) (Pi_pmf A dflt g)"
     unfolding map_pmf_def using set_Pi_pmf_subset'[of A dflt g]
     by (intro bind_pmf_cong refl arg_cong[of _ _ return_pmf])