src/Doc/System/Server.thy
changeset 68695 9072bfd24d8f
parent 68694 03e104be99af
child 68770 add44e2b8cb0
equal deleted inserted replaced
68694:03e104be99af 68695:9072bfd24d8f
   935   \<^medskip> Due to asynchronous nature of PIDE document processing, structurally
   935   \<^medskip> Due to asynchronous nature of PIDE document processing, structurally
   936   broken theories never reach the \<open>consolidated\<close> state: consequently
   936   broken theories never reach the \<open>consolidated\<close> state: consequently
   937   \<^verbatim>\<open>use_theories\<close> will wait forever. The status is checked every \<open>check_delay\<close>
   937   \<^verbatim>\<open>use_theories\<close> will wait forever. The status is checked every \<open>check_delay\<close>
   938   seconds, and bounded by \<open>check_limit\<close> attempts (default: 0, i.e.\
   938   seconds, and bounded by \<open>check_limit\<close> attempts (default: 0, i.e.\
   939   unbounded). A \<open>check_limit > 0\<close> effectively specifies a timeout of
   939   unbounded). A \<open>check_limit > 0\<close> effectively specifies a timeout of
   940   \<open>check_delay \<times> check_limit\<close> seconds.
   940   \<open>check_delay \<times> check_limit\<close> seconds; it needs to be greater than the system
       
   941   option @{system_option editor_consolidate_delay} to give PIDE processing a
       
   942   chance to consolidate document nodes in the first place.
   941 \<close>
   943 \<close>
   942 
   944 
   943 
   945 
   944 subsubsection \<open>Arguments\<close>
   946 subsubsection \<open>Arguments\<close>
   945 
   947