diff -r fcfb4aa8e6e6 -r 933f35c4e126 src/HOL/Fact.thy --- a/src/HOL/Fact.thy Tue Jan 17 11:15:36 2012 +0100 +++ b/src/HOL/Fact.thy Tue Jan 17 16:30:54 2012 +0100 @@ -255,8 +255,6 @@ fact m < fact ((m + 1) + k)" apply (induct k rule: int_ge_induct) apply (simp add: fact_plus_one_int) - apply (subst mult_less_cancel_right1) - apply (insert fact_gt_zero_int [of m], arith) apply (subst (2) fact_reduce_int) apply (auto simp add: add_ac) apply (erule order_less_le_trans)