src/HOL/Library/Array.thy
changeset 27656 d4f6e64ee7cc
parent 27596 bc47d30747e6
child 27673 52056ddac194
--- a/src/HOL/Library/Array.thy	Sat Jul 19 11:05:18 2008 +0200
+++ b/src/HOL/Library/Array.thy	Sat Jul 19 19:27:13 2008 +0200
@@ -93,7 +93,16 @@
      mapM (nth a) [0..<n]
    done)"
 
-hide (open) const new -- {* avoid clashed with some popular names *}
+definition
+   map :: "('a\<Colon>heap \<Rightarrow> 'a) \<Rightarrow> 'a array \<Rightarrow> 'a array Heap"
+where
+  "map f a = (do
+     n \<leftarrow> length a;
+     mapM (\<lambda>n. map_entry n f a) [0..<n];
+     return a
+   done)"
+
+hide (open) const new map -- {* avoid clashed with some popular names *}
 
 
 subsection {* Properties *}