diff -r 546958347e05 -r 7247cb62406c src/HOL/Filter.thy --- a/src/HOL/Filter.thy Mon Dec 28 17:43:30 2015 +0100 +++ b/src/HOL/Filter.thy Mon Dec 28 18:03:26 2015 +0100 @@ -39,9 +39,8 @@ definition eventually :: "('a \ bool) \ 'a filter \ bool" where "eventually P F \ Rep_filter F P" -syntax (xsymbols) - "_eventually" :: "pttrn => 'a filter => bool => bool" ("(3\\<^sub>F _ in _./ _)" [0, 0, 10] 10) - +syntax + "_eventually" :: "pttrn => 'a filter => bool => bool" ("(3\\<^sub>F _ in _./ _)" [0, 0, 10] 10) translations "\\<^sub>Fx in F. P" == "CONST eventually (\x. P) F" @@ -150,9 +149,8 @@ definition frequently :: "('a \ bool) \ 'a filter \ bool" where "frequently P F \ \ eventually (\x. \ P x) F" -syntax (xsymbols) - "_frequently" :: "pttrn \ 'a filter \ bool \ bool" ("(3\\<^sub>F _ in _./ _)" [0, 0, 10] 10) - +syntax + "_frequently" :: "pttrn \ 'a filter \ bool \ bool" ("(3\\<^sub>F _ in _./ _)" [0, 0, 10] 10) translations "\\<^sub>Fx in F. P" == "CONST frequently (\x. P) F"