src/ZF/Integ/IntDiv.thy
changeset 13612 55d32e76ef4e
parent 13560 d9651081578b
child 13615 449a70d88b38
equal deleted inserted replaced
13611:2edf034c902a 13612:55d32e76ef4e
   227  prefer 2
   227  prefer 2
   228  apply (subst int_succ_int_1)
   228  apply (subst int_succ_int_1)
   229  apply (erule natE)
   229  apply (erule natE)
   230 apply (simp_all add: zadd_zmult_distrib zadd_zless_mono zle_def)
   230 apply (simp_all add: zadd_zmult_distrib zadd_zless_mono zle_def)
   231 apply (frule nat_0_le)
   231 apply (frule nat_0_le)
   232 apply (erule (1) notE impE)
       
   233 apply (subgoal_tac "i $+ (i $+ $# xa $* i) $< j $+ (j $+ $# xa $* j) ")
   232 apply (subgoal_tac "i $+ (i $+ $# xa $* i) $< j $+ (j $+ $# xa $* j) ")
   234 apply (simp (no_asm_use))
   233 apply (simp (no_asm_use))
   235 apply (rule zadd_zless_mono)
   234 apply (rule zadd_zless_mono)
   236 apply (simp_all (no_asm_simp) add: zle_def)
   235 apply (simp_all (no_asm_simp) add: zle_def)
   237 done
   236 done
   390          q \<in> int; q' \<in> int;  
   389          q \<in> int; q' \<in> int;  
   391          r \<in> int; r' \<in> int |] ==> r = r'"
   390          r \<in> int; r' \<in> int |] ==> r = r'"
   392 apply (subgoal_tac "q = q'")
   391 apply (subgoal_tac "q = q'")
   393  prefer 2 apply (blast intro: unique_quotient)
   392  prefer 2 apply (blast intro: unique_quotient)
   394 apply (simp add: quorem_def)
   393 apply (simp add: quorem_def)
   395 apply auto
       
   396 done
   394 done
   397 
   395 
   398 
   396 
   399 subsection{*Correctness of posDivAlg, 
   397 subsection{*Correctness of posDivAlg, 
   400            the Division Algorithm for @{text "a\<ge>0"} and @{text "b>0"} *}
   398            the Division Algorithm for @{text "a\<ge>0"} and @{text "b>0"} *}