src/HOL/Hyperreal/Integration.thy
changeset 16588 8de758143786
parent 15944 9b00875e21f7
child 16775 c1b87ef4a1c3
--- a/src/HOL/Hyperreal/Integration.thy	Tue Jun 28 15:27:45 2005 +0200
+++ b/src/HOL/Hyperreal/Integration.thy	Tue Jun 28 15:28:04 2005 +0200
@@ -368,12 +368,8 @@
 
 text{*"Straddle Lemma" : Swartz and Thompson: AMM 95(7) 1988 *}
 
-lemma choiceP: "\<forall>x. P(x) --> (\<exists>y. Q x y) ==> \<exists>f. (\<forall>x. P(x) --> Q x (f x))"
-by meson
-
-lemma choiceP2: "\<forall>x. P(x) --> (\<exists>y. R(y) & (\<exists>z. Q x y z)) ==>
-      \<exists>f fa. (\<forall>x. P(x) --> R(f x) & Q x (f x) (fa x))"
-by meson
+lemma choiceP: "\<forall>x. P(x) --> (\<exists>y. Q x y) ==> \<exists>f. (\<forall>x. P(x) --> Q x (f x))" 
+by (insert bchoice [of "Collect P" Q], simp) 
 
 (*UNUSED
 lemma choice2: "\<forall>x. (\<exists>y. R(y) & (\<exists>z. Q x y z)) ==>