src/HOL/IMP/Procs_Stat_Vars_Stat.thy
changeset 51019 146f63c3f024
parent 47818 151d137f1095
child 52046 bc01725d7918
--- a/src/HOL/IMP/Procs_Stat_Vars_Stat.thy	Sun Feb 03 17:31:33 2013 +0100
+++ b/src/HOL/IMP/Procs_Stat_Vars_Stat.thy	Mon Feb 04 09:06:20 2013 +0100
@@ -32,7 +32,7 @@
    e \<turnstile> (WHILE b DO c, s\<^isub>1) \<Rightarrow> s\<^isub>3" |
 
 Var: "(pe,ve(x:=f),f+1) \<turnstile> (c,s) \<Rightarrow> t  \<Longrightarrow>
-      (pe,ve,f) \<turnstile> ({VAR x;; c}, s) \<Rightarrow> t(f := s f)" |
+      (pe,ve,f) \<turnstile> ({VAR x;; c}, s) \<Rightarrow> t" |
 
 Call1: "((p,c,ve)#pe,ve,f) \<turnstile> (c, s) \<Rightarrow> t  \<Longrightarrow>
         ((p,c,ve)#pe,ve',f) \<turnstile> (CALL p, s) \<Rightarrow> t" |
@@ -45,10 +45,8 @@
 code_pred big_step .
 
 
-values "{map t [0,1] |t. ([], <>, 0) \<turnstile> (CALL ''p'', nth [42, 43]) \<Rightarrow> t}"
-
-values "{map t [0, 1, 2] |t.
-  ([], <''x'' := 0, ''y'' := 1,''z'' := 2>, 0)
+values "{map t [10,11] |t.
+  ([], <''x'' := 10, ''y'' := 11>, 12)
   \<turnstile> (test_com, <>) \<Rightarrow> t}"
 
 end