src/ZF/ex/Primes.ML
changeset 9491 1a36151ee2fc
parent 5147 825877190618
child 11316 b4e71bd751e4
--- a/src/ZF/ex/Primes.ML	Tue Aug 01 13:43:22 2000 +0200
+++ b/src/ZF/ex/Primes.ML	Tue Aug 01 15:28:21 2000 +0200
@@ -8,8 +8,6 @@
 
 eta_contract:=false;
 
-open Primes;
-
 (************************************************)
 (** Divides Relation                           **)
 (************************************************)
@@ -125,10 +123,9 @@
 (* if f divides a and b then f divides egcd(a,b) *)
 
 Goalw [dvd_def] "[| f dvd a; f dvd b; 0<b |] ==> f dvd (a mod b)";
-by (safe_tac (claset() addSIs [mult_type, mod_type]));
+by (safe_tac (claset() addSIs [mod_type]));
 ren "m n" 1;
-by (rtac (zero_lt_mult_iff RS iffD1 RS conjE) 1);
-by (REPEAT_SOME assume_tac);
+by (Asm_full_simp_tac 1);
 by (res_inst_tac 
     [("x", "(((m div n)#*n #+ m mod n) #- ((f#*m) div (f#*n)) #* n)")] 
     bexI 1);