added lemma
authornipkow
Thu, 17 Aug 2017 07:27:17 +0200
changeset 66442 050bc74d55ed
parent 66441 b9468503742a
child 66443 657c517c7dc6
added lemma
src/HOL/List.thy
--- a/src/HOL/List.thy	Wed Aug 16 21:14:11 2017 +0200
+++ b/src/HOL/List.thy	Thu Aug 17 07:27:17 2017 +0200
@@ -4886,6 +4886,10 @@
       (meson assms transpD)
 qed simp_all
 
+lemma sorted_wrt_mono:
+  "(\<And>x y. P x y \<Longrightarrow> Q x y) \<Longrightarrow> sorted_wrt P xs \<Longrightarrow> sorted_wrt Q xs"
+by(induction xs rule: sorted_wrt_induct)(auto)
+
 text \<open>Strictly Ascending Sequences of Natural Numbers\<close>    
 
 lemma sorted_wrt_upt[simp]: "sorted_wrt (op <) [0..<n]"