equal
deleted
inserted
replaced
164 definition cosparse :: "'a set \<Rightarrow> 'a :: topological_space filter" where |
164 definition cosparse :: "'a set \<Rightarrow> 'a :: topological_space filter" where |
165 "cosparse A = Abs_filter (\<lambda>P. {x. \<not>P x} sparse_in A)" |
165 "cosparse A = Abs_filter (\<lambda>P. {x. \<not>P x} sparse_in A)" |
166 |
166 |
167 syntax |
167 syntax |
168 "_eventually_cosparse" :: "pttrn => 'a set => bool => bool" ("(3\<forall>\<^sub>\<approx>_\<in>_./ _)" [0, 0, 10] 10) |
168 "_eventually_cosparse" :: "pttrn => 'a set => bool => bool" ("(3\<forall>\<^sub>\<approx>_\<in>_./ _)" [0, 0, 10] 10) |
|
169 syntax_consts |
|
170 "_eventually_cosparse" == eventually |
169 translations |
171 translations |
170 "\<forall>\<^sub>\<approx>x\<in>A. P" == "CONST eventually (\<lambda>x. P) (CONST cosparse A)" |
172 "\<forall>\<^sub>\<approx>x\<in>A. P" == "CONST eventually (\<lambda>x. P) (CONST cosparse A)" |
171 |
173 |
172 syntax |
174 syntax |
173 "_qeventually_cosparse" :: "pttrn \<Rightarrow> bool \<Rightarrow> 'a \<Rightarrow> 'a" ("(3\<forall>\<^sub>\<approx>_ | (_)./ _)" [0, 0, 10] 10) |
175 "_qeventually_cosparse" :: "pttrn \<Rightarrow> bool \<Rightarrow> 'a \<Rightarrow> 'a" ("(3\<forall>\<^sub>\<approx>_ | (_)./ _)" [0, 0, 10] 10) |
|
176 syntax_consts |
|
177 "_qeventually_cosparse" == eventually |
174 translations |
178 translations |
175 "\<forall>\<^sub>\<approx>x|P. t" => "CONST eventually (\<lambda>x. t) (CONST cosparse {x. P})" |
179 "\<forall>\<^sub>\<approx>x|P. t" => "CONST eventually (\<lambda>x. t) (CONST cosparse {x. P})" |
176 |
180 |
177 print_translation \<open> |
181 print_translation \<open> |
178 let |
182 let |