merged
authorpaulson
Fri, 13 Apr 2018 17:00:57 +0100
changeset 67978 06bce659d41b
parent 67973 9ecc78bcf1ef (diff)
parent 67977 557ea2740125 (current diff)
child 67979 53323937ee25
merged
--- a/src/HOL/List.thy	Fri Apr 13 15:58:27 2018 +0100
+++ b/src/HOL/List.thy	Fri Apr 13 17:00:57 2018 +0100
@@ -4962,6 +4962,9 @@
   "(\<And>x y. P x y \<Longrightarrow> Q x y) \<Longrightarrow> sorted_wrt P xs \<Longrightarrow> sorted_wrt Q xs"
 by(induction xs rule: induct_list012)(auto)
 
+lemma sorted_wrt01: "length xs \<le> 1 \<Longrightarrow> sorted_wrt P xs"
+by(auto simp: le_Suc_eq length_Suc_conv)
+
 text \<open>Strictly Ascending Sequences of Natural Numbers\<close>
 
 lemma sorted_wrt_upt[simp]: "sorted_wrt (<) [0..<n]"