# HG changeset patch # User wenzelm # Date 1020794044 -7200 # Node ID 5eb9be7b72a51ce94fd72c85d4c9d7519022df42 # Parent 7275750553b7a22a42ce67bc5b792b3392d98ac6 rev_bexI [intro?]; diff -r 7275750553b7 -r 5eb9be7b72a5 src/HOL/Set.thy --- a/src/HOL/Set.thy Tue May 07 19:15:11 2002 +0200 +++ b/src/HOL/Set.thy Tue May 07 19:54:04 2002 +0200 @@ -260,7 +260,7 @@ choice of @{prop "x:A"}. *} by (unfold Bex_def) blast -lemma rev_bexI: "x:A ==> P x ==> EX x:A. P x" +lemma rev_bexI [intro?]: "x:A ==> P x ==> EX x:A. P x" -- {* The best argument order when there is only one @{prop "x:A"}. *} by (unfold Bex_def) blast