src/HOL/HoareParallel/OG_Examples.thy
changeset 25112 98824cc791c0
parent 24075 366d4d234814
child 27095 c1c27955d7dd
equal deleted inserted replaced
25111:d52a58b51f1f 25112:98824cc791c0
   437 apply(tactic {*ALLGOALS (conjI_Tac (K all_tac)) *})
   437 apply(tactic {*ALLGOALS (conjI_Tac (K all_tac)) *})
   438 --{* 930 subgoals left *}
   438 --{* 930 subgoals left *}
   439 apply(tactic {* ALLGOALS (clarify_tac @{claset}) *})
   439 apply(tactic {* ALLGOALS (clarify_tac @{claset}) *})
   440 apply(simp_all (asm_lr) only:length_0_conv [THEN sym])
   440 apply(simp_all (asm_lr) only:length_0_conv [THEN sym])
   441 --{* 44 subgoals left *}
   441 --{* 44 subgoals left *}
   442 apply (simp_all (asm_lr) del:length_0_conv add: nth_list_update mod_less_divisor mod_lemma)
   442 apply (simp_all (asm_lr) del:length_0_conv add: neq0_conv nth_list_update mod_less_divisor mod_lemma)
   443 --{* 32 subgoals left *}
   443 --{* 32 subgoals left *}
   444 apply(tactic {* ALLGOALS (clarify_tac @{claset}) *})
   444 apply(tactic {* ALLGOALS (clarify_tac @{claset}) *})
   445 
   445 
   446 apply(tactic {* TRYALL (simple_arith_tac @{context}) *})
   446 apply(tactic {* TRYALL (simple_arith_tac @{context}) *})
   447 --{* 9 subgoals left *}
   447 --{* 9 subgoals left *}