src/FOL/ex/Classical.thy
changeset 51717 9e7d1c139569
parent 42789 3a84b6947932
child 58889 5b7a9633cfa8
--- a/src/FOL/ex/Classical.thy	Tue Apr 16 17:54:14 2013 +0200
+++ b/src/FOL/ex/Classical.thy	Thu Apr 18 17:07:01 2013 +0200
@@ -300,7 +300,7 @@
 
 (*Other proofs: Can use auto, which cheats by using rewriting!  
   Deepen_tac alone requires 253 secs.  Or
-  by (mini_tac 1 THEN Deepen_tac 5 1) *)
+  by (mini_tac @{context} 1 THEN Deepen_tac 5 1) *)
 
 text{*44*}
 lemma "(\<forall>x. f(x) --> (\<exists>y. g(y) & h(x,y) & (\<exists>y. g(y) & ~ h(x,y)))) &