remove needless fact
authorblanchet
Wed, 06 Oct 2010 17:38:06 +0200
changeset 39960 03174b2d075c
parent 39959 12eb8fe15b00
child 39961 415556559fad
remove needless fact
src/HOL/Probability/Sigma_Algebra.thy
--- a/src/HOL/Probability/Sigma_Algebra.thy	Wed Oct 06 12:01:55 2010 +0200
+++ b/src/HOL/Probability/Sigma_Algebra.thy	Wed Oct 06 17:38:06 2010 +0200
@@ -242,7 +242,7 @@
 lemma sigma_sets_Un:
   "a \<in> sigma_sets sp A \<Longrightarrow> b \<in> sigma_sets sp A \<Longrightarrow> a \<union> b \<in> sigma_sets sp A"
 apply (simp add: Un_range_binary range_binary_eq)
-apply (rule Union, simp add: binary_def COMBK_def fun_upd_apply)
+apply (rule Union, simp add: binary_def fun_upd_apply)
 done
 
 lemma sigma_sets_Inter: