src/Doc/System/Misc.thy
changeset 49072 747835eb2782
parent 48985 5386df44a037
child 50132 180d086c30dd
equal deleted inserted replaced
49071:c1ca931b3647 49072:747835eb2782
   207 *}
   207 *}
   208 
   208 
   209 
   209 
   210 section {* Creating instances of the Isabelle logo *}
   210 section {* Creating instances of the Isabelle logo *}
   211 
   211 
   212 text {* The @{tool_def logo} tool creates any instance of the generic
   212 text {* The @{tool_def logo} tool creates instances of the generic
   213   Isabelle logo as EPS or PDF.
   213   Isabelle logo as EPS and PDF, for inclusion in {\LaTeX} documents.
   214 \begin{ttbox}
   214 \begin{ttbox}
   215 Usage: isabelle logo [OPTIONS] NAME
   215 Usage: isabelle logo [OPTIONS] XYZ
   216 
   216 
   217   Create instance NAME of the Isabelle logo (as EPS or PDF).
   217   Create instance XYZ of the Isabelle logo (as EPS and PDF).
   218 
   218 
   219   Options are:
   219   Options are:
   220     -o OUTFILE   specify output file and format
   220     -n NAME      alternative output base name (default "isabelle_xyx")
   221                  (default "isabelle_name.pdf")
       
   222     -q           quiet mode
   221     -q           quiet mode
   223 \end{ttbox}
   222 \end{ttbox}
   224 
   223 
   225   Option @{verbatim "-o"} specifies an explicit output file name and
   224   Option @{verbatim "-n"} specifies an altenative (base) name for the
   226   format, e.g.\ @{verbatim "mylogo.eps"} for an EPS logo.  The default
   225   generated files.  The default is @{verbatim "isabelle_"}@{text xyz}
   227   is @{verbatim "isabelle_"}@{text name}@{verbatim ".pdf"}, with the
   226   in lower-case.
   228   lower-case version of the given name and PDF output.
       
   229 
   227 
   230   Option @{verbatim "-q"} omits printing of the result file name.
   228   Option @{verbatim "-q"} omits printing of the result file name.
   231 
   229 
   232   \medskip Implementors of Isabelle tools and applications are
   230   \medskip Implementors of Isabelle tools and applications are
   233   encouraged to make derived Isabelle logos for their own projects
   231   encouraged to make derived Isabelle logos for their own projects