equal
deleted
inserted
replaced
288 lemma ITLIST[import_const ITLIST : List.foldr]: |
288 lemma ITLIST[import_const ITLIST : List.foldr]: |
289 "foldr (f\<Colon>'t18437 \<Rightarrow> 't18436 \<Rightarrow> 't18436) [] b = b \<and> |
289 "foldr (f\<Colon>'t18437 \<Rightarrow> 't18436 \<Rightarrow> 't18436) [] b = b \<and> |
290 foldr f (h # t) b = f h (foldr f t b)" |
290 foldr f (h # t) b = f h (foldr f t b)" |
291 by simp |
291 by simp |
292 |
292 |
293 lemma ALL2_DEF[import_const ALL2 : List.list_all2]: |
293 lemma ALL2_DEF[import_const ALL2 : List.list.list_all2]: |
294 "list_all2 (P\<Colon>'t18495 \<Rightarrow> 't18502 \<Rightarrow> bool) [] (l2\<Colon>'t18502 list) = (l2 = []) \<and> |
294 "list_all2 (P\<Colon>'t18495 \<Rightarrow> 't18502 \<Rightarrow> bool) [] (l2\<Colon>'t18502 list) = (l2 = []) \<and> |
295 list_all2 P ((h1\<Colon>'t18495) # (t1\<Colon>'t18495 list)) l2 = |
295 list_all2 P ((h1\<Colon>'t18495) # (t1\<Colon>'t18495 list)) l2 = |
296 (if l2 = [] then False else P h1 (hd l2) \<and> list_all2 P t1 (tl l2))" |
296 (if l2 = [] then False else P h1 (hd l2) \<and> list_all2 P t1 (tl l2))" |
297 by simp (induct_tac l2, simp_all) |
297 by simp (induct_tac l2, simp_all) |
298 |
298 |