|     67   @{verbatim [display] \<open>isabelle build -o browser_info -v -c FOL\<close>} |     67   @{verbatim [display] \<open>isabelle build -o browser_info -v -c FOL\<close>} | 
|     68  |     68  | 
|     69   The presentation output will appear in \<^verbatim>\<open>$ISABELLE_BROWSER_INFO/FOL/FOL\<close> as |     69   The presentation output will appear in \<^verbatim>\<open>$ISABELLE_BROWSER_INFO/FOL/FOL\<close> as | 
|     70   reported by the above verbose invocation of the build process. |     70   reported by the above verbose invocation of the build process. | 
|     71  |     71  | 
|     72   Many Isabelle sessions (such as \<^verbatim>\<open>HOL-Library\<close> in @{dir |     72   Many Isabelle sessions (such as \<^verbatim>\<open>HOL-Library\<close> in \<^dir>\<open>~~/src/HOL/Library\<close>) | 
|     73   "~~/src/HOL/Library"}) also provide printable documents in PDF. These are |     73   also provide printable documents in PDF. These are prepared automatically as | 
|     74   prepared automatically as well if enabled like this: |     74   well if enabled like this: | 
|     75   @{verbatim [display] \<open>isabelle build -o browser_info -o document=pdf -v -c HOL-Library\<close>} |     75   @{verbatim [display] \<open>isabelle build -o browser_info -o document=pdf -v -c HOL-Library\<close>} | 
|     76  |     76  | 
|     77   Enabling both browser info and document preparation simultaneously causes an |     77   Enabling both browser info and document preparation simultaneously causes an | 
|     78   appropriate ``document'' link to be included in the HTML index. Documents |     78   appropriate ``document'' link to be included in the HTML index. Documents | 
|     79   may be generated independently of browser information as well, see |     79   may be generated independently of browser information as well, see | 
|    175   regions. Tags are specified as a comma separated list of modifier/name |    175   regions. Tags are specified as a comma separated list of modifier/name | 
|    176   pairs: ``\<^verbatim>\<open>+\<close>\<open>foo\<close>'' (or just ``\<open>foo\<close>'') means to keep, ``\<^verbatim>\<open>-\<close>\<open>foo\<close>'' to |    176   pairs: ``\<^verbatim>\<open>+\<close>\<open>foo\<close>'' (or just ``\<open>foo\<close>'') means to keep, ``\<^verbatim>\<open>-\<close>\<open>foo\<close>'' to | 
|    177   drop, and ``\<^verbatim>\<open>/\<close>\<open>foo\<close>'' to fold text tagged as \<open>foo\<close>. The builtin default is |    177   drop, and ``\<^verbatim>\<open>/\<close>\<open>foo\<close>'' to fold text tagged as \<open>foo\<close>. The builtin default is | 
|    178   equivalent to the tag specification |    178   equivalent to the tag specification | 
|    179   ``\<^verbatim>\<open>+theory,+proof,+ML,+visible,-invisible\<close>''; see also the {\LaTeX} macros |    179   ``\<^verbatim>\<open>+theory,+proof,+ML,+visible,-invisible\<close>''; see also the {\LaTeX} macros | 
|    180   \<^verbatim>\<open>\isakeeptag\<close>, \<^verbatim>\<open>\isadroptag\<close>, and \<^verbatim>\<open>\isafoldtag\<close>, in @{file |    180   \<^verbatim>\<open>\isakeeptag\<close>, \<^verbatim>\<open>\isadroptag\<close>, and \<^verbatim>\<open>\isafoldtag\<close>, in | 
|    181   "~~/lib/texinputs/isabelle.sty"}. |    181   \<^file>\<open>~~/lib/texinputs/isabelle.sty\<close>. | 
|    182  |    182  | 
|    183   \<^medskip> |    183   \<^medskip> | 
|    184   Document preparation requires a \<^verbatim>\<open>document\<close> directory within the session |    184   Document preparation requires a \<^verbatim>\<open>document\<close> directory within the session | 
|    185   sources. This directory is supposed to contain all the files needed to |    185   sources. This directory is supposed to contain all the files needed to | 
|    186   produce the final document --- apart from the actual theories which are |    186   produce the final document --- apart from the actual theories which are | 
|    209   there as \<open>A\<close>\<^verbatim>\<open>.tex\<close>. Furthermore, a list of all generated theory files is |    209   there as \<open>A\<close>\<^verbatim>\<open>.tex\<close>. Furthermore, a list of all generated theory files is | 
|    210   put into \<^verbatim>\<open>session.tex\<close>. Typically, the root {\LaTeX} file provided by the |    210   put into \<^verbatim>\<open>session.tex\<close>. Typically, the root {\LaTeX} file provided by the | 
|    211   user would include \<^verbatim>\<open>session.tex\<close> to get a document containing all the |    211   user would include \<^verbatim>\<open>session.tex\<close> to get a document containing all the | 
|    212   theories. |    212   theories. | 
|    213  |    213  | 
|    214   The {\LaTeX} versions of the theories require some macros defined in @{file |    214   The {\LaTeX} versions of the theories require some macros defined in | 
|    215   "~~/lib/texinputs/isabelle.sty"}. Doing \<^verbatim>\<open>\usepackage{isabelle}\<close> in |    215   \<^file>\<open>~~/lib/texinputs/isabelle.sty\<close>. Doing \<^verbatim>\<open>\usepackage{isabelle}\<close> in | 
|    216   \<^verbatim>\<open>root.tex\<close> should be fine; the underlying @{tool latex} already includes an |    216   \<^verbatim>\<open>root.tex\<close> should be fine; the underlying @{tool latex} already includes an | 
|    217   appropriate path specification for {\TeX} inputs. |    217   appropriate path specification for {\TeX} inputs. | 
|    218  |    218  | 
|    219   If the text contains any references to Isabelle symbols (such as \<^verbatim>\<open>\<forall>\<close>) then |    219   If the text contains any references to Isabelle symbols (such as \<^verbatim>\<open>\<forall>\<close>) then | 
|    220   \<^verbatim>\<open>isabellesym.sty\<close> should be included as well. This package contains a |    220   \<^verbatim>\<open>isabellesym.sty\<close> should be included as well. This package contains a | 
|    221   standard set of {\LaTeX} macro definitions \<^verbatim>\<open>\isasym\<close>\<open>foo\<close> corresponding to |    221   standard set of {\LaTeX} macro definitions \<^verbatim>\<open>\isasym\<close>\<open>foo\<close> corresponding to | 
|    222   \<^verbatim>\<open>\\<close>\<^verbatim>\<open><\<close>\<open>foo\<close>\<^verbatim>\<open>>\<close>, see @{cite "isabelle-implementation"} for a complete list |    222   \<^verbatim>\<open>\\<close>\<^verbatim>\<open><\<close>\<open>foo\<close>\<^verbatim>\<open>>\<close>, see @{cite "isabelle-implementation"} for a complete list | 
|    223   of predefined Isabelle symbols. Users may invent further symbols as well, |    223   of predefined Isabelle symbols. Users may invent further symbols as well, | 
|    224   just by providing {\LaTeX} macros in a similar fashion as in @{file |    224   just by providing {\LaTeX} macros in a similar fashion as in | 
|    225   "~~/lib/texinputs/isabellesym.sty"} of the Isabelle distribution. |    225   \<^file>\<open>~~/lib/texinputs/isabellesym.sty\<close> of the Isabelle distribution. | 
|    226  |    226  | 
|    227   For proper setup of DVI and PDF documents (with hyperlinks and bookmarks), |    227   For proper setup of DVI and PDF documents (with hyperlinks and bookmarks), | 
|    228   we recommend to include @{file "~~/lib/texinputs/pdfsetup.sty"} as well. |    228   we recommend to include \<^file>\<open>~~/lib/texinputs/pdfsetup.sty\<close> as well. | 
|    229  |    229  | 
|    230   \<^medskip> |    230   \<^medskip> | 
|    231   As a final step of Isabelle document preparation, @{tool document}~\<^verbatim>\<open>-c\<close> is |    231   As a final step of Isabelle document preparation, @{tool document}~\<^verbatim>\<open>-c\<close> is | 
|    232   run on the resulting copy of the \<^verbatim>\<open>document\<close> directory. Thus the actual |    232   run on the resulting copy of the \<^verbatim>\<open>document\<close> directory. Thus the actual | 
|    233   output document is built and installed in its proper place. The generated |    233   output document is built and installed in its proper place. The generated |