diff -r 3f577308551e -r 293ede07b775 src/HOL/ex/Gauge_Integration.thy --- a/src/HOL/ex/Gauge_Integration.thy Tue Apr 26 22:39:17 2016 +0200 +++ b/src/HOL/ex/Gauge_Integration.thy Tue Apr 26 22:44:31 2016 +0200 @@ -133,7 +133,7 @@ proof (cases "b < x") case True with 2 obtain N where *: "N < length D" - and **: "\ d t e. D ! N = (d,t,e) \ d < x \ x \ e" by auto + and **: "D ! N = (d,t,e) \ d < x \ x \ e" for d t e by auto hence "Suc N < length ((a,t,b)#D) \ (\ d t' e. ((a,t,b)#D) ! Suc N = (d,t',e) \ d < x \ x \ e)" by auto thus ?thesis by auto @@ -372,11 +372,11 @@ hence "a < b" and "b < c" by auto obtain \1 where \1_gauge: "gauge {a..b} \1" - and I1: "\ D. fine \1 (a,b) D \ \ rsum D f - x1 \ < (\ / 2)" + and I1: "fine \1 (a,b) D \ \ rsum D f - x1 \ < (\ / 2)" for D using IntegralE [OF \Integral (a, b) f x1\ \0 < \/2\] by auto obtain \2 where \2_gauge: "gauge {b..c} \2" - and I2: "\ D. fine \2 (b,c) D \ \ rsum D f - x2 \ < (\ / 2)" + and I2: "fine \2 (b,c) D \ \ rsum D f - x2 \ < (\ / 2)" for D using IntegralE [OF \Integral (b, c) f x2\ \0 < \/2\] by auto define \ where "\ x = @@ -541,7 +541,7 @@ then have "\r>0. \s>0. \z. z \ x \ \z - x\ < s \ \(f z - f x) / (z - x) - f' x\ < r" by (simp add: DERIV_iff2 LIM_eq) with \0 < e\ obtain s - where "\z. z \ x \ \z - x\ < s \ \(f z - f x) / (z - x) - f' x\ < e/2" and "0 < s" + where "z \ x \ \z - x\ < s \ \(f z - f x) / (z - x) - f' x\ < e/2" and "0 < s" for z by (drule_tac x="e/2" in spec, auto) with strad1 [of x s f f' e] have strad: "\z. \z - x\ < s \ \f z - f x - f' x * (z - x)\ \ e/2 * \z - x\" @@ -586,8 +586,8 @@ from lemma_straddle [OF f' this] obtain \ where "gauge {a..b} \" - and \: "\x u v. \a \ u; u \ x; x \ v; v \ b; v - u < \ x\ \ - \f v - f u - f' x * (v - u)\ \ e * (v - u) / (b - a)" by auto + and \: "\a \ u; u \ x; x \ v; v \ b; v - u < \ x\ \ + \f v - f u - f' x * (v - u)\ \ e * (v - u) / (b - a)" for x u v by auto have "\D. fine \ (a, b) D \ \rsum D f' - (f b - f a)\ \ e" proof (clarify)