diff -r 181bd2050cf4 -r 0493188cff42 src/ZF/Integ/IntDiv.ML --- a/src/ZF/Integ/IntDiv.ML Mon Oct 22 12:01:35 2001 +0200 +++ b/src/ZF/Integ/IntDiv.ML Mon Oct 22 12:11:00 2001 +0200 @@ -333,9 +333,9 @@ (*** Correctness of posDivAlg, the division algorithm for a>=0 and b>0 ***) -Goal "adjust(a, b, ) = (let diff = r$-b in \ +Goal "adjust(b, ) = (let diff = r$-b in \ \ if #0 $<= diff then <#2$*q $+ #1,diff> \ -\ else <#2$*q,r>)"; +\ else <#2$*q,r>)"; by (simp_tac (simpset() addsimps [Let_def,adjust_def]) 1); qed "adjust_eq"; Addsimps [adjust_eq]; @@ -352,7 +352,7 @@ Goal "[| #0 $< b; a \\ int; b \\ int |] ==> \ \ posDivAlg() = \ -\ (if a$ else adjust(a, b, posDivAlg ()))"; +\ (if a$ else adjust(b, posDivAlg ()))"; by (rtac (posDivAlg_unfold RS trans) 1); by (asm_simp_tac (simpset() addsimps [not_zless_iff_zle RS iff_sym]) 1); by (asm_simp_tac (simpset() addsimps [vimage_iff, posDivAlg_termination]) 1); @@ -513,7 +513,7 @@ Goal "[| #0 $< b; a \\ int; b \\ int |] ==> \ \ negDivAlg() = \ \ (if #0 $<= a$+b then <#-1,a$+b> \ -\ else adjust(a, b, negDivAlg ()))"; +\ else adjust(b, negDivAlg ()))"; by (rtac (negDivAlg_unfold RS trans) 1); by (asm_simp_tac (simpset() addsimps [not_zless_iff_zle RS iff_sym]) 1); by (asm_simp_tac (simpset() addsimps [not_zle_iff_zless, vimage_iff,