src/HOL/IMP/Small_Step.thy
changeset 44036 d03f9f28d01d
parent 43158 686fa0a0696e
child 45015 fdac1e9880eb
--- a/src/HOL/IMP/Small_Step.thy	Fri Aug 05 14:16:44 2011 +0200
+++ b/src/HOL/IMP/Small_Step.thy	Thu Aug 04 16:49:57 2011 +0200
@@ -27,7 +27,7 @@
 
 values "{(c',map t [''x'',''y'',''z'']) |c' t.
    (''x'' ::= V ''z''; ''y'' ::= V ''x'',
-    [''x'' \<rightarrow> 3, ''y'' \<rightarrow> 7, ''z'' \<rightarrow> 5]) \<rightarrow>* (c',t)}"
+    <''x'' := 3, ''y'' := 7, ''z'' := 5>) \<rightarrow>* (c',t)}"
 
 
 subsection{* Proof infrastructure *}