diff -r 760e21900b01 -r 28e788ca2c5d src/Doc/Implementation/Logic.thy --- a/src/Doc/Implementation/Logic.thy Thu Oct 22 21:16:27 2015 +0200 +++ b/src/Doc/Implementation/Logic.thy Thu Oct 22 21:16:49 2015 +0200 @@ -636,11 +636,10 @@ \<^descr> @{ML Thm.peek_status}~\thm\ 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 oracle} - if the finished part contains some oracle invocation; @{verbatim - unfinished} if some future proofs are still pending; @{verbatim - failed} if some future proof has failed, rendering the theorem - invalid! + The three Boolean values indicate the following: \<^verbatim>\oracle\ + if the finished part contains some oracle invocation; \<^verbatim>\unfinished\ + if some future proofs are still pending; \<^verbatim>\failed\ if some future + proof has failed, rendering the theorem invalid! \<^descr> @{ML Logic.all}~\a B\ produces a Pure quantification \\a. B\, where occurrences of the atomic term \a\ in @@ -1219,18 +1218,18 @@ \begin{center} \begin{supertabular}{rclr} - @{syntax_def (inner) proof} & = & @{verbatim Lam} \params\ @{verbatim "."} \proof\ \\ - & \|\ & \\<^bold>\\ \params\ @{verbatim "."} \proof\ \\ - & \|\ & \proof\ @{verbatim "%"} \any\ \\ + @{syntax_def (inner) proof} & = & \<^verbatim>\Lam\ \params\ \<^verbatim>\.\ \proof\ \\ + & \|\ & \\<^bold>\\ \params\ \<^verbatim>\.\ \proof\ \\ + & \|\ & \proof\ \<^verbatim>\%\ \any\ \\ & \|\ & \proof\ \\\ \any\ \\ - & \|\ & \proof\ @{verbatim "%%"} \proof\ \\ + & \|\ & \proof\ \<^verbatim>\%%\ \proof\ \\ & \|\ & \proof\ \\\ \proof\ \\ & \|\ & \id | longid\ \\ \\ \param\ & = & \idt\ \\ - & \|\ & \idt\ @{verbatim ":"} \prop\ \\ - & \|\ & @{verbatim "("} \param\ @{verbatim ")"} \\ + & \|\ & \idt\ \<^verbatim>\:\ \prop\ \\ + & \|\ & \<^verbatim>\(\ \param\ \<^verbatim>\)\ \\ \\ \params\ & = & \param\ \\