diff -r 0ce594837524 -r fa53d267dab3 src/HOL/Isar_Examples/Drinker.thy --- a/src/HOL/Isar_Examples/Drinker.thy Thu Jul 01 14:32:57 2010 +0200 +++ b/src/HOL/Isar_Examples/Drinker.thy Thu Jul 01 18:31:46 2010 +0200 @@ -8,24 +8,21 @@ imports Main begin -text {* - Here is another example of classical reasoning: the Drinker's +text {* Here is another example of classical reasoning: the Drinker's Principle says that for some person, if he is drunk, everybody else is drunk! - We first prove a classical part of de-Morgan's law. -*} + We first prove a classical part of de-Morgan's law. *} -lemma deMorgan: +lemma de_Morgan: assumes "\ (\x. P x)" shows "\x. \ P x" - using prems + using assms proof (rule contrapos_np) assume a: "\ (\x. \ P x)" show "\x. P x" proof - fix x - show "P x" + fix x show "P x" proof (rule classical) assume "\ P x" then have "\x. \ P x" .. @@ -41,12 +38,12 @@ then show ?thesis .. next assume "\ (\x. drunk x)" - then have "\x. \ drunk x" by (rule deMorgan) + then have "\x. \ drunk x" by (rule de_Morgan) then obtain a where a: "\ drunk a" .. have "drunk a \ (\x. drunk x)" proof assume "drunk a" - with a show "\x. drunk x" by (contradiction) + with a show "\x. drunk x" by contradiction qed then show ?thesis .. qed