src/CCL/CCL.thy
changeset 47966 b8a94ed1646e
parent 42814 5af15f1e2ef6
child 51307 943ad9c0d99d
--- a/src/CCL/CCL.thy	Wed May 23 15:40:10 2012 +0200
+++ b/src/CCL/CCL.thy	Wed May 23 15:57:12 2012 +0200
@@ -349,7 +349,7 @@
 
 lemma po_lam: "lam x. f(x) [= lam x. f'(x) <-> (ALL x. f(x) [= f'(x))"
   apply (rule poXH [THEN iff_trans])
-  apply fastsimp
+  apply fastforce
   done
 
 lemmas ccl_porews = po_bot po_pair po_lam