src/HOL/Analysis/Topology_Euclidean_Space.thy
changeset 69260 0a9688695a1b
parent 69144 f13b82281715
child 69286 e4d5a07fecb6
--- a/src/HOL/Analysis/Topology_Euclidean_Space.thy	Wed Nov 07 23:03:45 2018 +0100
+++ b/src/HOL/Analysis/Topology_Euclidean_Space.thy	Thu Nov 08 09:11:52 2018 +0100
@@ -4189,7 +4189,7 @@
 next
   fix A
   assume A: "\<forall>a\<in>A. closed a" "\<forall>B\<subseteq>A. finite B \<longrightarrow> U \<inter> \<Inter>B \<noteq> {}" "U \<inter> \<Inter>A = {}"
-  define F where "F = (INF a:insert U A. principal a)"
+  define F where "F = (INF a\<in>insert U A. principal a)"
   have "F \<noteq> bot"
     unfolding F_def
   proof (rule INF_filter_not_bot)
@@ -4197,7 +4197,7 @@
     assume X: "X \<subseteq> insert U A" "finite X"
     with A(2)[THEN spec, of "X - {U}"] have "U \<inter> \<Inter>(X - {U}) \<noteq> {}"
       by auto
-    with X show "(INF a:X. principal a) \<noteq> bot"
+    with X show "(INF a\<in>X. principal a) \<noteq> bot"
       by (auto simp: INF_principal_finite principal_eq_bot_iff)
   qed
   moreover