src/CCL/Wfd.thy
changeset 58963 26bf09b95dda
parent 58957 c9e744ea8a38
child 58971 8c9a319821b3
--- a/src/CCL/Wfd.thy	Sun Nov 09 20:49:28 2014 +0100
+++ b/src/CCL/Wfd.thy	Mon Nov 10 21:49:48 2014 +0100
@@ -48,7 +48,7 @@
 
 ML {*
   fun wfd_strengthen_tac ctxt s i =
-    res_inst_tac ctxt [(("Q", 0), s)] @{thm wfd_strengthen_lemma} i THEN assume_tac (i+1)
+    res_inst_tac ctxt [(("Q", 0), s)] @{thm wfd_strengthen_lemma} i THEN assume_tac ctxt (i+1)
 *}
 
 lemma wf_anti_sym: "[| Wfd(r);  <a,x>:r;  <x,a>:r |] ==> P"