diff -r f7c00119e6e7 -r ca53150406c9 src/HOL/Finite_Set.thy --- a/src/HOL/Finite_Set.thy Sat Nov 14 18:37:49 2015 +0100 +++ b/src/HOL/Finite_Set.thy Sun Nov 15 12:39:51 2015 +0100 @@ -11,11 +11,17 @@ subsection \Predicate for finite sets\ +context + notes [[inductive_defs]] +begin + inductive finite :: "'a set \ bool" where emptyI [simp, intro!]: "finite {}" | insertI [simp, intro!]: "finite A \ finite (insert a A)" +end + simproc_setup finite_Collect ("finite (Collect P)") = \K Set_Comprehension_Pointfree.simproc\ declare [[simproc del: finite_Collect]]