src/HOL/List.thy
changeset 56953 e503d80f7f35
parent 56790 f54097170704
child 57091 1fa9c19ba2c9
--- a/src/HOL/List.thy	Tue May 13 22:14:12 2014 +0200
+++ b/src/HOL/List.thy	Wed May 14 11:33:38 2014 +0200
@@ -3262,6 +3262,10 @@
  "\<lbrakk> distinct xs; i < length xs; j < length xs \<rbrakk> \<Longrightarrow> (xs!i = xs!j) = (i = j)"
 by(auto simp: distinct_conv_nth)
 
+lemma set_update_distinct: "\<lbrakk> distinct xs;  n < length xs \<rbrakk> \<Longrightarrow>
+  set(xs[n := x]) = insert x (set xs - {xs!n})"
+by(auto simp: set_eq_iff in_set_conv_nth nth_list_update nth_eq_iff_index_eq)
+
 lemma distinct_card: "distinct xs ==> card (set xs) = size xs"
 by (induct xs) auto