src/HOL/HoareParallel/RG_Tran.thy
changeset 15425 6356d2523f73
parent 15236 f289e8ba2bb3
child 23746 a455e69c31cc
--- a/src/HOL/HoareParallel/RG_Tran.thy	Mon Dec 20 18:25:22 2004 +0100
+++ b/src/HOL/HoareParallel/RG_Tran.thy	Wed Dec 22 11:36:33 2004 +0100
@@ -1,6 +1,8 @@
 header {* \section{Operational Semantics} *}
 
-theory RG_Tran = RG_Com:
+theory RG_Tran
+imports RG_Com
+begin
 
 subsection {* Semantics of Component Programs *}
 
@@ -770,7 +772,7 @@
   (\<forall>i<length xs. (xs!i,s)#(clist!i) \<in> cptn))"
 apply(induct ys)
  apply(clarify)
- apply(rule_tac x="map (\<lambda>i. []) [0..length xs(]" in exI)
+ apply(rule_tac x="map (\<lambda>i. []) [0..<length xs]" in exI)
  apply(simp add: conjoin_def same_length_def same_state_def same_program_def compat_label_def)
  apply(rule conjI)
   apply(rule nth_equalityI,simp,simp)
@@ -781,7 +783,7 @@
  apply(erule_tac x="xs" in allE)
  apply(erule_tac x="t" in allE,simp)
  apply clarify
- apply(rule_tac x="(map (\<lambda>j. (P!j, t)#(clist!j)) [0..length P(])" in exI,simp)
+ apply(rule_tac x="(map (\<lambda>j. (P!j, t)#(clist!j)) [0..<length P])" in exI,simp)
  apply(rule conjI)
   prefer 2
   apply clarify
@@ -813,7 +815,7 @@
 apply(erule_tac x="Ps[i:=r]" in allE)
 apply(erule_tac x="ta" in allE,simp)
 apply clarify
-apply(rule_tac x="(map (\<lambda>j. (Ps!j, ta)#(clist!j)) [0..length Ps(]) [i:=((r, ta)#(clist!i))]" in exI,simp)
+apply(rule_tac x="(map (\<lambda>j. (Ps!j, ta)#(clist!j)) [0..<length Ps]) [i:=((r, ta)#(clist!i))]" in exI,simp)
 apply(rule conjI)
  prefer 2
  apply clarify