src/HOL/Probability/Sigma_Algebra.thy
changeset 50252 4aa34bd43228
parent 50245 dea9363887a6
child 50283 e79a8341dd6b
equal deleted inserted replaced
50251:227477f17c26 50252:4aa34bd43228
   385   using algebra.is_sigma_algebra[OF algebra_single_set[OF `X \<subseteq> S`]] by simp
   385   using algebra.is_sigma_algebra[OF algebra_single_set[OF `X \<subseteq> S`]] by simp
   386 
   386 
   387 subsection {* Binary Unions *}
   387 subsection {* Binary Unions *}
   388 
   388 
   389 definition binary :: "'a \<Rightarrow> 'a \<Rightarrow> nat \<Rightarrow> 'a"
   389 definition binary :: "'a \<Rightarrow> 'a \<Rightarrow> nat \<Rightarrow> 'a"
   390   where "binary a b =  (\<lambda>\<^isup>x. b)(0 := a)"
   390   where "binary a b =  (\<lambda>x. b)(0 := a)"
   391 
   391 
   392 lemma range_binary_eq: "range(binary a b) = {a,b}"
   392 lemma range_binary_eq: "range(binary a b) = {a,b}"
   393   by (auto simp add: binary_def)
   393   by (auto simp add: binary_def)
   394 
   394 
   395 lemma Un_range_binary: "a \<union> b = (\<Union>i::nat. binary a b i)"
   395 lemma Un_range_binary: "a \<union> b = (\<Union>i::nat. binary a b i)"
  2115 qed
  2115 qed
  2116 
  2116 
  2117 subsection {* A Two-Element Series *}
  2117 subsection {* A Two-Element Series *}
  2118 
  2118 
  2119 definition binaryset :: "'a set \<Rightarrow> 'a set \<Rightarrow> nat \<Rightarrow> 'a set "
  2119 definition binaryset :: "'a set \<Rightarrow> 'a set \<Rightarrow> nat \<Rightarrow> 'a set "
  2120   where "binaryset A B = (\<lambda>\<^isup>x. {})(0 := A, Suc 0 := B)"
  2120   where "binaryset A B = (\<lambda>x. {})(0 := A, Suc 0 := B)"
  2121 
  2121 
  2122 lemma range_binaryset_eq: "range(binaryset A B) = {A,B,{}}"
  2122 lemma range_binaryset_eq: "range(binaryset A B) = {A,B,{}}"
  2123   apply (simp add: binaryset_def)
  2123   apply (simp add: binaryset_def)
  2124   apply (rule set_eqI)
  2124   apply (rule set_eqI)
  2125   apply (auto simp add: image_iff)
  2125   apply (auto simp add: image_iff)