src/HOL/Integ/IntDiv.thy
changeset 13601 fd3e3d6b37b2
parent 13524 604d0f3622d6
child 13716 73de0ef7cb25
--- a/src/HOL/Integ/IntDiv.thy	Mon Sep 30 16:12:16 2002 +0200
+++ b/src/HOL/Integ/IntDiv.thy	Mon Sep 30 16:14:02 2002 +0200
@@ -365,10 +365,10 @@
 
 lemma self_quotient: "[| quorem((a,a),(q,r));  a ~= (0::int) |] ==> q = 1"
 apply (simp add: split_ifs quorem_def linorder_neq_iff)
-apply (rule order_antisym, auto)
+apply (rule order_antisym, safe, simp_all (no_asm_use))
 apply (rule_tac [3] a = "-a" and r = "-r" in self_quotient_aux1)
 apply (rule_tac a = "-a" and r = "-r" in self_quotient_aux2)
-apply (force intro: self_quotient_aux1 self_quotient_aux2 simp add: zadd_commute zmult_zminus)+
+apply (force intro: self_quotient_aux1 self_quotient_aux2 simp only: zadd_commute zmult_zminus)+
 done
 
 lemma self_remainder: "[| quorem((a,a),(q,r));  a ~= (0::int) |] ==> r = 0"