src/Doc/JEdit/JEdit.thy
changeset 82439 5bc783d81201
parent 82322 94fd80f0107d
equal deleted inserted replaced
82438:a9d8e2474d2e 82439:5bc783d81201
   149   The \<^emph>\<open>Isabelle\<close> plugin is responsible for the main Prover IDE functionality
   149   The \<^emph>\<open>Isabelle\<close> plugin is responsible for the main Prover IDE functionality
   150   of Isabelle/jEdit: it manages the prover session in the background. A few
   150   of Isabelle/jEdit: it manages the prover session in the background. A few
   151   additional plugins are bundled with Isabelle/jEdit for convenience or out of
   151   additional plugins are bundled with Isabelle/jEdit for convenience or out of
   152   necessity, notably \<^emph>\<open>Console\<close> with its \<^emph>\<open>Scala\<close> sub-plugin
   152   necessity, notably \<^emph>\<open>Console\<close> with its \<^emph>\<open>Scala\<close> sub-plugin
   153   (\secref{sec:scala-console}) and \<^emph>\<open>SideKick\<close> with some Isabelle-specific
   153   (\secref{sec:scala-console}) and \<^emph>\<open>SideKick\<close> with some Isabelle-specific
   154   parsers for document tree structure (\secref{sec:sidekick}). The
   154   parsers for document tree structure (\secref{sec:sidekick}). Other plugins
   155   \<^emph>\<open>Navigator\<close> plugin is particularly important for hyperlinks within the
   155   (e.g.\ \<^emph>\<open>Console\<close>, \<^emph>\<open>ErrorList\<close>, \<^emph>\<open>SideKick\<close>) are included to saturate the
   156   formal document-model (\secref{sec:tooltips-hyperlinks}). Further plugins
   156   dependencies of bundled plugins, but have no particular use in
   157   (e.g.\ \<^emph>\<open>ErrorList\<close>, \<^emph>\<open>Code2HTML\<close>) are included to saturate the dependencies
   157   Isabelle/jEdit.
   158   of bundled plugins, but have no particular use in Isabelle/jEdit.
       
   159 \<close>
   158 \<close>
   160 
   159 
   161 
   160 
   162 subsection \<open>Options \label{sec:options}\<close>
   161 subsection \<open>Options \label{sec:options}\<close>
   163 
   162 
  1265   nested tooltips are stacking up.
  1264   nested tooltips are stacking up.
  1266 
  1265 
  1267   \<^medskip>
  1266   \<^medskip>
  1268   A black rectangle in the text indicates a hyperlink that may be followed by
  1267   A black rectangle in the text indicates a hyperlink that may be followed by
  1269   a mouse click (while the \<^verbatim>\<open>CONTROL\<close> or \<^verbatim>\<open>COMMAND\<close> modifier key is still
  1268   a mouse click (while the \<^verbatim>\<open>CONTROL\<close> or \<^verbatim>\<open>COMMAND\<close> modifier key is still
  1270   pressed). Such jumps to other text locations are recorded by the
  1269   pressed). Such jumps to other text locations are recorded by the builtin
  1271   \<^emph>\<open>Navigator\<close> plugin, which is bundled with Isabelle/jEdit and enabled by
  1270   navigator, which provides actions to move backwards or forwards, with arrow
  1272   default. There are usually navigation arrows in the main jEdit toolbar.
  1271   icons in the \<^emph>\<open>Incremental Search Bar\<close> (action @{action_ref
       
  1272   "quick-search"}). The following keyboard shortcuts are available:
       
  1273 
       
  1274   \<^medskip>
       
  1275   \begin{tabular}[t]{l}
       
  1276   @{action_ref "navigate-backwards"} (\<^verbatim>\<open>AS+LEFT\<close>) \\
       
  1277   @{action_ref "navigate-forwards"} (\<^verbatim>\<open>AS+RIGHT\<close>) \\
       
  1278   \end{tabular}\quad
       
  1279   \<^medskip>
  1273 
  1280 
  1274   Note that the link target may be a file that is itself not subject to formal
  1281   Note that the link target may be a file that is itself not subject to formal
  1275   document processing of the editor session and thus prevents further
  1282   document processing of the editor session and thus prevents further
  1276   exploration: the chain of hyperlinks may end in some source file of the
  1283   exploration: the chain of hyperlinks may end in some source file of the
  1277   underlying logic image, or within the ML bootstrap sources of Isabelle/Pure.
  1284   underlying logic image, or within the ML bootstrap sources of Isabelle/Pure.