tuned op's
authornipkow
Wed, 20 Dec 2017 21:06:08 +0100
changeset 67231 754952c12293
parent 67230 b2800da9eb8a
child 67232 a00f5a71e672
tuned op's
src/HOL/Topological_Spaces.thy
--- a/src/HOL/Topological_Spaces.thy	Wed Dec 20 19:17:37 2017 +0100
+++ b/src/HOL/Topological_Spaces.thy	Wed Dec 20 21:06:08 2017 +0100
@@ -2158,11 +2158,11 @@
 
 lemma compactE_image:
   assumes "compact S"
-    and op: "\<And>T. T \<in> C \<Longrightarrow> open (f T)"
+    and opn: "\<And>T. T \<in> C \<Longrightarrow> open (f T)"
     and S: "S \<subseteq> (\<Union>c\<in>C. f c)"
   obtains C' where "C' \<subseteq> C" and "finite C'" and "S \<subseteq> (\<Union>c\<in>C'. f c)"
     apply (rule compactE[OF \<open>compact S\<close> S])
-    using op apply force
+    using opn apply force
     by (metis finite_subset_image)
 
 lemma compact_Int_closed [intro]: