src/HOL/Quotient_Examples/Quotient_FSet.thy
changeset 68249 949d93804740
parent 67399 eab6ce8368fa
child 68386 98cf1c823c48
--- a/src/HOL/Quotient_Examples/Quotient_FSet.thy	Tue May 22 14:12:15 2018 +0200
+++ b/src/HOL/Quotient_Examples/Quotient_FSet.thy	Tue May 22 11:08:37 2018 +0200
@@ -69,12 +69,12 @@
 definition
   inter_list :: "'a list \<Rightarrow> 'a list \<Rightarrow> 'a list"
 where
-  [simp]: "inter_list xs ys = [x \<leftarrow> xs. x \<in> set xs \<and> x \<in> set ys]"
+  [simp]: "inter_list xs ys = filter (\<lambda>x. x \<in> set xs \<and> x \<in> set ys) xs"
 
 definition
   diff_list :: "'a list \<Rightarrow> 'a list \<Rightarrow> 'a list"
 where
-  [simp]: "diff_list xs ys = [x \<leftarrow> xs. x \<notin> set ys]"
+  [simp]: "diff_list xs ys = filter (\<lambda>x. x \<notin> set ys) xs"
 
 definition
   rsp_fold :: "('a \<Rightarrow> 'b \<Rightarrow> 'b) \<Rightarrow> bool"