make preprocessor setup confluent
authorhaftmann
Thu, 21 Aug 2025 12:09:06 +0200
changeset 83018 e2cdcb656b24
parent 83017 5e5792b570b1
child 83019 ba4d3d4a1e0f
make preprocessor setup confluent
src/HOL/List.thy
--- a/src/HOL/List.thy	Wed Aug 20 14:09:06 2025 +0200
+++ b/src/HOL/List.thy	Thu Aug 21 12:09:06 2025 +0200
@@ -8037,6 +8037,10 @@
   \<open>member (x # xs) y \<longleftrightarrow> x = y \<or> member xs y\<close>
   by auto
 
+qualified lemma Collect_member [code_unfold, no_atp]: \<comment> \<open>make preprocessor setup confluent\<close>
+  \<open>{x. List.member xs x \<and> P x} = Set.filter P (set xs)\<close>
+  by simp
+
 end
 
 lemma list_all_iff [code_abbrev]: