src/HOL/HoareParallel/RG_Examples.thy
changeset 13187 e5434b822a96
parent 13103 66659a4b16f6
child 13517 42efec18f5b2
--- a/src/HOL/HoareParallel/RG_Examples.thy	Thu May 30 10:12:11 2002 +0200
+++ b/src/HOL/HoareParallel/RG_Examples.thy	Thu May 30 10:12:52 2002 +0200
@@ -147,7 +147,10 @@
     apply simp
    apply clarify
    apply simp
-   apply(case_tac j,simp,simp)
+   apply(subgoal_tac "j=0")
+    apply (rotate_tac -1)
+    apply simp
+   apply arith
   apply clarify
   apply(case_tac i,simp,simp)
  apply clarify   
@@ -324,7 +327,7 @@
     apply force
    apply(rule Basic)
       apply force
-     apply force
+     apply fastsimp
     apply force
    apply force
   apply(rule Basic)
@@ -340,7 +343,7 @@
      apply(erule_tac x=j in allE)
      apply force
     apply clarsimp
-    apply force
+    apply fastsimp
 apply force+
 done
 
@@ -399,4 +402,4 @@
 apply force+
 done
 
-end
\ No newline at end of file
+end