changeset 61424 | c3658c18b7bc |
parent 58874 | 7172c7ffb047 |
child 61799 | 4cf66f21b764 |
--- a/src/HOL/Word/Bool_List_Representation.thy Tue Oct 13 09:21:14 2015 +0200 +++ b/src/HOL/Word/Bool_List_Representation.thy Tue Oct 13 09:21:15 2015 +0200 @@ -14,7 +14,7 @@ definition map2 :: "('a \<Rightarrow> 'b \<Rightarrow> 'c) \<Rightarrow> 'a list \<Rightarrow> 'b list \<Rightarrow> 'c list" where - "map2 f as bs = map (split f) (zip as bs)" + "map2 f as bs = map (case_prod f) (zip as bs)" lemma map2_Nil [simp, code]: "map2 f [] ys = []"