src/Doc/Implementation/Logic.thy
changeset 70569 095dadc62bb5
parent 70568 6e055d313f73
child 70915 bd4d37edfee4
--- a/src/Doc/Implementation/Logic.thy	Sat Aug 17 17:57:10 2019 +0200
+++ b/src/Doc/Implementation/Logic.thy	Sat Aug 17 17:59:55 2019 +0200
@@ -579,7 +579,6 @@
   \end{mldecls}
   \begin{mldecls}
   @{index_ML_type thm} \\
-  @{index_ML Thm.peek_status: "thm -> {oracle: bool, unfinished: bool, failed: bool}"} \\
   @{index_ML Thm.transfer: "theory -> thm -> thm"} \\
   @{index_ML Thm.assume: "cterm -> thm"} \\
   @{index_ML Thm.forall_intr: "cterm -> thm -> thm"} \\
@@ -602,13 +601,6 @@
   @{index_ML Thm_Deps.all_oracles: "thm list -> (string * term option) list"} \\
   \end{mldecls}
 
-  \<^descr> \<^ML>\<open>Thm.peek_status\<close>~\<open>thm\<close> informs about the current status of the
-  derivation object behind the given theorem. This is a snapshot of a
-  potentially ongoing (parallel) evaluation of proofs. The three Boolean
-  values indicate the following: \<^verbatim>\<open>oracle\<close> if the finished part contains some
-  oracle invocation; \<^verbatim>\<open>unfinished\<close> if some future proofs are still pending;
-  \<^verbatim>\<open>failed\<close> if some future proof has failed, rendering the theorem invalid!
-
   \<^descr> \<^ML>\<open>Logic.all\<close>~\<open>a B\<close> produces a Pure quantification \<open>\<And>a. B\<close>, where
   occurrences of the atomic term \<open>a\<close> in the body proposition \<open>B\<close> are replaced
   by bound variables. (See also \<^ML>\<open>lambda\<close> on terms.)