src/Doc/Tutorial/Documents/Documents.thy
changeset 54936 30e2503f1aa2
parent 53015 a1119cf551e8
child 58620 7435b6a3f72e
equal deleted inserted replaced
54935:a7704d87f30a 54936:30e2503f1aa2
   341   batch-mode.  An Isabelle \bfindex{session} consists of a collection
   341   batch-mode.  An Isabelle \bfindex{session} consists of a collection
   342   of source files that may contribute to an output document.  Each
   342   of source files that may contribute to an output document.  Each
   343   session is derived from a single parent, usually an object-logic
   343   session is derived from a single parent, usually an object-logic
   344   image like \texttt{HOL}.  This results in an overall tree structure,
   344   image like \texttt{HOL}.  This results in an overall tree structure,
   345   which is reflected by the output location in the file system
   345   which is reflected by the output location in the file system
   346   (usually rooted at \verb,~/.isabelle/IsabelleXXXX/browser_info,).
   346   (the root directory is determined by the Isabelle settings variable
       
   347   \verb,ISABELLE_BROWSER_INFO,).
   347 
   348 
   348   \medskip The easiest way to manage Isabelle sessions is via
   349   \medskip The easiest way to manage Isabelle sessions is via
   349   \texttt{isabelle mkroot} (to generate an initial session source
   350   \texttt{isabelle mkroot} (to generate an initial session source
   350   setup) and \texttt{isabelle build} (to run sessions as specified in
   351   setup) and \texttt{isabelle build} (to run sessions as specified in
   351   the corresponding \texttt{ROOT} file).  These Isabelle tools are
   352   the corresponding \texttt{ROOT} file).  These Isabelle tools are