--- a/src/HOL/Probability/Giry_Monad.thy Sun Dec 30 10:34:56 2018 +0000
+++ b/src/HOL/Probability/Giry_Monad.thy Sun Dec 30 10:34:56 2018 +0000
@@ -1763,7 +1763,7 @@
qed
qed
-lemma bind_cong_strong: "M = N \<Longrightarrow> (\<And>x. x\<in>space M =simp=> f x = g x) \<Longrightarrow> bind M f = bind N g"
+lemma bind_cong_simp: "M = N \<Longrightarrow> (\<And>x. x\<in>space M =simp=> f x = g x) \<Longrightarrow> bind M f = bind N g"
by (auto simp: simp_implies_def intro!: bind_cong)
lemma sets_bind_measurable: