doc-src/System/Thy/Presentation.thy
changeset 41703 d27950860514
parent 40800 330eb65c9469
child 41819 2d84831dc1a0
equal deleted inserted replaced
41702:dca4c58c5d57 41703:d27950860514
   444   Options are:
   444   Options are:
   445     -C BOOL      copy existing document directory to -D PATH (default true)
   445     -C BOOL      copy existing document directory to -D PATH (default true)
   446     -D PATH      dump generated document sources into PATH
   446     -D PATH      dump generated document sources into PATH
   447     -M MAX       multithreading: maximum number of worker threads (default 1)
   447     -M MAX       multithreading: maximum number of worker threads (default 1)
   448     -P PATH      set path for remote theory browsing information
   448     -P PATH      set path for remote theory browsing information
       
   449     -Q INT       set threshold for sub-proof parallelization (default 100)
   449     -T LEVEL     multithreading: trace level (default 0)
   450     -T LEVEL     multithreading: trace level (default 0)
   450     -V VERSION   declare alternative document VERSION
   451     -V VERSION   declare alternative document VERSION
   451     -b           build mode (output heap image, using current dir)
   452     -b           build mode (output heap image, using current dir)
   452     -d FORMAT    build document as FORMAT (default false)
   453     -d FORMAT    build document as FORMAT (default false)
   453     -f NAME      use ML file NAME (default ROOT.ML)
   454     -f NAME      use ML file NAME (default ROOT.ML)
   563   Manual}~\cite{isabelle-ref}.
   564   Manual}~\cite{isabelle-ref}.
   564 
   565 
   565   \medskip The @{verbatim "-q"} option specifies the level of parallel
   566   \medskip The @{verbatim "-q"} option specifies the level of parallel
   566   proof checking: @{verbatim 0} no proofs, @{verbatim 1} toplevel
   567   proof checking: @{verbatim 0} no proofs, @{verbatim 1} toplevel
   567   proofs (default), @{verbatim 2} toplevel and nested Isar proofs.
   568   proofs (default), @{verbatim 2} toplevel and nested Isar proofs.
   568   The resulting speedup may vary, depending on the number of worker
   569   The option @{verbatim "-Q"} specifies a threshold for @{verbatim
   569   threads, granularity of proofs, and whether proof terms are enabled.
   570   "-q2"}: nested proofs are only parallelized when the current number
       
   571   of forked proofs falls below the given value (default 100).
   570 
   572 
   571   \medskip The @{verbatim "-t"} option produces a more detailed
   573   \medskip The @{verbatim "-t"} option produces a more detailed
   572   internal timing report of the session.
   574   internal timing report of the session.
   573 
   575 
   574   \medskip The @{verbatim "-v"} option causes additional information
   576   \medskip The @{verbatim "-v"} option causes additional information