src/Doc/JEdit/JEdit.thy
changeset 72150 510ebf846696
parent 71578 d59d557f4ee0
child 72249 4bf8a8a2d2ad
equal deleted inserted replaced
72149:36a34f3a8cb8 72150:510ebf846696
  2075 \<close>
  2075 \<close>
  2076 
  2076 
  2077 
  2077 
  2078 chapter \<open>Miscellaneous tools\<close>
  2078 chapter \<open>Miscellaneous tools\<close>
  2079 
  2079 
  2080 section \<open>Timing\<close>
  2080 section \<open>Timing and monitoring\<close>
  2081 
  2081 
  2082 text \<open>
  2082 text \<open>
  2083   Managed evaluation of commands within PIDE documents includes timing
  2083   Managed evaluation of commands within PIDE documents includes timing
  2084   information, which consists of elapsed (wall-clock) time, CPU time, and GC
  2084   information, which consists of elapsed (wall-clock) time, CPU time, and GC
  2085   (garbage collection) time. Note that in a multithreaded system it is
  2085   (garbage collection) time. Note that in a multithreaded system it is
  2101   Actual display of timing depends on the global option @{system_option_ref
  2101   Actual display of timing depends on the global option @{system_option_ref
  2102   jedit_timing_threshold}, which can be configured in \<^emph>\<open>Plugin Options~/
  2102   jedit_timing_threshold}, which can be configured in \<^emph>\<open>Plugin Options~/
  2103   Isabelle~/ General\<close>.
  2103   Isabelle~/ General\<close>.
  2104 
  2104 
  2105   \<^medskip>
  2105   \<^medskip>
       
  2106   The jEdit status line includes monitor widgets for current heap usage of
       
  2107   Java and Isabelle/ML, respectively. The one for ML includes information
       
  2108   about ongoing garbage collection (as ``ML cleanup''); a double-click opens
       
  2109   a new instance of the \<^emph>\<open>Monitor\<close> panel for further details.
       
  2110 
       
  2111   \<^medskip>
  2106   The \<^emph>\<open>Monitor\<close> panel visualizes various data collections about recent
  2112   The \<^emph>\<open>Monitor\<close> panel visualizes various data collections about recent
  2107   activity of the Isabelle/ML task farm and the underlying ML runtime system.
  2113   activity of the runtime system of Isabelle/ML and Java. There are buttons to
       
  2114   request a full garbage collection and sharing of live data on the ML heap.
  2108   The display is continuously updated according to @{system_option_ref
  2115   The display is continuously updated according to @{system_option_ref
  2109   editor_chart_delay}. Note that the painting of the chart takes considerable
  2116   editor_chart_delay}. Note that the painting of the chart takes considerable
  2110   runtime itself --- on the Java Virtual Machine that runs Isabelle/Scala, not
  2117   runtime itself --- on the Java Virtual Machine that runs Isabelle/Scala, not
  2111   Isabelle/ML. Internally, the Isabelle/Scala module \<^verbatim>\<open>isabelle.ML_Statistics\<close>
  2118   Isabelle/ML.
  2112   provides further access to statistics of Isabelle/ML.
       
  2113 \<close>
  2119 \<close>
  2114 
  2120 
  2115 
  2121 
  2116 section \<open>Low-level output\<close>
  2122 section \<open>Low-level output\<close>
  2117 
  2123