equal
deleted
inserted
replaced
220 all related examples. The @{verbatim all} target shall do |
220 all related examples. The @{verbatim all} target shall do |
221 @{verbatim images} and @{verbatim test}. |
221 @{verbatim images} and @{verbatim test}. |
222 *} |
222 *} |
223 |
223 |
224 |
224 |
225 section {* Make all logics *} |
|
226 |
|
227 text {* The @{tool_def makeall} tool applies Isabelle make to any |
|
228 Isabelle component (cf.\ \secref{sec:components}) that contains an |
|
229 @{verbatim IsaMakefile}: |
|
230 \begin{ttbox} |
|
231 Usage: isabelle makeall [ARGS ...] |
|
232 |
|
233 Apply isabelle make to all components with IsaMakefile (passing ARGS). |
|
234 \end{ttbox} |
|
235 |
|
236 The arguments @{verbatim ARGS} are just passed verbatim to each |
|
237 @{tool make} invocation. |
|
238 *} |
|
239 |
|
240 |
|
241 section {* Printing documents *} |
225 section {* Printing documents *} |
242 |
226 |
243 text {* |
227 text {* |
244 The @{tool_def print} tool prints documents: |
228 The @{tool_def print} tool prints documents: |
245 \begin{ttbox} |
229 \begin{ttbox} |