Rephrased forward proofs to avoid problems with HO unification
authorberghofe
Wed, 07 May 2008 10:59:22 +0200
changeset 26812 c0fa62fa0e5b
parent 26811 067cceb36e26
child 26813 6a4d5ca6d2e5
Rephrased forward proofs to avoid problems with HO unification
src/HOL/Isar_examples/KnasterTarski.thy
--- a/src/HOL/Isar_examples/KnasterTarski.thy	Wed May 07 10:59:21 2008 +0200
+++ b/src/HOL/Isar_examples/KnasterTarski.thy	Wed May 07 10:59:22 2008 +0200
@@ -63,7 +63,7 @@
       finally (order_antisym) show ?thesis .
     }
     from mono ge have "f (f ?a) <= f ?a" ..
-    hence "f ?a : ?H" ..
+    hence "f ?a : ?H" by simp
     thus "?a <= f ?a" by (rule Inter_lower)
   qed
 qed
@@ -100,7 +100,7 @@
     show "?a <= f ?a"
     proof (rule Inter_lower)
       from mono ge have "f (f ?a) <= f ?a" ..
-      thus "f ?a : ?H" ..
+      thus "f ?a : ?H" by simp
     qed
   qed
 qed