src/Doc/System/Misc.thy
changeset 57413 c14af83bd8db
parent 57330 d8a64a4cbfca
child 57414 fe1be2844fda
--- a/src/Doc/System/Misc.thy	Fri Jun 27 15:24:56 2014 +0200
+++ b/src/Doc/System/Misc.thy	Fri Jun 27 15:30:57 2014 +0200
@@ -472,26 +472,6 @@
   "();"} in ML will return to the Isar toplevel.  *}
 
 
-section {* Remove awkward symbol names from theory sources *}
-
-text {*
-  The @{tool_def unsymbolize} tool tunes Isabelle theory sources to
-  improve readability for plain ASCII output (e.g.\ in email
-  communication).  Most notably, @{tool unsymbolize} replaces awkward
-  arrow symbols such as @{verbatim "\\"}@{verbatim "<Longrightarrow>"}
-  by @{verbatim "==>"}.
-\begin{ttbox}
-Usage: isabelle unsymbolize [FILES|DIRS...]
-
-  Recursively find .thy/.ML files, removing unreadable symbol names.
-  Note: this is an ad-hoc script; there is no systematic way to replace
-  symbols independently of the inner syntax of a theory!
-
-  Renames old versions of FILES by appending "~~".
-\end{ttbox}
-*}
-
-
 section {* Output the version identifier of the Isabelle distribution *}
 
 text {*