# HG changeset patch # User wenzelm # Date 1457209408 -3600 # Node ID 5335e5c53312ddec63fe6dbb6bb84552a8493381 # Parent d32c23d29968943c99734c0bab80bbf474ef096f tuned; diff -r d32c23d29968 -r 5335e5c53312 src/HOL/Isar_Examples/Cantor.thy --- a/src/HOL/Isar_Examples/Cantor.thy Sat Mar 05 20:47:31 2016 +0100 +++ b/src/HOL/Isar_Examples/Cantor.thy Sat Mar 05 21:23:28 2016 +0100 @@ -17,7 +17,7 @@ \<^item> @{url "https://en.wikipedia.org/wiki/Cantor's_diagonal_argument"} \ -theorem Cantor: "\ (\f :: 'a \ 'a set. \A. \x. A = f x)" +theorem Cantor: "\f :: 'a \ 'a set. \A. \x. A = f x" proof assume "\f :: 'a \ 'a set. \A. \x. A = f x" then obtain f :: "'a \ 'a set" where *: "\A. \x. A = f x" .. @@ -35,10 +35,10 @@ works. \ -theorem "\ (\f :: 'a \ 'a set. \A. \x. f x = A)" +theorem "\f :: 'a \ 'a set. \A. \x. f x = A" by best -theorem "\ (\f :: 'a \ 'a set. \A. \x. f x = A)" +theorem "\f :: 'a \ 'a set. \A. \x. f x = A" by force @@ -63,7 +63,7 @@ with * show A .. qed -theorem Cantor': "\ (\f :: 'a \ 'a \ bool. \A. \x. A = f x)" +theorem Cantor': "\f :: 'a \ 'a \ bool. \A. \x. A = f x" proof assume "\f :: 'a \ 'a \ bool. \A. \x. A = f x" then obtain f :: "'a \ 'a \ bool" where *: "\A. \x. A = f x" .. diff -r d32c23d29968 -r 5335e5c53312 src/HOL/Isar_Examples/Drinker.thy --- a/src/HOL/Isar_Examples/Drinker.thy Sat Mar 05 20:47:31 2016 +0100 +++ b/src/HOL/Isar_Examples/Drinker.thy Sat Mar 05 21:23:28 2016 +0100 @@ -19,14 +19,14 @@ assumes "\ (\x. P x)" shows "\x. \ P x" proof (rule classical) - assume "\ (\x. \ P x)" + assume "\x. \ P x" have "\x. P x" proof fix x show "P x" 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