src/HOL/List.thy
changeset 41505 6d19301074cf
parent 41463 edbf0a86fb1c
child 41697 19890332febc
equal deleted inserted replaced
41503:a7462e442e35 41505:6d19301074cf
   878 
   878 
   879 lemma map_snd_zip[simp]:
   879 lemma map_snd_zip[simp]:
   880   "length xs = length ys \<Longrightarrow> map snd (zip xs ys) = ys"
   880   "length xs = length ys \<Longrightarrow> map snd (zip xs ys) = ys"
   881 by (induct rule:list_induct2, simp_all)
   881 by (induct rule:list_induct2, simp_all)
   882 
   882 
   883 type_lifting map: map
   883 enriched_type map: map
   884   by (simp_all add: fun_eq_iff id_def)
   884   by (simp_all add: fun_eq_iff id_def)
   885 
   885 
   886 
   886 
   887 subsubsection {* @{text rev} *}
   887 subsubsection {* @{text rev} *}
   888 
   888