src/HOL/Old_Number_Theory/Chinese.thy
changeset 57514 bdc2c6b40bf2
parent 57492 74bf65a1910a
child 58889 5b7a9633cfa8
equal deleted inserted replaced
57513:55b2afc5ddfc 57514:bdc2c6b40bf2
   236         apply (tactic {* stac (@{thm zcong_zmod} RS sym) 6 *})
   236         apply (tactic {* stac (@{thm zcong_zmod} RS sym) 6 *})
   237         apply (subgoal_tac [6]
   237         apply (subgoal_tac [6]
   238           "0 \<le> xilin_sol i n kf bf mf \<and> xilin_sol i n kf bf mf < mf i
   238           "0 \<le> xilin_sol i n kf bf mf \<and> xilin_sol i n kf bf mf < mf i
   239           \<and> [kf i * mhf mf n i * xilin_sol i n kf bf mf = bf i] (mod mf i)")
   239           \<and> [kf i * mhf mf n i * xilin_sol i n kf bf mf = bf i] (mod mf i)")
   240          prefer 6
   240          prefer 6
   241          apply (simp add: mult_ac)
   241          apply (simp add: ac_simps)
   242         apply (unfold xilin_sol_def)
   242         apply (unfold xilin_sol_def)
   243         apply (tactic {* asm_simp_tac @{context} 6 *})
   243         apply (tactic {* asm_simp_tac @{context} 6 *})
   244         apply (rule_tac [6] ex1_implies_ex [THEN someI_ex])
   244         apply (rule_tac [6] ex1_implies_ex [THEN someI_ex])
   245         apply (rule_tac [6] unique_xi_sol)
   245         apply (rule_tac [6] unique_xi_sol)
   246            apply (rule_tac [3] funprod_zdvd)
   246            apply (rule_tac [3] funprod_zdvd)