src/HOL/Quotient_Examples/Quotient_FSet.thy
changeset 68386 98cf1c823c48
parent 68249 949d93804740
child 69597 ff784d5a5bfb
--- a/src/HOL/Quotient_Examples/Quotient_FSet.thy	Sun Jun 03 19:06:56 2018 +0200
+++ b/src/HOL/Quotient_Examples/Quotient_FSet.thy	Wed Jun 06 11:12:37 2018 +0200
@@ -69,12 +69,12 @@
 definition
   inter_list :: "'a list \<Rightarrow> 'a list \<Rightarrow> 'a list"
 where
-  [simp]: "inter_list xs ys = filter (\<lambda>x. x \<in> set xs \<and> x \<in> set ys) xs"
+  [simp]: "inter_list xs ys = [x \<leftarrow> xs. x \<in> set xs \<and> x \<in> set ys]"
 
 definition
   diff_list :: "'a list \<Rightarrow> 'a list \<Rightarrow> 'a list"
 where
-  [simp]: "diff_list xs ys = filter (\<lambda>x. x \<notin> set ys) xs"
+  [simp]: "diff_list xs ys = [x \<leftarrow> xs. x \<notin> set ys]"
 
 definition
   rsp_fold :: "('a \<Rightarrow> 'b \<Rightarrow> 'b) \<Rightarrow> bool"