63 @{verbatim [display] |
63 @{verbatim [display] |
64 \<open>Usage: isabelle console [OPTIONS] |
64 \<open>Usage: isabelle console [OPTIONS] |
65 |
65 |
66 Options are: |
66 Options are: |
67 -d DIR include session directory |
67 -d DIR include session directory |
68 -l NAME logic session name (default ISABELLE_LOGIC) |
68 -l NAME logic session name (default ISABELLE_LOGIC="HOL") |
69 -m MODE add print mode for output |
69 -m MODE add print mode for output |
70 -n no build of session image on startup |
70 -n no build of session image on startup |
71 -o OPTION override Isabelle system OPTION (via NAME=VAL or NAME) |
71 -o OPTION override Isabelle system OPTION (via NAME=VAL or NAME) |
|
72 -r logic session is RAW_ML_SYSTEM |
72 -s system build mode for session image |
73 -s system build mode for session image |
73 |
74 |
74 Run Isabelle process with raw ML console and line editor |
75 Run Isabelle process with raw ML console and line editor |
75 (default ISABELLE_LINE_EDITOR).\<close>} |
76 (default ISABELLE_LINE_EDITOR).\<close>} |
76 |
77 |
77 The \<^verbatim>\<open>-l\<close> option specifies the logic session name. By default, its heap |
78 The \<^verbatim>\<open>-l\<close> option specifies the logic session name. By default, its heap |
78 image is checked and built on demand, but the option \<^verbatim>\<open>-n\<close> skips that. |
79 image is checked and built on demand, but the option \<^verbatim>\<open>-n\<close> skips that. |
|
80 |
|
81 Option \<^verbatim>\<open>-r\<close> abbreviates \<^verbatim>\<open>-l RAW_ML_SYSTEM\<close>, which is relevant to bootstrap |
|
82 Isabelle/Pure interactively. |
79 |
83 |
80 Options \<^verbatim>\<open>-d\<close>, \<^verbatim>\<open>-o\<close>, \<^verbatim>\<open>-s\<close> are passed directly to @{tool build} |
84 Options \<^verbatim>\<open>-d\<close>, \<^verbatim>\<open>-o\<close>, \<^verbatim>\<open>-s\<close> are passed directly to @{tool build} |
81 (\secref{sec:tool-build}). |
85 (\secref{sec:tool-build}). |
82 |
86 |
83 Options \<^verbatim>\<open>-m\<close>, \<^verbatim>\<open>-o\<close> are passed directly to the underlying Isabelle process |
87 Options \<^verbatim>\<open>-m\<close>, \<^verbatim>\<open>-o\<close> are passed directly to the underlying Isabelle process |