changeset 6444 | 2ebe9e630cab |
child 6494 | ab1442d2e4e1 |
--- /dev/null Thu Jan 01 00:00:00 1970 +0000 +++ b/src/HOL/Isar_examples/Cantor.thy Fri Apr 16 17:44:29 1999 +0200 @@ -0,0 +1,13 @@ +(* Title: HOL/Isar_examples/Cantor.thy + ID: $Id$ + Author: Markus Wenzel, TU Muenchen + +Cantor's theorem (see also 'Isabelle's Object-Logics'). +*) + +theory Cantor = Main:; + +theorem cantor: "EX S. S ~: range(f :: 'a => 'a set)"; +by (best elim: equalityCE); + +end;