doc-src/TutorialI/Documents/Documents.thy
changeset 28504 7ad7d7d6df47
parent 27027 63f0b638355c
child 28838 d5db6dfcb34a
equal deleted inserted replaced
28503:a30b7169fdd1 28504:7ad7d7d6df47
   345   image like \texttt{HOL}.  This results in an overall tree structure,
   345   image like \texttt{HOL}.  This results in an overall tree structure,
   346   which is reflected by the output location in the file system
   346   which is reflected by the output location in the file system
   347   (usually rooted at \verb,~/isabelle/browser_info,).
   347   (usually rooted at \verb,~/isabelle/browser_info,).
   348 
   348 
   349   \medskip The easiest way to manage Isabelle sessions is via
   349   \medskip The easiest way to manage Isabelle sessions is via
   350   \texttt{isatool mkdir} (generates an initial session source setup)
   350   \texttt{isabelle mkdir} (generates an initial session source setup)
   351   and \texttt{isatool make} (run sessions controlled by
   351   and \texttt{isabelle make} (run sessions controlled by
   352   \texttt{IsaMakefile}).  For example, a new session
   352   \texttt{IsaMakefile}).  For example, a new session
   353   \texttt{MySession} derived from \texttt{HOL} may be produced as
   353   \texttt{MySession} derived from \texttt{HOL} may be produced as
   354   follows:
   354   follows:
   355 
   355 
   356 \begin{verbatim}
   356 \begin{verbatim}
   357   isatool mkdir HOL MySession
   357   isabelle mkdir HOL MySession
   358   isatool make
   358   isabelle make
   359 \end{verbatim}
   359 \end{verbatim}
   360 
   360 
   361   The \texttt{isatool make} job also informs about the file-system
   361   The \texttt{isabelle make} job also informs about the file-system
   362   location of the ultimate results.  The above dry run should be able
   362   location of the ultimate results.  The above dry run should be able
   363   to produce some \texttt{document.pdf} (with dummy title, empty table
   363   to produce some \texttt{document.pdf} (with dummy title, empty table
   364   of contents etc.).  Any failure at this stage usually indicates
   364   of contents etc.).  Any failure at this stage usually indicates
   365   technical problems of the {\LaTeX} installation.
   365   technical problems of the {\LaTeX} installation.
   366 
   366 
   392   \item \texttt{IsaMakefile} holds appropriate dependencies and
   392   \item \texttt{IsaMakefile} holds appropriate dependencies and
   393   invocations of Isabelle tools to control the batch job.  In fact,
   393   invocations of Isabelle tools to control the batch job.  In fact,
   394   several sessions may be managed by the same \texttt{IsaMakefile}.
   394   several sessions may be managed by the same \texttt{IsaMakefile}.
   395   See the \emph{Isabelle System Manual} \cite{isabelle-sys} 
   395   See the \emph{Isabelle System Manual} \cite{isabelle-sys} 
   396   for further details, especially on
   396   for further details, especially on
   397   \texttt{isatool usedir} and \texttt{isatool make}.
   397   \texttt{isabelle usedir} and \texttt{isabelle make}.
   398 
   398 
   399   \end{itemize}
   399   \end{itemize}
   400 
   400 
   401   One may now start to populate the directory \texttt{MySession}, and
   401   One may now start to populate the directory \texttt{MySession}, and
   402   the file \texttt{MySession/ROOT.ML} accordingly.  The file
   402   the file \texttt{MySession/ROOT.ML} accordingly.  The file
   415 
   415 
   416   \medskip Any additional files for the {\LaTeX} stage go into the
   416   \medskip Any additional files for the {\LaTeX} stage go into the
   417   \texttt{MySession/document} directory as well.  In particular,
   417   \texttt{MySession/document} directory as well.  In particular,
   418   adding a file named \texttt{root.bib} causes an automatic run of
   418   adding a file named \texttt{root.bib} causes an automatic run of
   419   \texttt{bibtex} to process a bibliographic database; see also
   419   \texttt{bibtex} to process a bibliographic database; see also
   420   \texttt{isatool document} \cite{isabelle-sys}.
   420   \texttt{isabelle document} \cite{isabelle-sys}.
   421 
   421 
   422   \medskip Any failure of the document preparation phase in an
   422   \medskip Any failure of the document preparation phase in an
   423   Isabelle batch session leaves the generated sources in their target
   423   Isabelle batch session leaves the generated sources in their target
   424   location, identified by the accompanying error message.  This lets
   424   location, identified by the accompanying error message.  This lets
   425   you trace {\LaTeX} problems with the generated files at hand.
   425   you trace {\LaTeX} problems with the generated files at hand.
   751   same tag are joined into a single region.  The Isabelle document
   751   same tag are joined into a single region.  The Isabelle document
   752   preparation system allows the user to specify how to interpret a
   752   preparation system allows the user to specify how to interpret a
   753   tagged region, in order to keep, drop, or fold the corresponding
   753   tagged region, in order to keep, drop, or fold the corresponding
   754   parts of the document.  See the \emph{Isabelle System Manual}
   754   parts of the document.  See the \emph{Isabelle System Manual}
   755   \cite{isabelle-sys} for further details, especially on
   755   \cite{isabelle-sys} for further details, especially on
   756   \texttt{isatool usedir} and \texttt{isatool document}.
   756   \texttt{isabelle usedir} and \texttt{isabelle document}.
   757 
   757 
   758   Ignored material is specified by delimiting the original formal
   758   Ignored material is specified by delimiting the original formal
   759   source with special source comments
   759   source with special source comments
   760   \verb,(,\verb,*,\verb,<,\verb,*,\verb,), and
   760   \verb,(,\verb,*,\verb,<,\verb,*,\verb,), and
   761   \verb,(,\verb,*,\verb,>,\verb,*,\verb,),.  These parts are stripped
   761   \verb,(,\verb,*,\verb,>,\verb,*,\verb,),.  These parts are stripped