src/Doc/Tutorial/Documents/Documents.thy
changeset 67042 677cab7c2b85
parent 61593 810486f886bf
child 67398 5eb932e604a2
equal deleted inserted replaced
67041:f8b0367046bd 67042:677cab7c2b85
   349 
   349 
   350   For example, a new session \texttt{MySession} (with document
   350   For example, a new session \texttt{MySession} (with document
   351   preparation) may be produced as follows:
   351   preparation) may be produced as follows:
   352 
   352 
   353 \begin{verbatim}
   353 \begin{verbatim}
   354   isabelle mkroot -d MySession
   354   isabelle mkroot MySession
   355   isabelle build -D MySession
   355   isabelle build -D MySession
   356 \end{verbatim}
   356 \end{verbatim}
   357 
   357 
   358   The \texttt{isabelle build} job also informs about the file-system
   358   The \texttt{isabelle build} job also informs about the file-system
   359   location of the ultimate results.  The above dry run should be able
   359   location of the ultimate results.  The above dry run should be able