src/Doc/JEdit/JEdit.thy
changeset 56059 2390391584c2
parent 55880 12f9a54ac64f
child 56466 08982abdcdad
--- a/src/Doc/JEdit/JEdit.thy	Wed Mar 12 12:18:41 2014 +0100
+++ b/src/Doc/JEdit/JEdit.thy	Wed Mar 12 14:17:13 2014 +0100
@@ -536,7 +536,7 @@
   within the underlying text area.
 
   \paragraph{Explicit completion} is triggered by the keyboard
-  shortcut @{verbatim "C+b"} (action @{verbatim "isabelle.complete"}).
+  shortcut @{verbatim "C+b"} (action @{action "isabelle.complete"}).
   This overrides the original jEdit binding for action @{verbatim
   "complete-word"}, but the latter is used as fall-back for
   non-Isabelle edit modes.  It is also possible to restore the
@@ -753,10 +753,10 @@
   \medskip
   \begin{tabular}{llll}
     \textbf{style} & \textbf{symbol} & \textbf{shortcut} & \textbf{action} \\\hline
-    superscript & @{verbatim "\<^sup>"} & @{verbatim "C+e UP"} & @{verbatim "isabelle.control-sup"} \\
-    subscript & @{verbatim "\<^sub>"} & @{verbatim "C+e DOWN"} & @{verbatim "isabelle.control-sub"} \\
-    bold face & @{verbatim "\<^bold>"} & @{verbatim "C+e RIGHT"} & @{verbatim "isabelle.control-bold"} \\
-    reset & & @{verbatim "C+e LEFT"} & @{verbatim "isabelle.control-reset"} \\
+    superscript & @{verbatim "\<^sup>"} & @{verbatim "C+e UP"} & @{action "isabelle.control-sup"} \\
+    subscript & @{verbatim "\<^sub>"} & @{verbatim "C+e DOWN"} & @{action "isabelle.control-sub"} \\
+    bold face & @{verbatim "\<^bold>"} & @{verbatim "C+e RIGHT"} & @{action "isabelle.control-bold"} \\
+    reset & & @{verbatim "C+e LEFT"} & @{action "isabelle.control-reset"} \\
   \end{tabular}
   \medskip