doc-src/IsarImplementation/Thy/unused.thy
changeset 20429 116255c9209b
parent 18537 2681f9e34390
child 20460 351c63bb2704
--- a/doc-src/IsarImplementation/Thy/unused.thy	Tue Aug 29 14:31:15 2006 +0200
+++ b/doc-src/IsarImplementation/Thy/unused.thy	Tue Aug 29 18:49:33 2006 +0200
@@ -1,5 +1,12 @@
 
 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
@@ -8,9 +15,10 @@
   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.
 
+*}
+