diff -r b4c3af8ebada -r b115460e5c50 src/ZF/Integ/IntDiv.ML --- a/src/ZF/Integ/IntDiv.ML Thu Dec 07 22:35:25 2000 +0100 +++ b/src/ZF/Integ/IntDiv.ML Fri Dec 08 00:04:34 2000 +0100 @@ -383,8 +383,8 @@ Addsimps [adjust_eq]; -Goal "\\#0 $< b; \\ a $< b\\ \ -\ \\ nat_of(a $- #2 $\\ b $+ #1) < nat_of(a $- b $+ #1)"; +Goal "[| #0 $< b; \\ a $< b |] \ +\ ==> nat_of(a $- #2 $\\ b $+ #1) < nat_of(a $- b $+ #1)"; by (simp_tac (simpset() addsimps [zless_nat_conj]) 1); by (asm_full_simp_tac (simpset() addsimps [not_zless_iff_zle, zless_add1_iff_zle]@zcompare_rls) 1); @@ -404,7 +404,7 @@ Goal "[| !!a b. [| a: int; b: int; \ \ ~ (a $< b | b $<= #0) --> P() |] \ \ ==> P() |] \ -\ ==> : int*int \\ P()"; +\ ==> : int*int --> P()"; by (res_inst_tac [("a","")] wf_induct 1); by (res_inst_tac [("A","int*int"), ("f","%.nat_of (a $- b $+ #1)")] wf_measure 1);