src/HOL/Topological_Spaces.thy
changeset 63170 eae6549dbea2
parent 63092 a949b2a5f51d
child 63171 a0088f1c049d
--- a/src/HOL/Topological_Spaces.thy	Fri May 27 20:13:06 2016 +0200
+++ b/src/HOL/Topological_Spaces.thy	Fri May 27 20:23:55 2016 +0200
@@ -75,22 +75,22 @@
   using closed_Union [of "B ` A"] by simp
 
 lemma open_closed: "open S \<longleftrightarrow> closed (- S)"
-  unfolding closed_def by simp
+  by (simp add: closed_def)
 
 lemma closed_open: "closed S \<longleftrightarrow> open (- S)"
-  unfolding closed_def by simp
+  by (rule closed_def)
 
 lemma open_Diff [continuous_intros, intro]: "open S \<Longrightarrow> closed T \<Longrightarrow> open (S - T)"
-  unfolding closed_open Diff_eq by (rule open_Int)
+  by (simp add: closed_open Diff_eq open_Int)
 
 lemma closed_Diff [continuous_intros, intro]: "closed S \<Longrightarrow> open T \<Longrightarrow> closed (S - T)"
-  unfolding open_closed Diff_eq by (rule closed_Int)
+  by (simp add: open_closed Diff_eq closed_Int)
 
 lemma open_Compl [continuous_intros, intro]: "closed S \<Longrightarrow> open (- S)"
-  unfolding closed_open .
+  by (simp add: closed_open)
 
 lemma closed_Compl [continuous_intros, intro]: "open S \<Longrightarrow> closed (- S)"
-  unfolding open_closed .
+  by (simp add: open_closed)
 
 lemma open_Collect_neg: "closed {x. P x} \<Longrightarrow> open {x. \<not> P x}"
   unfolding Collect_neg_eq by (rule open_Compl)