doc-src/TutorialI/CTL/CTL.thy
changeset 16069 3f2a9f400168
parent 15904 a6fb4ddc05c7
child 17914 99ead7a7eb42
--- a/doc-src/TutorialI/CTL/CTL.thy	Wed May 25 09:03:53 2005 +0200
+++ b/doc-src/TutorialI/CTL/CTL.thy	Wed May 25 09:04:24 2005 +0200
@@ -244,7 +244,7 @@
 automatically. This is what happens in the step case.
 
 The induction step is similar, but more involved, because now we face nested
-occurrences of @{const SOME}. As a result, @{text fast} is no longer able to
+occurrences of @{text SOME}. As a result, @{text fast} is no longer able to
 solve the subgoal and we apply @{thm[source]someI2_ex} by hand.  We merely
 show the proof commands but do not describe the details:
 *};