diff -r cb34f5f49a08 -r ec32cdaab97b src/HOL/Probability/Giry_Monad.thy --- a/src/HOL/Probability/Giry_Monad.thy Tue Dec 19 14:51:27 2017 +0100 +++ b/src/HOL/Probability/Giry_Monad.thy Tue Dec 19 13:58:12 2017 +0100 @@ -1746,19 +1746,19 @@ shows "bind M f = bind N g" proof cases assume "space N = {}" then show ?thesis - using `M = N` by (simp add: bind_empty) + using \M = N\ by (simp add: bind_empty) next assume "space N \ {}" - show ?thesis unfolding `M = N` + show ?thesis unfolding \M = N\ proof (rule measure_eqI) have *: "sets (N \ f) = sets B" - using sets_bind[OF sets_kernel[OF f] `space N \ {}`] by simp + using sets_bind[OF sets_kernel[OF f] \space N \ {}\] by simp then show "sets (N \ f) = sets (N \ g)" - using sets_bind[OF sets_kernel[OF g] `space N \ {}`] by auto + using sets_bind[OF sets_kernel[OF g] \space N \ {}\] by auto fix A assume "A \ sets (N \ f)" then have "A \ sets B" unfolding * . - with ae f g `space N \ {}` show "emeasure (N \ f) A = emeasure (N \ g) A" + with ae f g \space N \ {}\ show "emeasure (N \ f) A = emeasure (N \ g) A" by (subst (1 2) emeasure_bind[where N=B]) (auto intro!: nn_integral_cong_AE) qed qed