src/HOL/Topological_Spaces.thy
changeset 67231 754952c12293
parent 67226 ec32cdaab97b
child 67453 afefc45ed4e9
--- 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]: