diff -r dd58f13a8eb4 -r eb85850d3eb7 src/HOL/ex/CTL.thy --- a/src/HOL/ex/CTL.thy Fri Nov 17 02:19:55 2006 +0100 +++ b/src/HOL/ex/CTL.thy Fri Nov 17 02:20:03 2006 +0100 @@ -25,7 +25,7 @@ types 'a ctl = "'a set" definition - imp :: "'a ctl \ 'a ctl \ 'a ctl" (infixr "\" 75) + imp :: "'a ctl \ 'a ctl \ 'a ctl" (infixr "\" 75) where "p \ q = - p \ q" lemma [intro!]: "p \ p \ q \ q" unfolding imp_def by auto @@ -58,9 +58,11 @@ *} definition - EX :: "'a ctl \ 'a ctl" ("\ _" [80] 90) "\ p = {s. \s'. (s, s') \ \ \ s' \ p}" - EF :: "'a ctl \ 'a ctl" ("\ _" [80] 90) "\ p = lfp (\s. p \ \ s)" - EG :: "'a ctl \ 'a ctl" ("\ _" [80] 90) "\ p = gfp (\s. p \ \ s)" + EX ("\ _" [80] 90) where "\ p = {s. \s'. (s, s') \ \ \ s' \ p}" +definition + EF ("\ _" [80] 90) where "\ p = lfp (\s. p \ \ s)" +definition + EG ("\ _" [80] 90) where "\ p = gfp (\s. p \ \ s)" text {* @{text "\"}, @{text "\"} and @{text "\"} are now defined @@ -69,9 +71,11 @@ *} definition - AX :: "'a ctl \ 'a ctl" ("\ _" [80] 90) "\ p = - \ - p" - AF :: "'a ctl \ 'a ctl" ("\ _" [80] 90) "\ p = - \ - p" - AG :: "'a ctl \ 'a ctl" ("\ _" [80] 90) "\ p = - \ - p" + AX ("\ _" [80] 90) where "\ p = - \ - p" +definition + AF ("\ _" [80] 90) where "\ p = - \ - p" +definition + AG ("\ _" [80] 90) where "\ p = - \ - p" lemmas [simp] = EX_def EG_def AX_def EF_def AF_def AG_def