src/Doc/JEdit/JEdit.thy
changeset 57589 e0e4ac981cf1
parent 57425 625a369b4f32
child 57603 0f58af858813
equal deleted inserted replaced
57588:ff31aad27661 57589:e0e4ac981cf1
  1223 
  1223 
  1224   The prover may produce \emph{no completion} markup in exceptional
  1224   The prover may produce \emph{no completion} markup in exceptional
  1225   situations, to tell that some language keywords should be excluded from
  1225   situations, to tell that some language keywords should be excluded from
  1226   further completion attempts. For example, @{verbatim ":"} within accepted
  1226   further completion attempts. For example, @{verbatim ":"} within accepted
  1227   Isar syntax looses its meaning as abbreviation for symbol @{text "\<in>"}.
  1227   Isar syntax looses its meaning as abbreviation for symbol @{text "\<in>"}.
       
  1228 
       
  1229   \medskip The completion context is \emph{ignored} for built-in templates and
       
  1230   symbols in their explicit form ``@{verbatim "\<foobar>"}''; see also
       
  1231   \secref{sec:completion-varieties}. This allows to complete within broken
       
  1232   input that escapes its normal semantic context, e.g.\ antiquotations or
       
  1233   string literals in ML, which do not allow arbitrary backslash sequences.
  1228 *}
  1234 *}
  1229 
  1235 
  1230 
  1236 
  1231 subsection {* Input events \label{sec:completion-input} *}
  1237 subsection {* Input events \label{sec:completion-input} *}
  1232 
  1238