src/HOL/Isar_examples/Cantor.thy
changeset 9474 b0ce3b7c9c26
parent 7982 d534b897ce39
child 10007 64bf7da1994a
--- a/src/HOL/Isar_examples/Cantor.thy	Sun Jul 30 13:02:14 2000 +0200
+++ b/src/HOL/Isar_examples/Cantor.thy	Sun Jul 30 13:02:56 2000 +0200
@@ -95,16 +95,15 @@
 
 text {*
  How much creativity is required?  As it happens, Isabelle can prove
- this theorem automatically.  The context of Isabelle's classical
- prover contains rules for most of the constructs of HOL's set theory.
- We must augment it with \name{equalityCE} to break up set equalities,
- and then apply best-first search.  Depth-first search would diverge,
- but best-first search successfully navigates through the large search
- space.
+ this theorem automatically using best-first search.  Depth-first
+ search would diverge, but best-first search successfully navigates
+ through the large search space.  The context of Isabelle's classical
+ prover contains rules for the relevant constructs of HOL's set
+ theory.
 *};
 
 theorem "EX S. S ~: range (f :: 'a => 'a set)";
-  by (best elim: equalityCE);
+  by best;
 
 text {*
  While this establishes the same theorem internally, we do not get any