haftmann [Sun, 15 Apr 2012 20:41:46 +0200] rev 47487
tuned whitespace
huffman [Sun, 15 Apr 2012 18:55:45 +0200] rev 47486
replace locale 'UFT' with new un-named context block feature;
use locale begin/end instead of 'in';
wenzelm [Sun, 15 Apr 2012 14:51:15 +0200] rev 47485
more CONTRIBUTORS;
wenzelm [Sun, 15 Apr 2012 14:50:09 +0200] rev 47484
some coverage of bundled declarations;
wenzelm [Sun, 15 Apr 2012 13:21:13 +0200] rev 47483
more uniform outline;
wenzelm [Sun, 15 Apr 2012 13:15:14 +0200] rev 47482
some coverage of unnamed contexts, which can be nested within other targets;
sultana [Sat, 14 Apr 2012 23:52:17 +0100] rev 47481
gathered mirabelle_sledgehammer's hardcoded defaults
sultana [Sat, 14 Apr 2012 23:52:17 +0100] rev 47480
Mirabelle's 'usage' description relating to Sledgehammer now synchs with the ML code of the Mirabelle-Sledgehammer action
sultana [Sat, 14 Apr 2012 23:52:17 +0100] rev 47479
Mirabelle now gives usage info when no arguments given
sultana [Sat, 14 Apr 2012 23:52:17 +0100] rev 47478
switched from using sed to perl in mirabelle tool
sultana [Sat, 14 Apr 2012 23:52:17 +0100] rev 47477
renamed mirabelle Tools directory to Actions, to make consistent with 'usage' description;
wenzelm [Sat, 14 Apr 2012 23:34:18 +0200] rev 47476
refined Cooper.tac / "presburger" method: Subgoal.FOCUS_PARAMS allows to solve more problems with outer quantifiers, e.g "!!x. [| 0 <= (x::int); x div 2 < f x |] ==> x < f x * 2";
clarified thin_prems_tac: fail as tactic without error;