src/Doc/JEdit/JEdit.thy
changeset 62249 c1d6dfd645e2
parent 62212 8addfff5965a
child 62250 9cf61c91b274
equal deleted inserted replaced
62248:dca0bac351b2 62249:c1d6dfd645e2
  1014 
  1014 
  1015 section \<open>Query \label{sec:query}\<close>
  1015 section \<open>Query \label{sec:query}\<close>
  1016 
  1016 
  1017 text \<open>
  1017 text \<open>
  1018   The \<^emph>\<open>Query\<close> panel provides various GUI forms to request extra information
  1018   The \<^emph>\<open>Query\<close> panel provides various GUI forms to request extra information
  1019   from the prover. In old times the user would have issued some diagnostic
  1019   from the prover, as a replacement of old-style diagnostic commands like
  1020   command like @{command find_theorems} and inspected its output, but this is
  1020   @{command find_theorems}. There are input fields and buttons for a
  1021   now integrated into the Prover IDE.
  1021   particular query command, with output in a dedicated text area.
  1022 
  1022 
  1023   A \<^emph>\<open>Query\<close> window provides some input fields and buttons for a particular
  1023   The main query modes are presented as separate tabs: \<^emph>\<open>Find Theorems\<close>,
  1024   query command, with output in a dedicated text area. There are various query
  1024   \<^emph>\<open>Find Constants\<close>, \<^emph>\<open>Print Context\<close>, e.g.\ see \figref{fig:query}. As usual
  1025   modes: \<^emph>\<open>Find Theorems\<close>, \<^emph>\<open>Find Constants\<close>, \<^emph>\<open>Print Context\<close>, e.g.\ see
  1025   in jEdit, multiple \<^emph>\<open>Query\<close> windows may be active at the same time: any
  1026   \figref{fig:query}. As usual in jEdit, multiple \<^emph>\<open>Query\<close> windows may be
  1026   number of floating instances, but at most one docked instance (which is used
  1027   active at the same time: any number of floating instances, but at most one
  1027   by default).
  1028   docked instance (which is used by default).
       
  1029 
  1028 
  1030   \begin{figure}[!htb]
  1029   \begin{figure}[!htb]
  1031   \begin{center}
  1030   \begin{center}
  1032   \includegraphics[scale=0.333]{query}
  1031   \includegraphics[scale=0.333]{query}
  1033   \end{center}
  1032   \end{center}
  1099 
  1098 
  1100 text \<open>
  1099 text \<open>
  1101   The \<^emph>\<open>Query\<close> panel in \<^emph>\<open>Print Context\<close> mode prints information from the
  1100   The \<^emph>\<open>Query\<close> panel in \<^emph>\<open>Print Context\<close> mode prints information from the
  1102   theory or proof context, or proof state. See also the Isar commands
  1101   theory or proof context, or proof state. See also the Isar commands
  1103   @{command_ref print_context}, @{command_ref print_cases}, @{command_ref
  1102   @{command_ref print_context}, @{command_ref print_cases}, @{command_ref
  1104   print_term_bindings}, @{command_ref print_theorems}, @{command_ref
  1103   print_term_bindings}, @{command_ref print_theorems}, described in @{cite
  1105   print_state} described in @{cite "isabelle-isar-ref"}.
  1104   "isabelle-isar-ref"}.
  1106 \<close>
  1105 \<close>
  1107 
  1106 
  1108 
  1107 
  1109 section \<open>Tooltips and hyperlinks \label{sec:tooltips-hyperlinks}\<close>
  1108 section \<open>Tooltips and hyperlinks \label{sec:tooltips-hyperlinks}\<close>
  1110 
  1109 
  1111 text \<open>
  1110 text \<open>
  1112   Formally processed text (prover input or output) contains rich markup
  1111   Formally processed text (prover input or output) contains rich markup that
  1113   information that can be explored further by using the \<^verbatim>\<open>CONTROL\<close> modifier
  1112   can be explored by using the \<^verbatim>\<open>CONTROL\<close> modifier key on Linux and Windows,
  1114   key on Linux and Windows, or \<^verbatim>\<open>COMMAND\<close> on Mac OS X. Hovering with the mouse
  1113   or \<^verbatim>\<open>COMMAND\<close> on Mac OS X. Hovering with the mouse while the modifier is
  1115   while the modifier is pressed reveals a \<^emph>\<open>tooltip\<close> (grey box over the text
  1114   pressed reveals a \<^emph>\<open>tooltip\<close> (grey box over the text with a yellow popup)
  1116   with a yellow popup) and/or a \<^emph>\<open>hyperlink\<close> (black rectangle over the text
  1115   and/or a \<^emph>\<open>hyperlink\<close> (black rectangle over the text with change of mouse
  1117   with change of mouse pointer); see also \figref{fig:tooltip}.
  1116   pointer); see also \figref{fig:tooltip}.
  1118 
  1117 
  1119   \begin{figure}[!htb]
  1118   \begin{figure}[!htb]
  1120   \begin{center}
  1119   \begin{center}
  1121   \includegraphics[scale=0.5]{popup1}
  1120   \includegraphics[scale=0.5]{popup1}
  1122   \end{center}
  1121   \end{center}
  1123   \caption{Tooltip and hyperlink for some formal entity}
  1122   \caption{Tooltip and hyperlink for some formal entity}
  1124   \label{fig:tooltip}
  1123   \label{fig:tooltip}
  1125   \end{figure}
  1124   \end{figure}
  1126 
  1125 
  1127   Tooltip popups use the same rendering mechanisms as the main text area, and
  1126   Tooltip popups use the same rendering technology as the main text area, and
  1128   further tooltips and/or hyperlinks may be exposed recursively by the same
  1127   further tooltips and/or hyperlinks may be exposed recursively by the same
  1129   mechanism; see \figref{fig:nested-tooltips}.
  1128   mechanism; see \figref{fig:nested-tooltips}.
  1130 
  1129 
  1131   \begin{figure}[!htb]
  1130   \begin{figure}[!htb]
  1132   \begin{center}
  1131   \begin{center}
  1144   \<^medskip>
  1143   \<^medskip>
  1145   A black rectangle in the text indicates a hyperlink that may be followed by
  1144   A black rectangle in the text indicates a hyperlink that may be followed by
  1146   a mouse click (while the \<^verbatim>\<open>CONTROL\<close> or \<^verbatim>\<open>COMMAND\<close> modifier key is still
  1145   a mouse click (while the \<^verbatim>\<open>CONTROL\<close> or \<^verbatim>\<open>COMMAND\<close> modifier key is still
  1147   pressed). Such jumps to other text locations are recorded by the
  1146   pressed). Such jumps to other text locations are recorded by the
  1148   \<^emph>\<open>Navigator\<close> plugin, which is bundled with Isabelle/jEdit and enabled by
  1147   \<^emph>\<open>Navigator\<close> plugin, which is bundled with Isabelle/jEdit and enabled by
  1149   default, including navigation arrows in the main jEdit toolbar.
  1148   default. There are usually navigation arrows in the main jEdit toolbar.
  1150 
  1149 
  1151   Also note that the link target may be a file that is itself not subject to
  1150   Note that the link target may be a file that is itself not subject to formal
  1152   formal document processing of the editor session and thus prevents further
  1151   document processing of the editor session and thus prevents further
  1153   exploration: the chain of hyperlinks may end in some source file of the
  1152   exploration: the chain of hyperlinks may end in some source file of the
  1154   underlying logic image, or within the ML bootstrap sources of
  1153   underlying logic image, or within the ML bootstrap sources of Isabelle/Pure.
  1155   Isabelle/Pure.
       
  1156 \<close>
  1154 \<close>
  1157 
  1155 
  1158 
  1156 
  1159 section \<open>Completion \label{sec:completion}\<close>
  1157 section \<open>Completion \label{sec:completion}\<close>
  1160 
  1158