Mirabelle: command-line action options may either be key=value or just key
authorboehmes
Sat, 05 Sep 2009 15:46:52 +0200
changeset 32522 1b70db55c811
parent 32521 f20cc66b2c74
child 32523 ba397aa0ff5d
Mirabelle: command-line action options may either be key=value or just key
src/HOL/Mirabelle/doc/options.txt
src/HOL/Mirabelle/lib/Tools/mirabelle
src/HOL/Mirabelle/lib/scripts/mirabelle.pl
--- a/src/HOL/Mirabelle/doc/options.txt	Sat Sep 05 11:45:57 2009 +0200
+++ b/src/HOL/Mirabelle/doc/options.txt	Sat Sep 05 15:46:52 2009 +0200
@@ -2,6 +2,5 @@
 
   * prover=NAME: name of the external prover to call
   * keep=PATH: path where to keep temporary files created by sledgehammer 
-  * metis=X: apply metis with the theorems found by sledgehammer (X may be any
-      non-empty string)
-  * full_types=X: turn on full-typed encoding (X may be any non-empty string)
+  * metis: apply metis with the theorems found by sledgehammer
+  * full_types: turn on full-typed encoding
--- a/src/HOL/Mirabelle/lib/Tools/mirabelle	Sat Sep 05 11:45:57 2009 +0200
+++ b/src/HOL/Mirabelle/lib/Tools/mirabelle	Sat Sep 05 15:46:52 2009 +0200
@@ -32,9 +32,12 @@
   echo "  at all proof steps in the given theory files."
   echo
   echo "  ACTIONS is a colon-separated list of actions, where each action is"
-  echo "  either NAME or NAME[KEY=VALUE,...,KEY=VALUE]. Available actions are:"
+  echo "  either NAME or NAME[OPTION,...,OPTION]. Available actions are:"
   print_action_names
   echo
+  echo "  A list of available OPTIONs can be found here:"
+  echo "    $MIRABELLE_HOME/doc/options.txt"
+  echo
   echo "  FILES is a list of theory files, where each file is either NAME.thy"
   echo "  or NAME.thy[START:END] and START and END are numbers indicating the"
   echo "  range the given actions are to be applied."
--- a/src/HOL/Mirabelle/lib/scripts/mirabelle.pl	Sat Sep 05 11:45:57 2009 +0200
+++ b/src/HOL/Mirabelle/lib/scripts/mirabelle.pl	Sat Sep 05 15:46:52 2009 +0200
@@ -82,6 +82,10 @@
         print SETUP_FILE "$sep(\"$1\", \"$2\")";
         $sep = ", ";
       }
+      elsif (m/\s*(.*)\s*/) {
+	print SETUP_FILE "$sep(\"$1\", \"\")";
+	$sep = ", ";
+      }
     }
     print SETUP_FILE "] *}\n";
   }