diff -r 8e9a8ede2f11 -r e187dacd248f doc-src/TutorialI/CTL/CTL.thy --- a/doc-src/TutorialI/CTL/CTL.thy Tue Oct 03 01:15:11 2000 +0200 +++ b/doc-src/TutorialI/CTL/CTL.thy Tue Oct 03 11:26:54 2000 +0200 @@ -1,7 +1,6 @@ -theory CTL = Main: +(*<*)theory CTL = Base:(*>*) -typedecl atom; -types state = "atom set"; +subsection{*Computation tree logic---CTL*} datatype ctl_form = Atom atom | NOT ctl_form @@ -11,13 +10,12 @@ | AF ctl_form; consts valid :: "state \ ctl_form \ bool" ("(_ \ _)" [80,80] 80) - M :: "(state \ state)set"; constdefs Paths :: "state \ (nat \ state)set" "Paths s \ {p. s = p 0 \ (\i. (p i, p(i+1)) \ M)}"; primrec -"s \ Atom a = (a\s)" +"s \ Atom a = (a \ L s)" "s \ NOT f = (~(s \ f))" "s \ And f g = (s \ f \ s \ g)" "s \ AX f = (\t. (s,t) \ M \ t \ f)" @@ -32,7 +30,7 @@ consts mc :: "ctl_form \ state set"; primrec -"mc(Atom a) = {s. a\s}" +"mc(Atom a) = {s. a \ L s}" "mc(NOT f) = -mc f" "mc(And f g) = mc f \ mc g" "mc(AX f) = {s. \t. (s,t) \ M \ t \ mc f}" @@ -231,4 +229,4 @@ apply(induct_tac f); by(auto simp add: lfp_conv_EF equalityI[OF lfp_subset_AF AF_subset_lfp]); -end; +(*<*)end(*>*)