author | nipkow |
Thu, 14 Sep 2017 17:36:06 +0200 | |
changeset 66657 | 6f82e2ad261a |
parent 66656 | 8f4d252ce2fe |
child 66658 | 59acf5e73176 |
src/HOL/List.thy | file | annotate | diff | comparison | revisions |
--- a/src/HOL/List.thy Wed Sep 13 17:40:54 2017 +0200 +++ b/src/HOL/List.thy Thu Sep 14 17:36:06 2017 +0200 @@ -2034,6 +2034,9 @@ lemma drop_Suc: "drop (Suc n) xs = drop n (tl xs)" by(cases xs, simp_all) +lemma hd_take: "j > 0 \<Longrightarrow> hd (take j xs) = hd xs" +by (metis gr0_conv_Suc list.sel(1) take.simps(1) take_Suc) + lemma take_tl: "take n (tl xs) = tl (take (Suc n) xs)" by (induct xs arbitrary: n) simp_all