src/Doc/JEdit/JEdit.thy
changeset 56059 2390391584c2
parent 55880 12f9a54ac64f
child 56466 08982abdcdad
equal deleted inserted replaced
56058:cd9ce893f2d6 56059:2390391584c2
   534   Movement within the popup is only active for multiple items.
   534   Movement within the popup is only active for multiple items.
   535   Otherwise the corresponding key event retains its standard meaning
   535   Otherwise the corresponding key event retains its standard meaning
   536   within the underlying text area.
   536   within the underlying text area.
   537 
   537 
   538   \paragraph{Explicit completion} is triggered by the keyboard
   538   \paragraph{Explicit completion} is triggered by the keyboard
   539   shortcut @{verbatim "C+b"} (action @{verbatim "isabelle.complete"}).
   539   shortcut @{verbatim "C+b"} (action @{action "isabelle.complete"}).
   540   This overrides the original jEdit binding for action @{verbatim
   540   This overrides the original jEdit binding for action @{verbatim
   541   "complete-word"}, but the latter is used as fall-back for
   541   "complete-word"}, but the latter is used as fall-back for
   542   non-Isabelle edit modes.  It is also possible to restore the
   542   non-Isabelle edit modes.  It is also possible to restore the
   543   original jEdit keyboard mapping of @{verbatim "complete-word"} via
   543   original jEdit keyboard mapping of @{verbatim "complete-word"} via
   544   \emph{Global Options / Shortcuts}.
   544   \emph{Global Options / Shortcuts}.
   751   appear in a certain style.
   751   appear in a certain style.
   752 
   752 
   753   \medskip
   753   \medskip
   754   \begin{tabular}{llll}
   754   \begin{tabular}{llll}
   755     \textbf{style} & \textbf{symbol} & \textbf{shortcut} & \textbf{action} \\\hline
   755     \textbf{style} & \textbf{symbol} & \textbf{shortcut} & \textbf{action} \\\hline
   756     superscript & @{verbatim "\<^sup>"} & @{verbatim "C+e UP"} & @{verbatim "isabelle.control-sup"} \\
   756     superscript & @{verbatim "\<^sup>"} & @{verbatim "C+e UP"} & @{action "isabelle.control-sup"} \\
   757     subscript & @{verbatim "\<^sub>"} & @{verbatim "C+e DOWN"} & @{verbatim "isabelle.control-sub"} \\
   757     subscript & @{verbatim "\<^sub>"} & @{verbatim "C+e DOWN"} & @{action "isabelle.control-sub"} \\
   758     bold face & @{verbatim "\<^bold>"} & @{verbatim "C+e RIGHT"} & @{verbatim "isabelle.control-bold"} \\
   758     bold face & @{verbatim "\<^bold>"} & @{verbatim "C+e RIGHT"} & @{action "isabelle.control-bold"} \\
   759     reset & & @{verbatim "C+e LEFT"} & @{verbatim "isabelle.control-reset"} \\
   759     reset & & @{verbatim "C+e LEFT"} & @{action "isabelle.control-reset"} \\
   760   \end{tabular}
   760   \end{tabular}
   761   \medskip
   761   \medskip
   762 
   762 
   763   To produce a single control symbol, it is also possible to complete
   763   To produce a single control symbol, it is also possible to complete
   764   on @{verbatim "\\"}@{verbatim sup}, @{verbatim "\\"}@{verbatim sub},
   764   on @{verbatim "\\"}@{verbatim sup}, @{verbatim "\\"}@{verbatim sub},