added lemma
authornipkow
Mon, 23 Oct 2017 14:45:10 +0200
changeset 66905 0d31dfa96aba
parent 66904 d9783ea1160c
child 66907 603a00f21817
added lemma
src/HOL/List.thy
--- a/src/HOL/List.thy	Mon Oct 23 14:12:09 2017 +0200
+++ b/src/HOL/List.thy	Mon Oct 23 14:45:10 2017 +0200
@@ -5022,6 +5022,9 @@
   with \<open>sorted xs\<close> show ?thesis by (simp add: sorted_append)
 qed
 
+lemma sorted_replicate [simp]: "sorted(replicate n x)"
+by(induction n) (auto simp: sorted_Cons)
+
 lemma sorted_remdups[simp]:
   "sorted l \<Longrightarrow> sorted (remdups l)"
 by (induct l) (auto simp: sorted_Cons)