# HG changeset patch # User nipkow # Date 1091605480 -7200 # Node ID e194d4d265fb72722b0de061d43fc6c53f15cc2a # Parent f14e0d9587bec6362b2d4ebd89d868445c5dc2ea fixed tex problem diff -r f14e0d9587be -r e194d4d265fb src/HOL/Hyperreal/Integration.thy --- a/src/HOL/Hyperreal/Integration.thy Tue Aug 03 14:48:59 2004 +0200 +++ b/src/HOL/Hyperreal/Integration.thy Wed Aug 04 09:44:40 2004 +0200 @@ -369,7 +369,7 @@ text{*Fundamental theorem of calculus (Part I)*} -text{*"Straddle Lemma" : Swartz & Thompson: AMM 95(7) 1988 *} +text{*"Straddle Lemma" : Swartz and Thompson: AMM 95(7) 1988 *} lemma choiceP: "\x. P(x) --> (\y. Q x y) ==> \f. (\x. P(x) --> Q x (f x))" by meson