src/HOL/Isar_examples/KnasterTarski.thy
changeset 7982 d534b897ce39
parent 7874 180364256231
child 8902 a705822f4e2a
--- a/src/HOL/Isar_examples/KnasterTarski.thy	Sat Oct 30 20:13:16 1999 +0200
+++ b/src/HOL/Isar_examples/KnasterTarski.thy	Sat Oct 30 20:20:48 1999 +0200
@@ -37,7 +37,8 @@
  The Isar proof below closely follows the original presentation.
  Virtually all of the prose narration has been rephrased in terms of
  formal Isar language elements.  Just as many textbook-style proofs,
- there is a strong bias towards forward reasoning.
+ there is a strong bias towards forward proof, and several bends
+ in the course of reasoning.
 *};
 
 theorem KnasterTarski: "mono f ==> EX a::'a set. f a = a";
@@ -72,11 +73,11 @@
  explicit block structure and weak assumptions.  Thus we have mimicked
  the particular way of reasoning of the original text.
 
- In the subsequent version of the proof the order of reasoning is
- changed to achieve structured top-down decomposition of the problem
- at the outer level, while the small inner steps of reasoning or done
- in a forward manner.  Note that this requires only the most basic
- features of the Isar language, we are certainly more at ease here.
+ In the subsequent version the order of reasoning is changed to
+ achieve structured top-down decomposition of the problem at the outer
+ level, while only the inner steps of reasoning are done in a forward
+ manner.  We are certainly more at ease here, requiring only the most
+ basic features of the Isar language.
 *};
 
 theorem KnasterTarski': "mono f ==> EX a::'a set. f a = a";