src/Doc/System/Sessions.thy
changeset 79652 93e6ca9e7595
parent 79647 b7187d4cdf68
child 79724 54d0f6edfe3a
equal deleted inserted replaced
79651:155bb0ae4ae2 79652:93e6ca9e7595
   277     \<^theory_text>\<open>section\<close> etc. The default is \<^verbatim>\<open>isamarkup\<close>, e.g. \<^theory_text>\<open>section\<close> becomes
   277     \<^theory_text>\<open>section\<close> etc. The default is \<^verbatim>\<open>isamarkup\<close>, e.g. \<^theory_text>\<open>section\<close> becomes
   278     \<^verbatim>\<open>\isamarkupsection\<close>.
   278     \<^verbatim>\<open>\isamarkupsection\<close>.
   279 
   279 
   280     \<^item> @{system_option_def "threads"} determines the number of worker threads
   280     \<^item> @{system_option_def "threads"} determines the number of worker threads
   281     for parallel checking of theories and proofs. The default \<open>0\<close> means that a
   281     for parallel checking of theories and proofs. The default \<open>0\<close> means that a
   282     sensible maximum value is determined by the underlying hardware. For
   282     sensible value is guessed from the underlying hardware. This sometimes
   283     machines with many cores or with hyperthreading, this sometimes requires
   283     requires manual adjustment (on the command-line or within personal
   284     manual adjustment (on the command-line or within personal settings or
   284     settings or preferences, not within a session \<^verbatim>\<open>ROOT\<close>).
   285     preferences, not within a session \<^verbatim>\<open>ROOT\<close>).
       
   286 
   285 
   287     \<^item> @{system_option_def "condition"} specifies a comma-separated list of
   286     \<^item> @{system_option_def "condition"} specifies a comma-separated list of
   288     process environment variables (or Isabelle settings) that are required for
   287     process environment variables (or Isabelle settings) that are required for
   289     the subsequent theories to be processed. Conditions are considered
   288     the subsequent theories to be processed. Conditions are considered
   290     ``true'' if the corresponding environment value is defined and non-empty.
   289     ``true'' if the corresponding environment value is defined and non-empty.