diff -r ce36bed06dee -r b5163b2132c5 src/HOL/Analysis/Function_Topology.thy --- a/src/HOL/Analysis/Function_Topology.thy Tue Jan 22 21:16:48 2019 +0000 +++ b/src/HOL/Analysis/Function_Topology.thy Tue Jan 22 22:57:16 2019 +0000 @@ -7,7 +7,7 @@ begin -section%important \Product Topology\ +section \Product Topology\ (* FIX see comments by the author *) text \We want to define the product topology. @@ -63,7 +63,7 @@ subsection \Topology without type classes\ -subsubsection \The topology generated by some (open) subsets\ +subsubsection%important \The topology generated by some (open) subsets\ text \In the definition below of a generated topology, the \Empty\ case is not necessary, as it follows from \UN\ taking for \K\ the empty set. However, it is convenient to have, @@ -257,7 +257,7 @@ qed qed -subsubsection \Continuity\ +subsubsection%important \Continuity\ text \We will need to deal with continuous maps in terms of topologies and not in terms of type classes, as defined below.\ @@ -335,7 +335,7 @@ using assms unfolding continuous_on_topo_def by auto -subsubsection \Pullback topology\ +subsubsection%important \Pullback topology\ text \Pulling back a topology by map gives again a topology. \subtopology\ is a special case of this notion, pulling back by the identity. We introduce the general notion as @@ -808,7 +808,7 @@ qed -subsubsection \Powers of a single topological space as a topological space, using type classes\ +subsubsection%important \Powers of a single topological space as a topological space, using type classes\ instantiation "fun" :: (type, topological_space) topological_space begin @@ -884,7 +884,7 @@ "continuous_on UNIV f \ (\i. continuous_on UNIV (\x. f x i))" by (auto intro: continuous_on_product_then_coordinatewise) -subsubsection \Topological countability for product spaces\ +subsubsection%important \Topological countability for product spaces\ text \The next two lemmas are useful to prove first or second countability of product spaces, but they have more to do with countability and could