Isar.goal: tactical goal only;
authorwenzelm
Thu, 10 Apr 2008 16:15:53 +0200
changeset 26617 e99719e70925
parent 26616 b5fd3ad271ec
child 26618 f3535afb58e8
Isar.goal: tactical goal only;
doc-src/IsarImplementation/Thy/document/integration.tex
doc-src/IsarImplementation/Thy/integration.thy
--- a/doc-src/IsarImplementation/Thy/document/integration.tex	Thu Apr 10 15:04:11 2008 +0200
+++ b/doc-src/IsarImplementation/Thy/document/integration.tex	Thu Apr 10 16:15:53 2008 +0200
@@ -335,7 +335,7 @@
   \indexml{Isar.state}\verb|Isar.state: unit -> Toplevel.state| \\
   \indexml{Isar.exn}\verb|Isar.exn: unit -> (exn * string) option| \\
   \indexml{Isar.context}\verb|Isar.context: unit -> Proof.context| \\
-  \indexml{Isar.goal}\verb|Isar.goal: unit -> thm list * thm| \\
+  \indexml{Isar.goal}\verb|Isar.goal: unit -> thm| \\
   \end{mldecls}
 
   \begin{description}
@@ -353,8 +353,8 @@
   \item \verb|Isar.context ()| produces the proof context from \verb|Isar.state ()|, analogous to \verb|Context.proof_of|
   (\secref{sec:generic-context}).
 
-  \item \verb|Isar.goal ()| picks the goal configuration from \verb|Isar.state ()|, consisting on the current facts and the goal
-  represented as a theorem according to \secref{sec:tactical-goals}.
+  \item \verb|Isar.goal ()| picks the tactical goal from \verb|Isar.state ()|, represented as a theorem according to
+  \secref{sec:tactical-goals}.
 
   \end{description}%
 \end{isamarkuptext}%
--- a/doc-src/IsarImplementation/Thy/integration.thy	Thu Apr 10 15:04:11 2008 +0200
+++ b/doc-src/IsarImplementation/Thy/integration.thy	Thu Apr 10 16:15:53 2008 +0200
@@ -275,7 +275,7 @@
   @{index_ML Isar.state: "unit -> Toplevel.state"} \\
   @{index_ML Isar.exn: "unit -> (exn * string) option"} \\
   @{index_ML Isar.context: "unit -> Proof.context"} \\
-  @{index_ML Isar.goal: "unit -> thm list * thm"} \\
+  @{index_ML Isar.goal: "unit -> thm"} \\
   \end{mldecls}
 
   \begin{description}
@@ -294,9 +294,9 @@
   "Isar.state ()"}, analogous to @{ML Context.proof_of}
   (\secref{sec:generic-context}).
 
-  \item @{ML "Isar.goal ()"} picks the goal configuration from @{ML
-  "Isar.state ()"}, consisting on the current facts and the goal
-  represented as a theorem according to \secref{sec:tactical-goals}.
+  \item @{ML "Isar.goal ()"} picks the tactical goal from @{ML
+  "Isar.state ()"}, represented as a theorem according to
+  \secref{sec:tactical-goals}.
 
   \end{description}
 *}