src/HOL/Word/Bool_List_Representation.thy
changeset 61424 c3658c18b7bc
parent 58874 7172c7ffb047
child 61799 4cf66f21b764
equal deleted inserted replaced
61423:9b6a0fb85fa3 61424:c3658c18b7bc
    12 imports Main Bits_Int
    12 imports Main Bits_Int
    13 begin
    13 begin
    14 
    14 
    15 definition map2 :: "('a \<Rightarrow> 'b \<Rightarrow> 'c) \<Rightarrow> 'a list \<Rightarrow> 'b list \<Rightarrow> 'c list"
    15 definition map2 :: "('a \<Rightarrow> 'b \<Rightarrow> 'c) \<Rightarrow> 'a list \<Rightarrow> 'b list \<Rightarrow> 'c list"
    16 where
    16 where
    17   "map2 f as bs = map (split f) (zip as bs)"
    17   "map2 f as bs = map (case_prod f) (zip as bs)"
    18 
    18 
    19 lemma map2_Nil [simp, code]:
    19 lemma map2_Nil [simp, code]:
    20   "map2 f [] ys = []"
    20   "map2 f [] ys = []"
    21   unfolding map2_def by auto
    21   unfolding map2_def by auto
    22 
    22