added code equation for subset
authorhaftmann
Mon, 01 Dec 2008 14:56:08 +0100
changeset 28939 08004ce1b167
parent 28927 7e631979922f
child 28940 df0cb410be35
added code equation for subset
src/HOL/Library/Executable_Set.thy
--- a/src/HOL/Library/Executable_Set.thy	Mon Dec 01 13:43:32 2008 +0100
+++ b/src/HOL/Library/Executable_Set.thy	Mon Dec 01 14:56:08 2008 +0100
@@ -16,7 +16,7 @@
 
 declare subset_def [symmetric, code unfold]
 
-lemma "subset A B \<longleftrightarrow> (\<forall>x\<in>A. x \<in> B)"
+lemma [code]: "subset A B \<longleftrightarrow> (\<forall>x\<in>A. x \<in> B)"
   unfolding subset_def subset_eq ..
 
 definition is_empty :: "'a set \<Rightarrow> bool" where
@@ -32,8 +32,7 @@
   "a \<in> A \<longleftrightarrow> (\<exists>x\<in>A. x = a)"
   unfolding bex_triv_one_point1 ..
 
-definition
-  filter_set :: "('a \<Rightarrow> bool) \<Rightarrow> 'a set \<Rightarrow> 'a set" where
+definition filter_set :: "('a \<Rightarrow> bool) \<Rightarrow> 'a set \<Rightarrow> 'a set" where
   "filter_set P xs = {x\<in>xs. P x}"