reverted half-baken 7d1127ac2251
authorhaftmann
Sat, 14 Nov 2015 08:45:51 +0100
changeset 61668 9a51e4dfc5d9
parent 61667 4b53042d7a40
child 61669 27ca6147e3b3
reverted half-baken 7d1127ac2251
src/HOL/List.thy
--- a/src/HOL/List.thy	Sat Nov 14 08:45:51 2015 +0100
+++ b/src/HOL/List.thy	Sat Nov 14 08:45:51 2015 +0100
@@ -6408,15 +6408,6 @@
   "map f (filter P xs) = map_filter (\<lambda>x. if P x then Some (f x) else None) xs"
   by (simp add: map_filter_def)
 
-definition map_range :: "(nat \<Rightarrow> 'a) \<Rightarrow> nat \<Rightarrow> 'a list"
-where
-  [code_abbrev]: "map_range f n = map f [0..<n]"
-
-lemma map_range_simps [simp, code]:
-  "map_range f 0 = []"
-  "map_range f (Suc n) = map_range f n @ [f n]"
-  by (simp_all add: map_range_def)
-
 text \<open>Optimized code for @{text"\<forall>i\<in>{a..b::int}"} and @{text"\<forall>n:{a..<b::nat}"}
 and similiarly for @{text"\<exists>"}.\<close>