doc-src/TutorialI/Documents/Documents.thy
changeset 28838 d5db6dfcb34a
parent 28504 7ad7d7d6df47
child 28914 f993cbffc42a
equal deleted inserted replaced
28837:c6b17889237a 28838:d5db6dfcb34a
   105   user-interface of Proof~General + X-Symbol and the Isabelle document
   105   user-interface of Proof~General + X-Symbol and the Isabelle document
   106   processor (see \S\ref{sec:document-preparation}) display the
   106   processor (see \S\ref{sec:document-preparation}) display the
   107   \verb,\,\verb,<forall>, symbol as~@{text \<forall>}.
   107   \verb,\,\verb,<forall>, symbol as~@{text \<forall>}.
   108 
   108 
   109   A list of standard Isabelle symbols is given in
   109   A list of standard Isabelle symbols is given in
   110   \cite[appendix~A]{isabelle-sys}.  You may introduce your own
   110   \cite{isabelle-isar-ref}.  You may introduce your own
   111   interpretation of further symbols by configuring the appropriate
   111   interpretation of further symbols by configuring the appropriate
   112   front-end tool accordingly, e.g.\ by defining certain {\LaTeX}
   112   front-end tool accordingly, e.g.\ by defining certain {\LaTeX}
   113   macros (see also \S\ref{sec:doc-prep-symbols}).  There are also a
   113   macros (see also \S\ref{sec:doc-prep-symbols}).  There are also a
   114   few predefined control symbols, such as \verb,\,\verb,<^sub>, and
   114   few predefined control symbols, such as \verb,\,\verb,<^sub>, and
   115   \verb,\,\verb,<^sup>, for sub- and superscript of the subsequent
   115   \verb,\,\verb,<^sup>, for sub- and superscript of the subsequent
   664   As has been pointed out before (\S\ref{sec:syntax-symbols}),
   664   As has been pointed out before (\S\ref{sec:syntax-symbols}),
   665   Isabelle symbols are the smallest syntactic entities --- a
   665   Isabelle symbols are the smallest syntactic entities --- a
   666   straightforward generalization of ASCII characters.  While Isabelle
   666   straightforward generalization of ASCII characters.  While Isabelle
   667   does not impose any interpretation of the infinite collection of
   667   does not impose any interpretation of the infinite collection of
   668   named symbols, {\LaTeX} documents use canonical glyphs for certain
   668   named symbols, {\LaTeX} documents use canonical glyphs for certain
   669   standard symbols \cite[appendix~A]{isabelle-sys}.
   669   standard symbols \cite{isabelle-isar-ref}.
   670 
   670 
   671   The {\LaTeX} code produced from Isabelle text follows a simple
   671   The {\LaTeX} code produced from Isabelle text follows a simple
   672   scheme.  You can tune the final appearance by redefining certain
   672   scheme.  You can tune the final appearance by redefining certain
   673   macros, say in \texttt{root.tex} of the document.
   673   macros, say in \texttt{root.tex} of the document.
   674 
   674