doc-src/IsarImplementation/Thy/Proof.thy
changeset 39864 f3b4fde34cd1
parent 39861 b8d89db3e238
child 40126 916cb4a28ffd
--- a/doc-src/IsarImplementation/Thy/Proof.thy	Mon Oct 18 12:33:13 2010 +0100
+++ b/doc-src/IsarImplementation/Thy/Proof.thy	Mon Oct 18 15:35:20 2010 +0100
@@ -289,11 +289,11 @@
 
   \begin{description}
 
-  \item @{ML_type Assumption.export} represents arbitrary export
-  rules, which is any function of type @{ML_type "bool -> cterm list -> thm -> thm"},
-  where the @{ML_type "bool"} indicates goal mode, and the @{ML_type
-  "cterm list"} the collection of assumptions to be discharged
-  simultaneously.
+  \item Type @{ML_type Assumption.export} represents arbitrary export
+  rules, which is any function of type @{ML_type "bool -> cterm list
+  -> thm -> thm"}, where the @{ML_type "bool"} indicates goal mode,
+  and the @{ML_type "cterm list"} the collection of assumptions to be
+  discharged simultaneously.
 
   \item @{ML Assumption.assume}~@{text "A"} turns proposition @{text
   "A"} into a primitive assumption @{text "A \<turnstile> A'"}, where the