# HG changeset patch # User nipkow # Date 1504795300 -7200 # Node ID c375b64a6c24926ff9379223c94413abd7763f60 # Parent 98b7ba7b1e9a026ce0884b3b6077da8360be2904 adapted to better linear arith diff -r 98b7ba7b1e9a -r c375b64a6c24 src/HOL/Analysis/Complex_Transcendental.thy --- a/src/HOL/Analysis/Complex_Transcendental.thy Thu Sep 07 15:12:40 2017 +0200 +++ b/src/HOL/Analysis/Complex_Transcendental.thy Thu Sep 07 16:41:40 2017 +0200 @@ -752,7 +752,7 @@ lemma e_approx_32: "\exp(1) - 5837465777 / 2147483648\ \ (inverse(2 ^ 32)::real)" using Taylor_exp [of 1 14] exp_le apply (simp add: sum_distrib_right in_Reals_norm Re_exp atMost_nat_numeral fact_numeral) - apply (simp only: pos_le_divide_eq [symmetric], linarith) + apply (simp only: pos_le_divide_eq [symmetric]) done lemma e_less_272: "exp 1 < (272/100::real)"