# HG changeset patch # User hoelzl # Date 1283450236 -7200 # Node ID 21e9bd6cf0a8bf2b9d0c70a997d9fad6d9b8ed47 # Parent 943c7b348524f0e10916a7780d05cdc5c87c37cf Corrected definition and hence removed sorry. diff -r 943c7b348524 -r 21e9bd6cf0a8 src/HOL/Probability/Product_Measure.thy --- a/src/HOL/Probability/Product_Measure.thy Thu Sep 02 19:51:53 2010 +0200 +++ b/src/HOL/Probability/Product_Measure.thy Thu Sep 02 19:57:16 2010 +0200 @@ -5,7 +5,7 @@ definition "dynkin M \ space M \ sets M \ (\ A \ sets M. A \ space M) \ - (\ a \ sets M. \ b \ sets M. b - a \ sets M) \ + (\ a \ sets M. \ b \ sets M. a \ b \ b - a \ sets M) \ (\A. disjoint_family A \ range A \ sets M \ (\i::nat. A i) \ sets M)" lemma dynkinI: @@ -14,7 +14,7 @@ assumes "\ a. (\ i j :: nat. i \ j \ a i \ a j = {}) \ (\ i :: nat. a i \ sets M) \ UNION UNIV a \ sets M" shows "dynkin M" -using assms unfolding dynkin_def sorry +using assms by (auto simp: dynkin_def disjoint_family_on_def image_subset_iff) lemma dynkin_subset: assumes "dynkin M" @@ -41,7 +41,7 @@ assumes "\ i j :: nat. i \ j \ a i \ a j = {}" assumes "\ i :: nat. a i \ sets M" shows "UNION UNIV a \ sets M" -using assms unfolding dynkin_def sorry +using assms by (auto simp: dynkin_def disjoint_family_on_def image_subset_iff) definition "Int_stable M \ (\ a \ sets M. \ b \ sets M. a \ b \ sets M)"