src/Doc/JEdit/JEdit.thy
changeset 64514 27914a4f8c70
parent 64513 56972c755027
child 64515 29f0b8d2f952
equal deleted inserted replaced
64513:56972c755027 64514:27914a4f8c70
  1168   exploration: the chain of hyperlinks may end in some source file of the
  1168   exploration: the chain of hyperlinks may end in some source file of the
  1169   underlying logic image, or within the ML bootstrap sources of Isabelle/Pure.
  1169   underlying logic image, or within the ML bootstrap sources of Isabelle/Pure.
  1170 \<close>
  1170 \<close>
  1171 
  1171 
  1172 
  1172 
       
  1173 section \<open>Formal scopes and semantic selection\<close>
       
  1174 
       
  1175 text \<open>
       
  1176   Formal entities are semantically annotated in the source text as explained
       
  1177   in \secref{sec:tooltips-hyperlinks}. A \<^emph>\<open>formal scope\<close> consists of the
       
  1178   defining position with all its referencing positions. This correspondence is
       
  1179   highlighted in the text according to the cursor position, see also
       
  1180   \figref{fig:scope1}. Here the referencing positions are rendered with an
       
  1181   additional border, in reminiscence to a hyperlink: clicking there moves the
       
  1182   cursor to the original defining position.
       
  1183 
       
  1184   \begin{figure}[!htb]
       
  1185   \begin{center}
       
  1186   \includegraphics[scale=0.5]{scope1}
       
  1187   \end{center}
       
  1188   \caption{Scope of formal entity: defining vs.\ referencing positions}
       
  1189   \label{fig:scope1}
       
  1190   \end{figure}
       
  1191 
       
  1192   The action @{action_def "isabelle.select-entity"} (shortcut \<^verbatim>\<open>CS+ENTER\<close>)
       
  1193   supports semantic selection of all occurrences of the formal entity at the
       
  1194   caret position. This facilitates systematic renaming, using regular jEdit
       
  1195   editing of a multi-selection, see also \figref{fig:scope2}.
       
  1196 
       
  1197   \begin{figure}[!htb]
       
  1198   \begin{center}
       
  1199   \includegraphics[scale=0.5]{scope2}
       
  1200   \end{center}
       
  1201   \caption{The result of semantic selection and systematic renaming}
       
  1202   \label{fig:scope2}
       
  1203   \end{figure}
       
  1204 \<close>
       
  1205 
       
  1206 
  1173 section \<open>Completion \label{sec:completion}\<close>
  1207 section \<open>Completion \label{sec:completion}\<close>
  1174 
  1208 
  1175 text \<open>
  1209 text \<open>
  1176   Smart completion of partial input is the IDE functionality \<^emph>\<open>par
  1210   Smart completion of partial input is the IDE functionality \<^emph>\<open>par
  1177   excellance\<close>. Isabelle/jEdit combines several sources of information to
  1211   excellance\<close>. Isabelle/jEdit combines several sources of information to