diff -r 4a16f8e41879 -r 7338eb25226c src/HOL/Isar_Examples/Drinker.thy --- a/src/HOL/Isar_Examples/Drinker.thy Tue Oct 07 20:43:18 2014 +0200 +++ b/src/HOL/Isar_Examples/Drinker.thy Tue Oct 07 20:59:46 2014 +0200 @@ -2,17 +2,17 @@ Author: Makarius *) -header {* The Drinker's Principle *} +header \The Drinker's Principle\ theory Drinker 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 de_Morgan: assumes "\ (\x. P x)" @@ -25,10 +25,10 @@ proof (rule classical) assume "\ P x" then have "\x. \ P x" .. - with `\ (\x. \ P x)` show ?thesis by contradiction + with \\ (\x. \ P x)\ show ?thesis by contradiction qed qed - with `\ (\x. P x)` show ?thesis by contradiction + with \\ (\x. P x)\ show ?thesis by contradiction qed theorem Drinker's_Principle: "\x. drunk x \ (\x. drunk x)"