doc-src/IsarImplementation/Thy/unused.thy
author wenzelm
Thu, 31 Aug 2006 22:55:49 +0200
changeset 20451 27ea2ba48fa3
parent 20429 116255c9209b
child 20460 351c63bb2704
permissions -rw-r--r--
misc cleanup;
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 {*
20429
116255c9209b more on contexts;
wenzelm
parents: 18537
diff changeset
     3
  In practice, super-contexts emerge either by merging existing ones,
116255c9209b more on contexts;
wenzelm
parents: 18537
diff changeset
     4
  or by adding explicit declarations.  For example, new theories are
116255c9209b more on contexts;
wenzelm
parents: 18537
diff changeset
     5
  usually derived by importing existing theories from the library
116255c9209b more on contexts;
wenzelm
parents: 18537
diff changeset
     6
  @{text "\<Theta> = \<Theta>\<^sub>1 + \<dots> + \<Theta>\<^isub>n"}, or 
116255c9209b more on contexts;
wenzelm
parents: 18537
diff changeset
     7
116255c9209b more on contexts;
wenzelm
parents: 18537
diff changeset
     8
116255c9209b more on contexts;
wenzelm
parents: 18537
diff changeset
     9
18537
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
    10
  The Isar toplevel works differently for interactive developments
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
    11
  vs.\ batch processing of theory sources.  For example, diagnostic
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
    12
  commands produce a warning batch mode, because they are considered
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
    13
  alien to the final theory document being produced eventually.
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
    14
  Moreover, full @{text undo} with intermediate checkpoints to protect
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
    15
  against destroying theories accidentally are limited to interactive
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
    16
  mode.  In batch mode there is only a single strictly linear stream
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
    17
  of potentially desctructive theory transformations.
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
    18
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
    19
  \item @{ML Toplevel.empty} is an empty transition; the Isar command
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
    20
  dispatcher internally applies @{ML Toplevel.name} (for the command)
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
    21
  name and @{ML Toplevel.position} for the source position.
2681f9e34390 "The Isabelle/Isar Implementation" manual;
wenzelm
parents:
diff changeset
    22
20429
116255c9209b more on contexts;
wenzelm
parents: 18537
diff changeset
    23
*}
116255c9209b more on contexts;
wenzelm
parents: 18537
diff changeset
    24