# HG changeset patch # User traytel # Date 1573071823 -3600 # Node ID 98ac9a4323a2faa3944f71d7aaea73124fe9c3e9 # Parent c9c1a64eeb6912591422beb9b9b679a85fafaefd# Parent d628bbdce79a1978e13155fd78f1cfeebb11c163 merged diff -r c9c1a64eeb69 -r 98ac9a4323a2 src/HOL/Analysis/Elementary_Topology.thy --- a/src/HOL/Analysis/Elementary_Topology.thy Wed Nov 06 16:57:51 2019 +0100 +++ b/src/HOL/Analysis/Elementary_Topology.thy Wed Nov 06 21:23:43 2019 +0100 @@ -16,11 +16,6 @@ section \Elementary Topology\ -subsection \TODO: move?\ - -lemma open_subopen: "open S \ (\x\S. \T. open T \ x \ T \ T \ S)" - using openI by auto - subsubsection\<^marker>\tag unimportant\ \Affine transformations of intervals\ @@ -49,7 +44,6 @@ by (simp add: field_simps) - subsection \Topological Basis\ context topological_space diff -r c9c1a64eeb69 -r 98ac9a4323a2 src/HOL/Topological_Spaces.thy --- a/src/HOL/Topological_Spaces.thy Wed Nov 06 16:57:51 2019 +0100 +++ b/src/HOL/Topological_Spaces.thy Wed Nov 06 21:23:43 2019 +0100 @@ -49,6 +49,9 @@ ultimately show "open S" by simp qed +lemma open_subopen: "open S \ (\x\S. \T. open T \ x \ T \ T \ S)" +by (auto intro: openI) + lemma closed_empty [continuous_intros, intro, simp]: "closed {}" unfolding closed_def by simp