src/Doc/JEdit/JEdit.thy
changeset 72931 fa3fbbfc1f17
parent 72896 4e63acc435bd
child 72944 50c48773b954
equal deleted inserted replaced
72930:0cc298e29aff 72931:fa3fbbfc1f17
  1285   Formal entities are semantically annotated in the source text as explained
  1285   Formal entities are semantically annotated in the source text as explained
  1286   in \secref{sec:tooltips-hyperlinks}. A \<^emph>\<open>formal scope\<close> consists of the
  1286   in \secref{sec:tooltips-hyperlinks}. A \<^emph>\<open>formal scope\<close> consists of the
  1287   defining position with all its referencing positions. This correspondence is
  1287   defining position with all its referencing positions. This correspondence is
  1288   highlighted in the text according to the cursor position, see also
  1288   highlighted in the text according to the cursor position, see also
  1289   \figref{fig:scope1}. Here the referencing positions are rendered with an
  1289   \figref{fig:scope1}. Here the referencing positions are rendered with an
  1290   additional border, in reminiscence to a hyperlink: clicking there moves the
  1290   additional border, in reminiscence to a hyperlink. A mouse click with \<^verbatim>\<open>C\<close>
  1291   cursor to the original defining position.
  1291   modifier, or the action @{action_def "isabelle.goto-entity"} (shortcut
       
  1292   \<^verbatim>\<open>CS+d\<close>) jumps to the original defining position.
  1292 
  1293 
  1293   \begin{figure}[!htb]
  1294   \begin{figure}[!htb]
  1294   \begin{center}
  1295   \begin{center}
  1295   \includegraphics[scale=0.333]{scope1}
  1296   \includegraphics[scale=0.333]{scope1}
  1296   \end{center}
  1297   \end{center}
  1298   \label{fig:scope1}
  1299   \label{fig:scope1}
  1299   \end{figure}
  1300   \end{figure}
  1300 
  1301 
  1301   The action @{action_def "isabelle.select-entity"} (shortcut \<^verbatim>\<open>CS+ENTER\<close>)
  1302   The action @{action_def "isabelle.select-entity"} (shortcut \<^verbatim>\<open>CS+ENTER\<close>)
  1302   supports semantic selection of all occurrences of the formal entity at the
  1303   supports semantic selection of all occurrences of the formal entity at the
  1303   caret position. This facilitates systematic renaming, using regular jEdit
  1304   caret position, with a defining position in the current editor buffer. This
  1304   editing of a multi-selection, see also \figref{fig:scope2}.
  1305   facilitates systematic renaming, using regular jEdit editing of a
       
  1306   multi-selection, see also \figref{fig:scope2}.
  1305 
  1307 
  1306   \begin{figure}[!htb]
  1308   \begin{figure}[!htb]
  1307   \begin{center}
  1309   \begin{center}
  1308   \includegraphics[scale=0.333]{scope2}
  1310   \includegraphics[scale=0.333]{scope2}
  1309   \end{center}
  1311   \end{center}
  1310   \caption{The result of semantic selection and systematic renaming}
  1312   \caption{The result of semantic selection and systematic renaming}
  1311   \label{fig:scope2}
  1313   \label{fig:scope2}
  1312   \end{figure}
  1314   \end{figure}
       
  1315 
       
  1316   By default, the visual feedback on scopes is restricted to definitions
       
  1317   within the visible text area. The keyboard modifier \<^verbatim>\<open>CS\<close> overrides this:
       
  1318   then all defining and referencing positions are shown. This modifier may be
       
  1319   configured via option @{system_option jedit_focus_modifier}; the default
       
  1320   coincides with the modifier for the above keyboard actions.
  1313 \<close>
  1321 \<close>
  1314 
  1322 
  1315 
  1323 
  1316 section \<open>Completion \label{sec:completion}\<close>
  1324 section \<open>Completion \label{sec:completion}\<close>
  1317 
  1325