treat map_filter similar to list_all, list_ex, list_ex1
authorhaftmann
Thu, 19 Jun 2025 17:15:40 +0200
changeset 82734 89347c0cc6a3
parent 82733 8b537e1af2ec
child 82735 5d0d35680311
child 82737 4694d8cce777
treat map_filter similar to list_all, list_ex, list_ex1
src/HOL/List.thy
--- a/src/HOL/List.thy	Tue Jun 17 14:11:40 2025 +0200
+++ b/src/HOL/List.thy	Thu Jun 19 17:15:40 2025 +0200
@@ -8306,9 +8306,9 @@
   intermediate lists on execution -- do not use for proving.
 \<close>
 
-lemma map_filter_simps [code]:
+lemma map_filter_simps [simp, code, no_atp]:
+  \<open>map_filter f [] = []\<close>
   \<open>map_filter f (x # xs) = (case f x of None \<Rightarrow> map_filter f xs | Some y \<Rightarrow> y # map_filter f xs)\<close>
-  \<open>map_filter f [] = []\<close>
   by (simp_all add: map_filter_def split: option.split)
 
 lemma map_filter_map_filter [code_unfold]: