diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/Analysis/Sparse_In.thy --- a/src/HOL/Analysis/Sparse_In.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/Analysis/Sparse_In.thy Fri Sep 20 19:51:08 2024 +0200 @@ -10,7 +10,7 @@ subsection \A set of points sparse in another set\ definition sparse_in:: "'a :: topological_space set \ 'a set \ bool" - (infixl "(sparse'_in)" 50) + (infixl \(sparse'_in)\ 50) where "pts sparse_in A = (\x\A. \B. x\B \ open B \ (\y\B. \ y islimpt pts))" @@ -165,14 +165,14 @@ "cosparse A = Abs_filter (\P. {x. \P x} sparse_in A)" syntax - "_eventually_cosparse" :: "pttrn => 'a set => bool => bool" ("(3\\<^sub>\_\_./ _)" [0, 0, 10] 10) + "_eventually_cosparse" :: "pttrn => 'a set => bool => bool" (\(3\\<^sub>\_\_./ _)\ [0, 0, 10] 10) syntax_consts "_eventually_cosparse" == eventually translations "\\<^sub>\x\A. P" == "CONST eventually (\x. P) (CONST cosparse A)" syntax - "_qeventually_cosparse" :: "pttrn \ bool \ 'a \ 'a" ("(3\\<^sub>\_ | (_)./ _)" [0, 0, 10] 10) + "_qeventually_cosparse" :: "pttrn \ bool \ 'a \ 'a" (\(3\\<^sub>\_ | (_)./ _)\ [0, 0, 10] 10) syntax_consts "_qeventually_cosparse" == eventually translations