src/HOL/List.thy
changeset 70183 3ea80c950023
parent 69850 5f993636ac07
child 70226 accbd801fefa
--- a/src/HOL/List.thy	Wed Apr 17 16:57:06 2019 +0000
+++ b/src/HOL/List.thy	Thu Apr 18 06:06:54 2019 +0000
@@ -1995,6 +1995,9 @@
   using longest_common_prefix[of "rev xs" "rev ys"]
   unfolding rev_swap rev_append by (metis last_rev rev_is_Nil_conv)
 
+lemma butlast_rev [simp]: "butlast (rev xs) = rev (tl xs)"
+  by (cases xs) simp_all
+
 
 subsubsection \<open>\<^const>\<open>take\<close> and \<^const>\<open>drop\<close>\<close>
 
@@ -3150,7 +3153,7 @@
 lemma hd_upt[simp]: "i < j \<Longrightarrow> hd[i..<j] = i"
   by(simp add:upt_conv_Cons)
 
-lemma tl_upt: "tl [m..<n] = [Suc m..<n]"
+lemma tl_upt [simp]: "tl [m..<n] = [Suc m..<n]"
   by (simp add: upt_rec)
 
 lemma last_upt[simp]: "i < j \<Longrightarrow> last[i..<j] = j - 1"