doc-src/IsarImplementation/Thy/unused.thy
author wenzelm
Thu, 31 Aug 2006 18:27:40 +0200
changeset 20450 725a91601ed1
parent 20429 116255c9209b
child 20460 351c63bb2704
permissions -rw-r--r--
tuned;


text {*
  In practice, super-contexts emerge either by merging existing ones,
  or by adding explicit declarations.  For example, new theories are
  usually derived by importing existing theories from the library
  @{text "\<Theta> = \<Theta>\<^sub>1 + \<dots> + \<Theta>\<^isub>n"}, or 



  The Isar toplevel works differently for interactive developments
  vs.\ batch processing of theory sources.  For example, diagnostic
  commands produce a warning batch mode, because they are considered
  alien to the final theory document being produced eventually.
  Moreover, full @{text undo} with intermediate checkpoints to protect
  against destroying theories accidentally are limited to interactive
  mode.  In batch mode there is only a single strictly linear stream
  of potentially desctructive theory transformations.

  \item @{ML Toplevel.empty} is an empty transition; the Isar command
  dispatcher internally applies @{ML Toplevel.name} (for the command)
  name and @{ML Toplevel.position} for the source position.

*}