diff -r f6e595e4f608 -r 261cd8722677 src/HOL/Filter.thy --- a/src/HOL/Filter.thy Mon Sep 23 12:59:10 2024 +0200 +++ b/src/HOL/Filter.thy Mon Sep 23 13:32:38 2024 +0200 @@ -40,7 +40,7 @@ where "eventually P F \ Rep_filter F P" syntax - "_eventually" :: "pttrn => 'a filter => bool => bool" ("(3\\<^sub>F _ in _./ _)" [0, 0, 10] 10) + "_eventually" :: "pttrn => 'a filter => bool => bool" (\(3\\<^sub>F _ in _./ _)\ [0, 0, 10] 10) syntax_consts "_eventually" == eventually translations @@ -160,7 +160,7 @@ where "frequently P F \ \ eventually (\x. \ P x) F" syntax - "_frequently" :: "pttrn \ 'a filter \ bool \ bool" ("(3\\<^sub>F _ in _./ _)" [0, 0, 10] 10) + "_frequently" :: "pttrn \ 'a filter \ bool \ bool" (\(3\\<^sub>F _ in _./ _)\ [0, 0, 10] 10) syntax_consts "_frequently" == frequently translations @@ -1033,15 +1033,15 @@ definition "cofinite = Abs_filter (\P. finite {x. \ P x})" -abbreviation Inf_many :: "('a \ bool) \ bool" (binder "\\<^sub>\" 10) +abbreviation Inf_many :: "('a \ bool) \ bool" (binder \\\<^sub>\\ 10) where "Inf_many P \ frequently P cofinite" -abbreviation Alm_all :: "('a \ bool) \ bool" (binder "\\<^sub>\" 10) +abbreviation Alm_all :: "('a \ bool) \ bool" (binder \\\<^sub>\\ 10) where "Alm_all P \ eventually P cofinite" notation (ASCII) - Inf_many (binder "INFM " 10) and - Alm_all (binder "MOST " 10) + Inf_many (binder \INFM \ 10) and + Alm_all (binder \MOST \ 10) lemma eventually_cofinite: "eventually P cofinite \ finite {x. \ P x}" unfolding cofinite_def @@ -1080,7 +1080,7 @@ subsubsection \Product of filters\ -definition prod_filter :: "'a filter \ 'b filter \ ('a \ 'b) filter" (infixr "\\<^sub>F" 80) where +definition prod_filter :: "'a filter \ 'b filter \ ('a \ 'b) filter" (infixr \\\<^sub>F\ 80) where "prod_filter F G = (\(P, Q)\{(P, Q). eventually P F \ eventually Q G}. principal {(x, y). P x \ Q y})" @@ -1307,7 +1307,7 @@ "filterlim f F2 F1 \ filtermap f F1 \ F2" syntax - "_LIM" :: "pttrns \ 'a \ 'b \ 'a \ bool" ("(3LIM (_)/ (_)./ (_) :> (_))" [1000, 10, 0, 10] 10) + "_LIM" :: "pttrns \ 'a \ 'b \ 'a \ bool" (\(3LIM (_)/ (_)./ (_) :> (_))\ [1000, 10, 0, 10] 10) syntax_consts "_LIM" == filterlim