src/HOL/MicroJava/BV/BVExample.thy
changeset 47399 b72fa7bf9a10
parent 45990 b7b905b23b2a
child 51272 9c8d63b4b6be
--- a/src/HOL/MicroJava/BV/BVExample.thy	Fri Apr 06 19:18:00 2012 +0200
+++ b/src/HOL/MicroJava/BV/BVExample.thy	Fri Apr 06 19:23:51 2012 +0200
@@ -408,7 +408,7 @@
 
 lemma [code]:
   "unstables r step ss = 
-   foldr (\<lambda>p A. if \<not>stable r step ss p then insert p A else A) [0..<size ss] {}"
+   fold (\<lambda>p A. if \<not>stable r step ss p then insert p A else A) [0..<size ss] {}"
 proof -
   have "unstables r step ss = (UN p:{..<size ss}. if \<not>stable r step ss p then {p} else {})"
     apply (unfold unstables_def)
@@ -425,7 +425,7 @@
     apply simp+
     done
   also have "\<And>f. (UN p:{..<size ss}. f p) = Union (set (map f [0..<size ss]))" by auto
-  also note Sup_set_foldr also note foldr_map
+  also note Sup_set_fold also note fold_map
   also have "op \<union> \<circ> (\<lambda>p. if \<not> stable r step ss p then {p} else {}) = 
             (\<lambda>p A. if \<not>stable r step ss p then insert p A else A)"
     by(auto simp add: fun_eq_iff)
@@ -486,3 +486,4 @@
 *}
 
 end
+