src/HOL/Probability/Finite_Product_Measure.thy
changeset 61166 5976fe402824
parent 60580 7e741e22d7fc
child 61169 4de9ff3ea29a
--- a/src/HOL/Probability/Finite_Product_Measure.thy	Sun Sep 13 16:50:12 2015 +0200
+++ b/src/HOL/Probability/Finite_Product_Measure.thy	Sun Sep 13 20:20:16 2015 +0200
@@ -193,7 +193,7 @@
   assumes "I = J" "\<And>x. x \<in> I \<Longrightarrow> M x = N x"
   shows "PiM I M = PiM J N"
   unfolding PiM_def
-proof (rule extend_measure_cong, goals)
+proof (rule extend_measure_cong, goal_cases)
   case 1
   show ?case using assms
     by (subst assms(1), intro PiE_cong[of J "\<lambda>i. space (M i)" "\<lambda>i. space (N i)"]) simp_all