# HG changeset patch # User nipkow # Date 1526411962 -7200 # Node ID 4ac04fe61e9856d23aa30065ea3c55fff1d0daf2 # Parent 695ff8a207b0fd9a1847d0f4fed47666703b0c96 removed duplicates diff -r 695ff8a207b0 -r 4ac04fe61e98 src/HOL/List.thy --- a/src/HOL/List.thy Tue May 15 20:34:46 2018 +0200 +++ b/src/HOL/List.thy Tue May 15 21:19:22 2018 +0200 @@ -4984,15 +4984,11 @@ lemma sorted_wrt_upt[simp]: "sorted_wrt (<) [m.. n < m" - hence "m \ n" by simp - thus ?thesis - by(induction m rule:int_le_induct)(auto simp: upto_rec1) -qed +lemma sorted_wrt_upto[simp]: "sorted_wrt (<) [i..j]" +apply(induction i j rule: upto.induct) +apply(subst upto.simps) +apply(simp) +done text \Each element is greater or equal to its index:\ @@ -5381,18 +5377,11 @@ end -lemma sorted_upt[simp]: "sorted[i.. \x \ set xs. P x \ List.find P xs = Some (Min {x\set xs. P x})"