src/Doc/JEdit/JEdit.thy
changeset 57425 625a369b4f32
parent 57420 8103a3f6f342
child 57589 e0e4ac981cf1
equal deleted inserted replaced
57424:966b12f636b9 57425:625a369b4f32
  1263   determines an additional delay (0.5 by default), before opening a completion
  1263   determines an additional delay (0.5 by default), before opening a completion
  1264   popup.  The delay gives the prover a chance to provide semantic completion
  1264   popup.  The delay gives the prover a chance to provide semantic completion
  1265   information, notably the context (\secref{sec:completion-context}).
  1265   information, notably the context (\secref{sec:completion-context}).
  1266 
  1266 
  1267   \item The system option @{system_option_ref jedit_completion_immediate}
  1267   \item The system option @{system_option_ref jedit_completion_immediate}
  1268   (disabled by default) controls whether replacement text should be inserted
  1268   (enabled by default) controls whether replacement text should be inserted
  1269   immediately without popup, regardless of @{system_option
  1269   immediately without popup, regardless of @{system_option
  1270   jedit_completion_delay}. This aggressive mode of completion is restricted to
  1270   jedit_completion_delay}. This aggressive mode of completion is restricted to
  1271   Isabelle symbols and their abbreviations (\secref{sec:symbols}).
  1271   Isabelle symbols and their abbreviations (\secref{sec:symbols}).
  1272 
  1272 
  1273   \item Completion of symbol abbreviations with only one relevant
  1273   \item Completion of symbol abbreviations with only one relevant