src/Doc/System/Environment.thy
changeset 83524 d76a77fe5d7a
parent 83321 7505b5e592b1
child 83532 87d095351f8e
equal deleted inserted replaced
83523:fd12aa8c49ba 83524:d76a77fe5d7a
   323   The @{tool_def process} tool runs the raw ML process in batch mode:
   323   The @{tool_def process} tool runs the raw ML process in batch mode:
   324   @{verbatim [display]
   324   @{verbatim [display]
   325 \<open>Usage: isabelle process [OPTIONS]
   325 \<open>Usage: isabelle process [OPTIONS]
   326 
   326 
   327   Options are:
   327   Options are:
       
   328     -C DIR       change working directory
   328     -d DIR       include session directory
   329     -d DIR       include session directory
   329     -e ML_EXPR   evaluate ML expression on startup
   330     -e ML_EXPR   evaluate ML expression on startup
   330     -f ML_FILE   evaluate ML file on startup
   331     -f ML_FILE   evaluate ML file on startup
   331     -l NAME      logic session name (default ISABELLE_LOGIC="HOL")
   332     -l NAME      logic session name (default ISABELLE_LOGIC="HOL")
   332     -m MODE      add print mode for output
   333     -m MODE      add print mode for output
   333     -o OPTION    override Isabelle system OPTION (via NAME=VAL or NAME)
   334     -o OPTION    override Isabelle system OPTION (via NAME=VAL or NAME)
       
   335     -r           redirect stderr to stdout
   334 
   336 
   335   Run the raw Isabelle ML process in batch mode.\<close>}
   337   Run the raw Isabelle ML process in batch mode.\<close>}
   336 
   338 
   337   \<^medskip>
   339   \<^medskip>
   338   Options \<^verbatim>\<open>-e\<close> and \<^verbatim>\<open>-f\<close> allow to evaluate ML code, before the ML process is
   340   Options \<^verbatim>\<open>-e\<close> and \<^verbatim>\<open>-f\<close> allow to evaluate ML code, before the ML process is
   350   mathematical Isabelle symbols.
   352   mathematical Isabelle symbols.
   351 
   353 
   352   \<^medskip>
   354   \<^medskip>
   353   Option \<^verbatim>\<open>-o\<close> allows to override Isabelle system options for this process,
   355   Option \<^verbatim>\<open>-o\<close> allows to override Isabelle system options for this process,
   354   see also \secref{sec:system-options}.
   356   see also \secref{sec:system-options}.
       
   357 
       
   358   \<^medskip>
       
   359   Option \<^verbatim>\<open>-C\<close> specifies an explicit working directory. Option \<^verbatim>\<open>-r\<close> redirects
       
   360   \<^verbatim>\<open>stderr\<close> to \<^verbatim>\<open>stdout\<close>.
   355 \<close>
   361 \<close>
   356 
   362 
   357 
   363 
   358 subsubsection \<open>Examples\<close>
   364 subsubsection \<open>Examples\<close>
   359 
   365