author | haftmann |
Fri, 30 Mar 2007 16:19:00 +0200 | |
changeset 22551 | e52f5400e331 |
parent 22550 | c5039bee2602 |
child 22552 | 70f5cf8a0fad |
src/HOL/List.thy | file | annotate | diff | comparison | revisions |
--- a/src/HOL/List.thy Fri Mar 30 16:18:59 2007 +0200 +++ b/src/HOL/List.thy Fri Mar 30 16:19:00 2007 +0200 @@ -1601,6 +1601,10 @@ apply (case_tac y, auto) done +lemma list_all2_eq: + "xs = ys \<longleftrightarrow> list_all2 (op =) xs ys" + by (induct xs ys rule: list_induct2') auto + subsubsection {* @{text foldl} and @{text foldr} *}