src/HOL/Enum.thy
changeset 46329 cf3b387ba667
parent 45963 1c7e6454883e
child 46336 39fe503602fb
--- a/src/HOL/Enum.thy	Tue Jan 24 09:13:24 2012 +0100
+++ b/src/HOL/Enum.thy	Wed Jan 25 09:32:23 2012 +0100
@@ -776,11 +776,16 @@
     unfolding enum_the_def by (auto split: list.split)
 qed
 
+code_abort enum_the
+
+subsection {* Further operations on finite types *}
+
+lemma [code]:
+  "Collect P = set (filter P enum)"
+by (auto simp add: enum_UNIV)
 
 subsection {* Closing up *}
 
-code_abort enum_the
-
 hide_const (open) a\<^isub>1 a\<^isub>2 a\<^isub>3 a\<^isub>4 a\<^isub>5