author | nipkow |
Wed, 04 May 2022 07:20:20 +0200 | |
changeset 75448 | 53a60eae475f |
parent 75447 | d1417d9c6deb |
child 75449 | 51e05af57455 |
src/HOL/List.thy | file | annotate | diff | comparison | revisions |
--- a/src/HOL/List.thy Fri Apr 22 16:55:48 2022 +0200 +++ b/src/HOL/List.thy Wed May 04 07:20:20 2022 +0200 @@ -970,6 +970,8 @@ lemma tl_append2 [simp]: "xs \<noteq> [] \<Longrightarrow> tl (xs @ ys) = tl xs @ ys" by (simp add: tl_append split: list.split) +lemma tl_append_if: "tl (xs @ ys) = (if xs = [] then tl ys else tl xs @ ys)" +by (simp) lemma Cons_eq_append_conv: "x#xs = ys@zs = (ys = [] \<and> x#xs = zs \<or> (\<exists>ys'. x#ys' = ys \<and> xs = ys'@zs))"