src/Sequents/ILL.thy
changeset 42814 5af15f1e2ef6
parent 39159 0dec18004e75
child 51309 473303ef6e34
--- a/src/Sequents/ILL.thy	Sun May 15 17:06:35 2011 +0200
+++ b/src/Sequents/ILL.thy	Sun May 15 17:45:53 2011 +0200
@@ -274,10 +274,10 @@
 
 
 method_setup best_safe =
-  {* Scan.succeed (K (SIMPLE_METHOD' (best_tac safe_cs))) *} ""
+  {* Scan.succeed (K (SIMPLE_METHOD' (best_tac safe_cs))) *}
 
 method_setup best_power =
-  {* Scan.succeed (K (SIMPLE_METHOD' (best_tac power_cs))) *} ""
+  {* Scan.succeed (K (SIMPLE_METHOD' (best_tac power_cs))) *}
 
 
 (* Some examples from Troelstra and van Dalen *)