doc-src/TutorialI/CTL/CTL.thy
changeset 27027 63f0b638355c
parent 27015 f8537d69f514
child 35416 d8d7d1b785af
--- a/doc-src/TutorialI/CTL/CTL.thy	Fri May 30 17:03:37 2008 +0200
+++ b/doc-src/TutorialI/CTL/CTL.thy	Fri May 30 17:52:10 2008 +0200
@@ -337,12 +337,12 @@
 an auxiliary function:
 *}
 
-consts until:: "state set \<Rightarrow> state set \<Rightarrow> state \<Rightarrow> state list \<Rightarrow> bool"
 primrec
-"until A B s []    = (s \<in> B)"
+until:: "state set \<Rightarrow> state set \<Rightarrow> state \<Rightarrow> state list \<Rightarrow> bool" where
+"until A B s []    = (s \<in> B)" |
 "until A B s (t#p) = (s \<in> A \<and> (s,t) \<in> M \<and> until A B t p)"
-(*<*)constdefs
- eusem :: "state set \<Rightarrow> state set \<Rightarrow> state set"
+(*<*)definition
+ eusem :: "state set \<Rightarrow> state set \<Rightarrow> state set" where
 "eusem A B \<equiv> {s. \<exists>p. until A B s p}"(*>*)
 
 text{*\noindent