doc-src/IsarImplementation/Thy/unused.thy
author krauss
Fri, 04 Aug 2006 18:01:45 +0200
changeset 20338 ecdfc96cf4d0
parent 18537 2681f9e34390
child 20429 116255c9209b
permissions -rw-r--r--
Added Keywords: "otherwise" and "sequential", needed for function package's sequential mode.
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
18537
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
     1
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
     2
text {*
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
     3
  The Isar toplevel works differently for interactive developments
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
     4
  vs.\ batch processing of theory sources.  For example, diagnostic
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
     5
  commands produce a warning batch mode, because they are considered
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
     6
  alien to the final theory document being produced eventually.
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
     7
  Moreover, full @{text undo} with intermediate checkpoints to protect
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
     8
  against destroying theories accidentally are limited to interactive
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
     9
  mode.  In batch mode there is only a single strictly linear stream
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
    10
  of potentially desctructive theory transformations.
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
    11
*}
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
    12
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
    13
  \item @{ML Toplevel.empty} is an empty transition; the Isar command
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
    14
  dispatcher internally applies @{ML Toplevel.name} (for the command)
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
    15
  name and @{ML Toplevel.position} for the source position.
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
    16