src/HOL/Probability/Sigma_Algebra.thy
changeset 61952 546958347e05
parent 61847 9e38cde3d672
child 62083 7582b39f51ed
--- a/src/HOL/Probability/Sigma_Algebra.thy	Mon Dec 28 16:34:26 2015 +0100
+++ b/src/HOL/Probability/Sigma_Algebra.thy	Mon Dec 28 17:43:30 2015 +0100
@@ -75,7 +75,7 @@
   assumes Un [intro]: "\<And>a b. a \<in> M \<Longrightarrow> b \<in> M \<Longrightarrow> a \<union> b \<in> M"
 
 lemma (in ring_of_sets) finite_Union [intro]:
-  "finite X \<Longrightarrow> X \<subseteq> M \<Longrightarrow> Union X \<in> M"
+  "finite X \<Longrightarrow> X \<subseteq> M \<Longrightarrow> \<Union>X \<in> M"
   by (induct set: finite) (auto simp add: Un)
 
 lemma (in ring_of_sets) finite_UN[intro]:
@@ -261,7 +261,7 @@
 qed
 
 lemma (in sigma_algebra) countable_Union [intro]:
-  assumes "countable X" "X \<subseteq> M" shows "Union X \<in> M"
+  assumes "countable X" "X \<subseteq> M" shows "\<Union>X \<in> M"
 proof cases
   assume "X \<noteq> {}"
   hence "\<Union>X = (\<Union>n. from_nat_into X n)"