avoid Isabelle symbols in URL;
authorwenzelm
Fri, 12 Apr 2019 22:52:00 +0200
changeset 70139 fd4960dfad2a
parent 70138 bd42cc1e10d0
child 70140 d13865c21e36
avoid Isabelle symbols in URL;
src/HOL/Analysis/Change_Of_Vars.thy
--- a/src/HOL/Analysis/Change_Of_Vars.thy	Fri Apr 12 22:24:57 2019 +0200
+++ b/src/HOL/Analysis/Change_Of_Vars.thy	Fri Apr 12 22:52:00 2019 +0200
@@ -423,7 +423,7 @@
 
 subsection\<open>\<open>F_sigma\<close> and \<open>G_delta\<close> sets.\<close>(*FIX ME mv *)
 
-\<comment> \<open>\<^url>\<open>https://en.wikipedia.org/wiki/F\<sigma>_set\<close>\<close>
+\<comment> \<open>\<^url>\<open>https://en.wikipedia.org/wiki/F-sigma_set\<close>\<close>
 inductive\<^marker>\<open>tag important\<close> fsigma :: "'a::topological_space set \<Rightarrow> bool" where
   "(\<And>n::nat. closed (F n)) \<Longrightarrow> fsigma (\<Union>(F ` UNIV))"