doc-src/TutorialI/CTL/CTL.thy
changeset 10995 ef0b521698b7
parent 10983 59961d32b1ae
child 11149 e258b536a137
--- a/doc-src/TutorialI/CTL/CTL.thy	Mon Jan 29 19:24:17 2001 +0100
+++ b/doc-src/TutorialI/CTL/CTL.thy	Mon Jan 29 22:25:45 2001 +0100
@@ -110,8 +110,10 @@
 txt{*\noindent
 In contrast to the analogous property for @{term EF}, and just
 for a change, we do not use fixed point induction but a weaker theorem,
-@{thm[source]lfp_lowerbound}:
-@{thm[display]lfp_lowerbound[of _ "S",no_vars]}
+also known in the literature (after David Park) as \emph{Park-induction}:
+\begin{center}
+@{thm lfp_lowerbound[of _ "S",no_vars]} \hfill (@{thm[source]lfp_lowerbound})
+\end{center}
 The instance of the premise @{prop"f S \<subseteq> S"} is proved pointwise,
 a decision that clarification takes for us:
 *};