src/HOL/IOA/IOA.ML
changeset 3842 b55686a7b22c
parent 3346 5101517c2614
child 3919 c036caebfc75
--- a/src/HOL/IOA/IOA.ML	Fri Oct 10 18:37:49 1997 +0200
+++ b/src/HOL/IOA/IOA.ML	Fri Oct 10 19:02:28 1997 +0200
@@ -47,7 +47,7 @@
 qed "mk_trace_thm";
 
 goalw IOA.thy [reachable_def] "!!A. s:starts_of(A) ==> reachable A s";
-  by (res_inst_tac [("x","(%i.None,%i.s)")] bexI 1);
+  by (res_inst_tac [("x","(%i. None,%i. s)")] bexI 1);
   by (Simp_tac 1);
   by (asm_simp_tac (!simpset addsimps exec_rws) 1);
 qed "reachable_0";
@@ -56,9 +56,9 @@
 "!!A. [| reachable A s; (s,a,t) : trans_of(A) |] ==> reachable A t";
   by (asm_full_simp_tac (!simpset delsimps bex_simps) 1);
   by (safe_tac (!claset));
-  by (res_inst_tac [("x","(%i.if i<n then fst ex i                    \
+  by (res_inst_tac [("x","(%i. if i<n then fst ex i                    \
 \                            else (if i=n then Some a else None),    \
-\                         %i.if i<Suc n then snd ex i else t)")] bexI 1);
+\                         %i. if i<Suc n then snd ex i else t)")] bexI 1);
   by (res_inst_tac [("x","Suc(n)")] exI 1);
   by (Simp_tac 1);
   by (Asm_simp_tac 1);