138 You may have to change @{verbatim |
138 You may have to change @{verbatim |
139 "$ISABELLE_HOME/contrib/ProofGeneral"} to the actual installation |
139 "$ISABELLE_HOME/contrib/ProofGeneral"} to the actual installation |
140 directory of Proof~General. |
140 directory of Proof~General. |
141 |
141 |
142 \medskip Apart from the Isabelle command line, defaults for |
142 \medskip Apart from the Isabelle command line, defaults for |
143 interface options may be given by the \texttt{PROOFGENERAL_OPTIONS} |
143 interface options may be given by the @{verbatim PROOFGENERAL_OPTIONS} |
144 setting. For example, the Emacs executable to be used may be |
144 setting. For example, the Emacs executable to be used may be |
145 configured in Isabelle's settings like this: |
145 configured in Isabelle's settings like this: |
146 \begin{ttbox} |
146 \begin{ttbox} |
147 PROOFGENERAL_OPTIONS="-p xemacs-mule" |
147 PROOFGENERAL_OPTIONS="-p xemacs-mule" |
148 \end{ttbox} |
148 \end{ttbox} |
149 |
149 |
150 Occasionally, a user's @{verbatim "~/.emacs"} file contains code |
150 Occasionally, a user's @{verbatim "~/.emacs"} file contains code |
151 that is incompatible with the (X)Emacs version used by |
151 that is incompatible with the (X)Emacs version used by |
152 Proof~General, causing the interface startup to fail prematurely. |
152 Proof~General, causing the interface startup to fail prematurely. |
153 Here the \texttt{-u false} option helps to get the interface process |
153 Here the @{verbatim "-u false"} option helps to get the interface |
154 up and running. Note that additional Lisp customization code may |
154 process up and running. Note that additional Lisp customization |
155 reside in \texttt{proofgeneral-settings.el} of @{verbatim |
155 code may reside in @{verbatim "proofgeneral-settings.el"} of |
156 "$ISABELLE_HOME/etc"} or @{verbatim "$ISABELLE_HOME_USER/etc"}. |
156 @{verbatim "$ISABELLE_HOME/etc"} or @{verbatim |
|
157 "$ISABELLE_HOME_USER/etc"}. |
157 *} |
158 *} |
158 |
159 |
159 |
160 |
160 subsubsection {* The X-Symbol package *} |
161 subsubsection {* The X-Symbol package *} |
161 |
162 |
162 text {* |
163 text {* |
163 Proof~General incorporates a version of the Emacs X-Symbol package |
164 Proof~General incorporates a version of the Emacs X-Symbol package |
164 \cite{x-symbol}, which handles proper mathematical symbols displayed |
165 \cite{x-symbol}, which handles proper mathematical symbols displayed |
165 on screen. Pass option \texttt{-x true} to the Isabelle interface |
166 on screen. Pass option @{verbatim "-x true"} to the Isabelle |
166 script, or check the appropriate Proof~General menu setting by hand. |
167 interface script, or check the appropriate Proof~General menu |
167 The main challenge of getting X-Symbol to work properly is the |
168 setting by hand. The main challenge of getting X-Symbol to work |
168 underlying (semi-automated) X11 font setup. |
169 properly is the underlying (semi-automated) X11 font setup. |
169 |
170 |
170 \medskip Using proper mathematical symbols in Isabelle theories can |
171 \medskip Using proper mathematical symbols in Isabelle theories can |
171 be very convenient for readability of large formulas. On the other |
172 be very convenient for readability of large formulas. On the other |
172 hand, the plain ASCII sources easily become somewhat unintelligible. |
173 hand, the plain ASCII sources easily become somewhat unintelligible. |
173 For example, @{text "\<Longrightarrow>"} would appear as @{verbatim "\<Longrightarrow>"} according |
174 For example, @{text "\<Longrightarrow>"} would appear as @{verbatim "\<Longrightarrow>"} according |
233 tools. First invoke |
234 tools. First invoke |
234 \begin{ttbox} |
235 \begin{ttbox} |
235 isatool mkdir Foo |
236 isatool mkdir Foo |
236 \end{ttbox} |
237 \end{ttbox} |
237 to initialize a separate directory for session @{verbatim Foo} --- |
238 to initialize a separate directory for session @{verbatim Foo} --- |
238 it is safe to experiment, since \texttt{isatool mkdir} never |
239 it is safe to experiment, since @{verbatim "isatool mkdir"} never |
239 overwrites existing files. Ensure that @{verbatim "Foo/ROOT.ML"} |
240 overwrites existing files. Ensure that @{verbatim "Foo/ROOT.ML"} |
240 holds ML commands to load all theories required for this session; |
241 holds ML commands to load all theories required for this session; |
241 furthermore @{verbatim "Foo/document/root.tex"} should include any |
242 furthermore @{verbatim "Foo/document/root.tex"} should include any |
242 special {\LaTeX} macro packages required for your document (the |
243 special {\LaTeX} macro packages required for your document (the |
243 default is usually sufficient as a start). |
244 default is usually sufficient as a start). |