| author | wenzelm | 
| Mon, 24 Apr 2017 11:52:51 +0200 | |
| changeset 65573 | 0f3fdf689bf9 | 
| parent 65388 | a8d868477bc0 | 
| child 67399 | eab6ce8368fa | 
| permissions | -rw-r--r-- | 
| 58199 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 1 | (* Author: Andreas Lochbihler, ETH Zürich | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 2 | Author: Florian Haftmann, TU Muenchen *) | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 3 | |
| 58881 | 4 | section \<open>Less common functions on lists\<close> | 
| 58199 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 5 | |
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 6 | theory More_List | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 7 | imports Main | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 8 | begin | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 9 | |
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 10 | definition strip_while :: "('a \<Rightarrow> bool) \<Rightarrow> 'a list \<Rightarrow> 'a list"
 | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 11 | where | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 12 | "strip_while P = rev \<circ> dropWhile P \<circ> rev" | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 13 | |
| 58295 | 14 | lemma strip_while_rev [simp]: | 
| 15 | "strip_while P (rev xs) = rev (dropWhile P xs)" | |
| 16 | by (simp add: strip_while_def) | |
| 17 | ||
| 58199 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 18 | lemma strip_while_Nil [simp]: | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 19 | "strip_while P [] = []" | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 20 | by (simp add: strip_while_def) | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 21 | |
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 22 | lemma strip_while_append [simp]: | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 23 | "\<not> P x \<Longrightarrow> strip_while P (xs @ [x]) = xs @ [x]" | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 24 | by (simp add: strip_while_def) | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 25 | |
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 26 | lemma strip_while_append_rec [simp]: | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 27 | "P x \<Longrightarrow> strip_while P (xs @ [x]) = strip_while P xs" | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 28 | by (simp add: strip_while_def) | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 29 | |
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 30 | lemma strip_while_Cons [simp]: | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 31 | "\<not> P x \<Longrightarrow> strip_while P (x # xs) = x # strip_while P xs" | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 32 | by (induct xs rule: rev_induct) (simp_all add: strip_while_def) | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 33 | |
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 34 | lemma strip_while_eq_Nil [simp]: | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 35 | "strip_while P xs = [] \<longleftrightarrow> (\<forall>x\<in>set xs. P x)" | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 36 | by (simp add: strip_while_def) | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 37 | |
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 38 | lemma strip_while_eq_Cons_rec: | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 39 | "strip_while P (x # xs) = x # strip_while P xs \<longleftrightarrow> \<not> (P x \<and> (\<forall>x\<in>set xs. P x))" | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 40 | by (induct xs rule: rev_induct) (simp_all add: strip_while_def) | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 41 | |
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 42 | lemma split_strip_while_append: | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 43 | fixes xs :: "'a list" | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 44 | obtains ys zs :: "'a list" | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 45 | where "strip_while P xs = ys" and "\<forall>x\<in>set zs. P x" and "xs = ys @ zs" | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 46 | proof (rule that) | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 47 | show "strip_while P xs = strip_while P xs" .. | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 48 | show "\<forall>x\<in>set (rev (takeWhile P (rev xs))). P x" by (simp add: takeWhile_eq_all_conv [symmetric]) | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 49 | have "rev xs = rev (strip_while P xs @ rev (takeWhile P (rev xs)))" | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 50 | by (simp add: strip_while_def) | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 51 | then show "xs = strip_while P xs @ rev (takeWhile P (rev xs))" | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 52 | by (simp only: rev_is_rev_conv) | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 53 | qed | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 54 | |
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 55 | lemma strip_while_snoc [simp]: | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 56 | "strip_while P (xs @ [x]) = (if P x then strip_while P xs else xs @ [x])" | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 57 | by (simp add: strip_while_def) | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 58 | |
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 59 | lemma strip_while_map: | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 60 | "strip_while P (map f xs) = map f (strip_while (P \<circ> f) xs)" | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 61 | by (simp add: strip_while_def rev_map dropWhile_map) | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 62 | |
| 65388 | 63 | lemma strip_while_dropWhile_commute: | 
| 64 | "strip_while P (dropWhile Q xs) = dropWhile Q (strip_while P xs)" | |
| 65 | proof (induct xs) | |
| 66 | case Nil | |
| 67 | then show ?case | |
| 68 | by simp | |
| 69 | next | |
| 70 | case (Cons x xs) | |
| 71 | show ?case | |
| 72 | proof (cases "\<forall>y\<in>set xs. P y") | |
| 73 | case True | |
| 74 | with dropWhile_append2 [of "rev xs"] show ?thesis | |
| 75 | by (auto simp add: strip_while_def dest: set_dropWhileD) | |
| 76 | next | |
| 77 | case False | |
| 78 | then obtain y where "y \<in> set xs" and "\<not> P y" | |
| 79 | by blast | |
| 80 | with Cons dropWhile_append3 [of P y "rev xs"] show ?thesis | |
| 81 | by (simp add: strip_while_def) | |
| 82 | qed | |
| 83 | qed | |
| 84 | ||
| 85 | lemma dropWhile_strip_while_commute: | |
| 86 | "dropWhile P (strip_while Q xs) = strip_while Q (dropWhile P xs)" | |
| 87 | by (simp add: strip_while_dropWhile_commute) | |
| 88 | ||
| 58295 | 89 | |
| 90 | definition no_leading :: "('a \<Rightarrow> bool) \<Rightarrow> 'a list \<Rightarrow> bool"
 | |
| 91 | where | |
| 92 | "no_leading P xs \<longleftrightarrow> (xs \<noteq> [] \<longrightarrow> \<not> P (hd xs))" | |
| 93 | ||
| 94 | lemma no_leading_Nil [simp, intro!]: | |
| 95 | "no_leading P []" | |
| 96 | by (simp add: no_leading_def) | |
| 97 | ||
| 98 | lemma no_leading_Cons [simp, intro!]: | |
| 99 | "no_leading P (x # xs) \<longleftrightarrow> \<not> P x" | |
| 100 | by (simp add: no_leading_def) | |
| 101 | ||
| 102 | lemma no_leading_append [simp]: | |
| 103 | "no_leading P (xs @ ys) \<longleftrightarrow> no_leading P xs \<and> (xs = [] \<longrightarrow> no_leading P ys)" | |
| 104 | by (induct xs) simp_all | |
| 105 | ||
| 106 | lemma no_leading_dropWhile [simp]: | |
| 107 | "no_leading P (dropWhile P xs)" | |
| 108 | by (induct xs) simp_all | |
| 109 | ||
| 110 | lemma dropWhile_eq_obtain_leading: | |
| 111 | assumes "dropWhile P xs = ys" | |
| 112 | obtains zs where "xs = zs @ ys" and "\<And>z. z \<in> set zs \<Longrightarrow> P z" and "no_leading P ys" | |
| 113 | proof - | |
| 114 | from assms have "\<exists>zs. xs = zs @ ys \<and> (\<forall>z \<in> set zs. P z) \<and> no_leading P ys" | |
| 115 | proof (induct xs arbitrary: ys) | |
| 116 | case Nil then show ?case by simp | |
| 117 | next | |
| 118 | case (Cons x xs ys) | |
| 119 | show ?case proof (cases "P x") | |
| 120 | case True with Cons.hyps [of ys] Cons.prems | |
| 121 | have "\<exists>zs. xs = zs @ ys \<and> (\<forall>a\<in>set zs. P a) \<and> no_leading P ys" | |
| 122 | by simp | |
| 123 | then obtain zs where "xs = zs @ ys" and "\<And>z. z \<in> set zs \<Longrightarrow> P z" | |
| 124 | and *: "no_leading P ys" | |
| 125 | by blast | |
| 126 | with True have "x # xs = (x # zs) @ ys" and "\<And>z. z \<in> set (x # zs) \<Longrightarrow> P z" | |
| 127 | by auto | |
| 128 | with * show ?thesis | |
| 129 | by blast next | |
| 130 | case False | |
| 131 | with Cons show ?thesis by (cases ys) simp_all | |
| 132 | qed | |
| 133 | qed | |
| 134 | with that show thesis | |
| 135 | by blast | |
| 136 | qed | |
| 137 | ||
| 138 | lemma dropWhile_idem_iff: | |
| 139 | "dropWhile P xs = xs \<longleftrightarrow> no_leading P xs" | |
| 140 | by (cases xs) (auto elim: dropWhile_eq_obtain_leading) | |
| 141 | ||
| 58199 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 142 | |
| 58295 | 143 | abbreviation no_trailing :: "('a \<Rightarrow> bool) \<Rightarrow> 'a list \<Rightarrow> bool"
 | 
| 144 | where | |
| 145 | "no_trailing P xs \<equiv> no_leading P (rev xs)" | |
| 146 | ||
| 147 | lemma no_trailing_unfold: | |
| 148 | "no_trailing P xs \<longleftrightarrow> (xs \<noteq> [] \<longrightarrow> \<not> P (last xs))" | |
| 149 | by (induct xs) simp_all | |
| 150 | ||
| 151 | lemma no_trailing_Nil [simp, intro!]: | |
| 152 | "no_trailing P []" | |
| 153 | by simp | |
| 154 | ||
| 155 | lemma no_trailing_Cons [simp]: | |
| 156 | "no_trailing P (x # xs) \<longleftrightarrow> no_trailing P xs \<and> (xs = [] \<longrightarrow> \<not> P x)" | |
| 157 | by simp | |
| 158 | ||
| 65388 | 159 | lemma no_trailing_append: | 
| 160 | "no_trailing P (xs @ ys) \<longleftrightarrow> no_trailing P ys \<and> (ys = [] \<longrightarrow> no_trailing P xs)" | |
| 161 | by (induct xs) simp_all | |
| 162 | ||
| 58295 | 163 | lemma no_trailing_append_Cons [simp]: | 
| 164 | "no_trailing P (xs @ y # ys) \<longleftrightarrow> no_trailing P (y # ys)" | |
| 165 | by simp | |
| 166 | ||
| 167 | lemma no_trailing_strip_while [simp]: | |
| 168 | "no_trailing P (strip_while P xs)" | |
| 169 | by (induct xs rule: rev_induct) simp_all | |
| 170 | ||
| 65388 | 171 | lemma strip_while_idem [simp]: | 
| 172 | "no_trailing P xs \<Longrightarrow> strip_while P xs = xs" | |
| 173 | by (cases xs rule: rev_cases) simp_all | |
| 174 | ||
| 58295 | 175 | lemma strip_while_eq_obtain_trailing: | 
| 176 | assumes "strip_while P xs = ys" | |
| 177 | obtains zs where "xs = ys @ zs" and "\<And>z. z \<in> set zs \<Longrightarrow> P z" and "no_trailing P ys" | |
| 178 | proof - | |
| 179 | from assms have "rev (rev (dropWhile P (rev xs))) = rev ys" | |
| 180 | by (simp add: strip_while_def) | |
| 181 | then have "dropWhile P (rev xs) = rev ys" | |
| 182 | by simp | |
| 183 | then obtain zs where A: "rev xs = zs @ rev ys" and B: "\<And>z. z \<in> set zs \<Longrightarrow> P z" | |
| 184 | and C: "no_trailing P ys" | |
| 185 | using dropWhile_eq_obtain_leading by blast | |
| 186 | from A have "rev (rev xs) = rev (zs @ rev ys)" | |
| 187 | by simp | |
| 188 | then have "xs = ys @ rev zs" | |
| 189 | by simp | |
| 190 | moreover from B have "\<And>z. z \<in> set (rev zs) \<Longrightarrow> P z" | |
| 191 | by simp | |
| 192 | ultimately show thesis using that C by blast | |
| 193 | qed | |
| 194 | ||
| 195 | lemma strip_while_idem_iff: | |
| 196 | "strip_while P xs = xs \<longleftrightarrow> no_trailing P xs" | |
| 197 | proof - | |
| 63040 | 198 | define ys where "ys = rev xs" | 
| 58295 | 199 | moreover have "strip_while P (rev ys) = rev ys \<longleftrightarrow> no_trailing P (rev ys)" | 
| 200 | by (simp add: dropWhile_idem_iff) | |
| 201 | ultimately show ?thesis by simp | |
| 202 | qed | |
| 203 | ||
| 204 | lemma no_trailing_map: | |
| 65388 | 205 | "no_trailing P (map f xs) \<longleftrightarrow> no_trailing (P \<circ> f) xs" | 
| 58295 | 206 | by (simp add: last_map no_trailing_unfold) | 
| 207 | ||
| 65388 | 208 | lemma no_trailing_drop [simp]: | 
| 209 | "no_trailing P (drop n xs)" if "no_trailing P xs" | |
| 210 | proof - | |
| 211 | from that have "no_trailing P (take n xs @ drop n xs)" | |
| 212 | by simp | |
| 213 | then show ?thesis | |
| 214 | by (simp only: no_trailing_append) | |
| 215 | qed | |
| 216 | ||
| 58295 | 217 | lemma no_trailing_upt [simp]: | 
| 218 | "no_trailing P [n..<m] \<longleftrightarrow> (n < m \<longrightarrow> \<not> P (m - 1))" | |
| 219 | by (auto simp add: no_trailing_unfold) | |
| 58199 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 220 | |
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 221 | |
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 222 | definition nth_default :: "'a \<Rightarrow> 'a list \<Rightarrow> nat \<Rightarrow> 'a" | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 223 | where | 
| 58437 | 224 | "nth_default dflt xs n = (if n < length xs then xs ! n else dflt)" | 
| 58199 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 225 | |
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 226 | lemma nth_default_nth: | 
| 58437 | 227 | "n < length xs \<Longrightarrow> nth_default dflt xs n = xs ! n" | 
| 58199 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 228 | by (simp add: nth_default_def) | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 229 | |
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 230 | lemma nth_default_beyond: | 
| 58437 | 231 | "length xs \<le> n \<Longrightarrow> nth_default dflt xs n = dflt" | 
| 232 | by (simp add: nth_default_def) | |
| 233 | ||
| 234 | lemma nth_default_Nil [simp]: | |
| 235 | "nth_default dflt [] n = dflt" | |
| 236 | by (simp add: nth_default_def) | |
| 237 | ||
| 238 | lemma nth_default_Cons: | |
| 239 | "nth_default dflt (x # xs) n = (case n of 0 \<Rightarrow> x | Suc n' \<Rightarrow> nth_default dflt xs n')" | |
| 240 | by (simp add: nth_default_def split: nat.split) | |
| 241 | ||
| 242 | lemma nth_default_Cons_0 [simp]: | |
| 243 | "nth_default dflt (x # xs) 0 = x" | |
| 244 | by (simp add: nth_default_Cons) | |
| 245 | ||
| 246 | lemma nth_default_Cons_Suc [simp]: | |
| 247 | "nth_default dflt (x # xs) (Suc n) = nth_default dflt xs n" | |
| 248 | by (simp add: nth_default_Cons) | |
| 249 | ||
| 250 | lemma nth_default_replicate_dflt [simp]: | |
| 251 | "nth_default dflt (replicate n dflt) m = dflt" | |
| 58199 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 252 | by (simp add: nth_default_def) | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 253 | |
| 58437 | 254 | lemma nth_default_append: | 
| 255 | "nth_default dflt (xs @ ys) n = | |
| 256 | (if n < length xs then nth xs n else nth_default dflt ys (n - length xs))" | |
| 257 | by (auto simp add: nth_default_def nth_append) | |
| 258 | ||
| 259 | lemma nth_default_append_trailing [simp]: | |
| 260 | "nth_default dflt (xs @ replicate n dflt) = nth_default dflt xs" | |
| 261 | by (simp add: fun_eq_iff nth_default_append) (simp add: nth_default_def) | |
| 262 | ||
| 263 | lemma nth_default_snoc_default [simp]: | |
| 264 | "nth_default dflt (xs @ [dflt]) = nth_default dflt xs" | |
| 265 | by (auto simp add: nth_default_def fun_eq_iff nth_append) | |
| 266 | ||
| 267 | lemma nth_default_eq_dflt_iff: | |
| 268 | "nth_default dflt xs k = dflt \<longleftrightarrow> (k < length xs \<longrightarrow> xs ! k = dflt)" | |
| 269 | by (simp add: nth_default_def) | |
| 270 | ||
| 271 | lemma in_enumerate_iff_nth_default_eq: | |
| 272 | "x \<noteq> dflt \<Longrightarrow> (n, x) \<in> set (enumerate 0 xs) \<longleftrightarrow> nth_default dflt xs n = x" | |
| 273 | by (auto simp add: nth_default_def in_set_conv_nth enumerate_eq_zip) | |
| 274 | ||
| 275 | lemma last_conv_nth_default: | |
| 276 | assumes "xs \<noteq> []" | |
| 277 | shows "last xs = nth_default dflt xs (length xs - 1)" | |
| 278 | using assms by (simp add: nth_default_def last_conv_nth) | |
| 279 | ||
| 280 | lemma nth_default_map_eq: | |
| 281 | "f dflt' = dflt \<Longrightarrow> nth_default dflt (map f xs) n = f (nth_default dflt' xs n)" | |
| 282 | by (simp add: nth_default_def) | |
| 283 | ||
| 284 | lemma finite_nth_default_neq_default [simp]: | |
| 285 |   "finite {k. nth_default dflt xs k \<noteq> dflt}"
 | |
| 286 | by (simp add: nth_default_def) | |
| 287 | ||
| 288 | lemma sorted_list_of_set_nth_default: | |
| 289 |   "sorted_list_of_set {k. nth_default dflt xs k \<noteq> dflt} = map fst (filter (\<lambda>(_, x). x \<noteq> dflt) (enumerate 0 xs))"
 | |
| 290 | by (rule sorted_distinct_set_unique) (auto simp add: nth_default_def in_set_conv_nth | |
| 291 | sorted_filter distinct_map_filter enumerate_eq_zip intro: rev_image_eqI) | |
| 292 | ||
| 293 | lemma map_nth_default: | |
| 294 | "map (nth_default x xs) [0..<length xs] = xs" | |
| 295 | proof - | |
| 296 | have *: "map (nth_default x xs) [0..<length xs] = map (List.nth xs) [0..<length xs]" | |
| 297 | by (rule map_cong) (simp_all add: nth_default_nth) | |
| 298 | show ?thesis by (simp add: * map_nth) | |
| 299 | qed | |
| 300 | ||
| 58199 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 301 | lemma range_nth_default [simp]: | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 302 | "range (nth_default dflt xs) = insert dflt (set xs)" | 
| 58437 | 303 | by (auto simp add: nth_default_def [abs_def] in_set_conv_nth) | 
| 58199 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 304 | |
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 305 | lemma nth_strip_while: | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 306 | assumes "n < length (strip_while P xs)" | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 307 | shows "strip_while P xs ! n = xs ! n" | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 308 | proof - | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 309 | have "length (dropWhile P (rev xs)) + length (takeWhile P (rev xs)) = length xs" | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 310 | by (subst add.commute) | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 311 | (simp add: arg_cong [where f=length, OF takeWhile_dropWhile_id, unfolded length_append]) | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 312 | then show ?thesis using assms | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 313 | by (simp add: strip_while_def rev_nth dropWhile_nth) | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 314 | qed | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 315 | |
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 316 | lemma length_strip_while_le: | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 317 | "length (strip_while P xs) \<le> length xs" | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 318 | unfolding strip_while_def o_def length_rev | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 319 | by (subst (2) length_rev[symmetric]) | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 320 | (simp add: strip_while_def length_dropWhile_le del: length_rev) | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 321 | |
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 322 | lemma nth_default_strip_while_dflt [simp]: | 
| 58437 | 323 | "nth_default dflt (strip_while (op = dflt) xs) = nth_default dflt xs" | 
| 58199 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 324 | by (induct xs rule: rev_induct) auto | 
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 325 | |
| 58437 | 326 | lemma nth_default_eq_iff: | 
| 327 | "nth_default dflt xs = nth_default dflt ys | |
| 328 | \<longleftrightarrow> strip_while (HOL.eq dflt) xs = strip_while (HOL.eq dflt) ys" (is "?P \<longleftrightarrow> ?Q") | |
| 329 | proof | |
| 330 | let ?xs = "strip_while (HOL.eq dflt) xs" and ?ys = "strip_while (HOL.eq dflt) ys" | |
| 331 | assume ?P | |
| 332 | then have eq: "nth_default dflt ?xs = nth_default dflt ?ys" | |
| 333 | by simp | |
| 334 | have len: "length ?xs = length ?ys" | |
| 335 | proof (rule ccontr) | |
| 336 | assume len: "length ?xs \<noteq> length ?ys" | |
| 337 |     { fix xs ys :: "'a list"
 | |
| 338 | let ?xs = "strip_while (HOL.eq dflt) xs" and ?ys = "strip_while (HOL.eq dflt) ys" | |
| 339 | assume eq: "nth_default dflt ?xs = nth_default dflt ?ys" | |
| 340 | assume len: "length ?xs < length ?ys" | |
| 341 | then have "length ?ys > 0" by arith | |
| 342 | then have "?ys \<noteq> []" by simp | |
| 343 | with last_conv_nth_default [of ?ys dflt] | |
| 344 | have "last ?ys = nth_default dflt ?ys (length ?ys - 1)" | |
| 345 | by auto | |
| 60500 | 346 | moreover from \<open>?ys \<noteq> []\<close> no_trailing_strip_while [of "HOL.eq dflt" ys] | 
| 58437 | 347 | have "last ?ys \<noteq> dflt" by (simp add: no_trailing_unfold) | 
| 348 | ultimately have "nth_default dflt ?xs (length ?ys - 1) \<noteq> dflt" | |
| 349 | using eq by simp | |
| 350 | moreover from len have "length ?ys - 1 \<ge> length ?xs" by simp | |
| 351 | ultimately have False by (simp only: nth_default_beyond) simp | |
| 352 | } | |
| 353 | from this [of xs ys] this [of ys xs] len eq show False | |
| 354 | by (auto simp only: linorder_class.neq_iff) | |
| 355 | qed | |
| 356 | then show ?Q | |
| 357 | proof (rule nth_equalityI [rule_format]) | |
| 358 | fix n | |
| 63540 | 359 | assume n: "n < length ?xs" | 
| 360 | with len have "n < length ?ys" | |
| 58437 | 361 | by simp | 
| 63540 | 362 | with n have xs: "nth_default dflt ?xs n = ?xs ! n" | 
| 58437 | 363 | and ys: "nth_default dflt ?ys n = ?ys ! n" | 
| 364 | by (simp_all only: nth_default_nth) | |
| 365 | with eq show "?xs ! n = ?ys ! n" | |
| 366 | by simp | |
| 367 | qed | |
| 368 | next | |
| 369 | assume ?Q | |
| 370 | then have "nth_default dflt (strip_while (HOL.eq dflt) xs) = nth_default dflt (strip_while (HOL.eq dflt) ys)" | |
| 371 | by simp | |
| 372 | then show ?P | |
| 373 | by simp | |
| 374 | qed | |
| 58199 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 375 | |
| 
5fbe474b5da8
explicit theory with additional, less commonly used list operations
 haftmann parents: diff
changeset | 376 | end | 
| 58295 | 377 |