src/HOL/IMP/BExp.thy
changeset 44036 d03f9f28d01d
parent 43158 686fa0a0696e
child 45015 fdac1e9880eb
--- a/src/HOL/IMP/BExp.thy	Fri Aug 05 14:16:44 2011 +0200
+++ b/src/HOL/IMP/BExp.thy	Thu Aug 04 16:49:57 2011 +0200
@@ -11,7 +11,7 @@
 "bval (Less a1 a2) s = (aval a1 s < aval a2 s)"
 
 value "bval (Less (V ''x'') (Plus (N 3) (V ''y'')))
-            [''x'' \<rightarrow> 3, ''y'' \<rightarrow> 1]"
+            <''x'' := 3, ''y'' := 1>"
 
 
 subsection "Optimization"