src/HOL/HoareParallel/RG_Examples.thy
changeset 13187 e5434b822a96
parent 13103 66659a4b16f6
child 13517 42efec18f5b2
equal deleted inserted replaced
13186:ef8ed6adcb38 13187:e5434b822a96
   145    apply(erule disjE)
   145    apply(erule disjE)
   146     apply clarify
   146     apply clarify
   147     apply simp
   147     apply simp
   148    apply clarify
   148    apply clarify
   149    apply simp
   149    apply simp
   150    apply(case_tac j,simp,simp)
   150    apply(subgoal_tac "j=0")
       
   151     apply (rotate_tac -1)
       
   152     apply simp
       
   153    apply arith
   151   apply clarify
   154   apply clarify
   152   apply(case_tac i,simp,simp)
   155   apply(case_tac i,simp,simp)
   153  apply clarify   
   156  apply clarify   
   154  apply simp
   157  apply simp
   155  apply(erule_tac x=0 in all_dupE)
   158  apply(erule_tac x=0 in all_dupE)
   322     apply(rule subset_refl)+
   325     apply(rule subset_refl)+
   323  apply(rule Cond)
   326  apply(rule Cond)
   324     apply force
   327     apply force
   325    apply(rule Basic)
   328    apply(rule Basic)
   326       apply force
   329       apply force
   327      apply force
   330      apply fastsimp
   328     apply force
   331     apply force
   329    apply force
   332    apply force
   330   apply(rule Basic)
   333   apply(rule Basic)
   331      apply simp
   334      apply simp
   332      apply clarify
   335      apply clarify
   338         apply assumption+
   341         apply assumption+
   339        apply simp+
   342        apply simp+
   340      apply(erule_tac x=j in allE)
   343      apply(erule_tac x=j in allE)
   341      apply force
   344      apply force
   342     apply clarsimp
   345     apply clarsimp
   343     apply force
   346     apply fastsimp
   344 apply force+
   347 apply force+
   345 done
   348 done
   346 
   349 
   347 text {* Same but with a list as auxiliary variable: *}
   350 text {* Same but with a list as auxiliary variable: *}
   348 
   351