fix code equation for RBT_Impl.fold
authorAndreas Lochbihler
Wed, 10 Oct 2012 16:18:27 +0200
changeset 49810 53f14f62cca2
parent 49809 39db47ed6d54
child 49811 3fc6b3289c31
fix code equation for RBT_Impl.fold
src/HOL/Library/RBT_Impl.thy
--- a/src/HOL/Library/RBT_Impl.thy	Wed Oct 10 15:17:18 2012 +0200
+++ b/src/HOL/Library/RBT_Impl.thy	Wed Oct 10 16:18:27 2012 +0200
@@ -1076,8 +1076,8 @@
   by (simp_all add: fold_def fun_eq_iff)
 
 lemma fold_code [code]:
-  "fold f Empty c = c"
-  "fold f (Branch c lt k v rt) c = fold f rt (f k v (fold f lt c))"
+  "fold f Empty x = x"
+  "fold f (Branch c lt k v rt) x = fold f rt (f k v (fold f lt x))"
 by(simp_all)
 
 (* fold with continuation predicate *)