src/HOL/Filter.thy
changeset 62102 877463945ce9
parent 62101 26c0a70f78a3
child 62123 df65f5c27c15
--- a/src/HOL/Filter.thy	Fri Jan 08 17:40:59 2016 +0100
+++ b/src/HOL/Filter.thy	Fri Jan 08 17:41:04 2016 +0100
@@ -26,6 +26,11 @@
   show "(\<lambda>x. True) \<in> ?filter" by (auto intro: is_filter.intro)
 qed
 
+text \<open>Kill code generation for filters\<close>
+
+code_datatype Abs_filter
+declare [[code abort: Rep_filter]]
+
 lemma is_filter_Rep_filter: "is_filter (Rep_filter F)"
   using Rep_filter [of F] by simp