src/Doc/JEdit/JEdit.thy
changeset 61483 07c8d5d8acab
parent 61477 e467ae7aa808
child 61493 0debd22f0c0e
--- a/src/Doc/JEdit/JEdit.thy	Mon Oct 19 16:26:01 2015 +0200
+++ b/src/Doc/JEdit/JEdit.thy	Mon Oct 19 16:37:45 2015 +0200
@@ -579,13 +579,19 @@
     superscript & @{verbatim "\<^sup>"} & @{verbatim "C+e UP"} & @{action_ref "isabelle.control-sup"} \\
     subscript & @{verbatim "\<^sub>"} & @{verbatim "C+e DOWN"} & @{action_ref "isabelle.control-sub"} \\
     bold face & @{verbatim "\<^bold>"} & @{verbatim "C+e RIGHT"} & @{action_ref "isabelle.control-bold"} \\
-    reset & & @{verbatim "C+e LEFT"} & @{action_ref "isabelle.control-reset"} \\
+    emphasized & @{verbatim "\<^emph>"} & @{verbatim "C+e LEF"} & @{action_ref "isabelle.control-emph"} \\
+    reset & & @{verbatim "C+e BACK_SPACE"} & @{action_ref "isabelle.control-reset"} \\
   \end{tabular}
   \<^medskip>
- 
-  To produce a single control symbol, it is also possible to complete
-  on @{verbatim "\\"}@{verbatim sup}, @{verbatim "\\"}@{verbatim sub},
-  @{verbatim "\\"}@{verbatim bold} as for regular symbols.\<close>
+
+  To produce a single control symbol, it is also possible to complete on
+  @{verbatim "\\"}@{verbatim sup}, @{verbatim "\\"}@{verbatim sub}, @{verbatim
+  "\\"}@{verbatim bold}, @{verbatim "\\"}@{verbatim emph} as for regular
+  symbols.
+
+  The emphasized style only takes effect in document output, not in the
+  editor.
+\<close>
 
 
 section \<open>SideKick parsers \label{sec:sidekick}\<close>