src/HOL/Analysis/Function_Topology.thy
changeset 69597 ff784d5a5bfb
parent 69566 c41954ee87cf
child 69677 a06b204527e6
--- a/src/HOL/Analysis/Function_Topology.thy	Sat Jan 05 17:00:43 2019 +0100
+++ b/src/HOL/Analysis/Function_Topology.thy	Sat Jan 05 17:24:33 2019 +0100
@@ -17,7 +17,7 @@
 to each factor is continuous.
 
 To form a product of objects in Isabelle/HOL, all these objects should be subsets of a common type
-'a. The product is then @{term "Pi\<^sub>E I X"}, the set of elements from \<open>'i\<close> to \<open>'a\<close> such that the \<open>i\<close>-th
+'a. The product is then \<^term>\<open>Pi\<^sub>E I X\<close>, the set of elements from \<open>'i\<close> to \<open>'a\<close> such that the \<open>i\<close>-th
 coordinate belongs to \<open>X i\<close> for all \<open>i \<in> I\<close>.
 
 Hence, to form a product of topological spaces, all these spaces should be subsets of a common type.