doc-src/IsarImplementation/Thy/unused.thy
changeset 20474 af069653f1d7
parent 20470 c839b38a1f32
child 20477 e623b0e30541
--- a/doc-src/IsarImplementation/Thy/unused.thy	Mon Sep 04 18:41:33 2006 +0200
+++ b/doc-src/IsarImplementation/Thy/unused.thy	Mon Sep 04 19:49:39 2006 +0200
@@ -1,6 +1,24 @@
 
 text {*
 
+
+  \medskip The general concept supports block-structured reasoning
+  nicely, with arbitrary mechanisms for introducing local assumptions.
+  The common reasoning pattern is as follows:
+
+  \medskip
+  \begin{tabular}{l}
+  @{text "add_assms e\<^isub>1 A\<^isub>1"} \\
+  @{text "\<dots>"} \\
+  @{text "add_assms e\<^isub>n A\<^isub>n"} \\
+  @{text "export"} \\
+  \end{tabular}
+  \medskip
+
+  \noindent The final @{text "export"} will turn any fact @{text
+  "A\<^isub>1, \<dots>, A\<^isub>n \<turnstile> B"} into some @{text "\<turnstile> B'"}, by
+  applying the export rules @{text "e\<^isub>1, \<dots>, e\<^isub>n"}
+  inside-out.
   
 
   A \emph{fixed variable} acts like a local constant in the current