Sat, 05 Mar 2016 17:01:45 +0100 |
wenzelm |
tuned signature -- clarified modules;
|
file |
diff |
annotate
|
Thu, 03 Mar 2016 15:23:02 +0100 |
wenzelm |
clarified modules;
|
file |
diff |
annotate
|
Wed, 22 Apr 2015 20:14:43 +0200 |
wenzelm |
allow diagnostic proof commands with skip_proofs;
|
file |
diff |
annotate
|
Thu, 16 Apr 2015 14:18:32 +0200 |
wenzelm |
explicit error for Toplevel.proof_of;
|
file |
diff |
annotate
|
Mon, 06 Apr 2015 17:06:48 +0200 |
wenzelm |
@{command_spec} is superseded by @{command_keyword};
|
file |
diff |
annotate
|
Wed, 04 Mar 2015 19:53:18 +0100 |
wenzelm |
tuned signature -- prefer qualified names;
|
file |
diff |
annotate
|
Tue, 23 Dec 2014 20:46:42 +0100 |
wenzelm |
explicit message channels for "state", "information";
|
file |
diff |
annotate
|
Thu, 06 Nov 2014 15:47:04 +0100 |
wenzelm |
more explicit Keyword.keywords;
|
file |
diff |
annotate
|
Mon, 03 Nov 2014 14:50:27 +0100 |
wenzelm |
eliminated unused int_only flag (see also c12484a27367);
|
file |
diff |
annotate
|
Mon, 03 Nov 2014 14:31:15 +0100 |
wenzelm |
eliminated obsolete Proof.goal_message -- print outcome more directly;
|
file |
diff |
annotate
|
Fri, 31 Oct 2014 17:08:54 +0100 |
wenzelm |
eliminated odd flags and hook;
|
file |
diff |
annotate
|
Fri, 31 Oct 2014 11:36:41 +0100 |
wenzelm |
discontinued obsolete Output.urgent_message;
|
file |
diff |
annotate
|
Fri, 31 Oct 2014 11:18:17 +0100 |
wenzelm |
discontinued Proof General;
|
file |
diff |
annotate
|
Tue, 08 Apr 2014 14:59:36 +0200 |
wenzelm |
more uniform ML/document antiquotations;
|
file |
diff |
annotate
|
Tue, 24 Sep 2013 13:23:25 +0200 |
wenzelm |
avoid clash of auto print functions with query operations, notably sledgehammer (cf. 3461985dcbc3);
|
file |
diff |
annotate
|
Fri, 23 Aug 2013 20:35:50 +0200 |
wenzelm |
added Theory.setup convenience;
|
file |
diff |
annotate
|
Sat, 10 Aug 2013 10:59:56 +0200 |
wenzelm |
explicit "strict" flag for print functions (flipped internal meaning);
|
file |
diff |
annotate
|
Fri, 02 Aug 2013 16:00:14 +0200 |
wenzelm |
support print functions with explicit arguments, as provided by overlays;
|
file |
diff |
annotate
|
Mon, 29 Jul 2013 13:28:27 +0200 |
wenzelm |
tuned signature;
|
file |
diff |
annotate
|
Sat, 13 Jul 2013 19:55:53 +0200 |
wenzelm |
avoid spurious warnings, notably of 'try0' about already declared simps etc.;
|
file |
diff |
annotate
|
Sat, 13 Jul 2013 18:33:33 +0200 |
wenzelm |
initial delay for automatically tried tools;
|
file |
diff |
annotate
|
Sat, 13 Jul 2013 16:45:47 +0200 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
Sat, 13 Jul 2013 16:34:57 +0200 |
wenzelm |
determine print function parameters dynamically, e.g. depending on runtime options;
|
file |
diff |
annotate
|
Sat, 13 Jul 2013 14:11:48 +0200 |
wenzelm |
clarified some default options;
|
file |
diff |
annotate
|
Sat, 13 Jul 2013 13:58:13 +0200 |
wenzelm |
gutter icon for information messages;
|
file |
diff |
annotate
|
Sat, 13 Jul 2013 00:50:49 +0200 |
wenzelm |
hybrid "auto" tool setup, for TTY (within theory) and PIDE (global print function);
|
file |
diff |
annotate
|
Fri, 12 Jul 2013 23:45:05 +0200 |
wenzelm |
system options for Isabelle/HOL proof tools;
|
file |
diff |
annotate
|
Wed, 15 May 2013 22:30:24 +0200 |
wenzelm |
clarified preferences: "override" re-initialized on prover startup, and "default" sent to PG -- thus recover typical defaults like auto-quickcheck in PG 4.x;
|
file |
diff |
annotate
|
Wed, 15 May 2013 20:22:46 +0200 |
wenzelm |
maintain ProofGeneral preferences within ProofGeneral module;
|
file |
diff |
annotate
|
Wed, 15 May 2013 17:39:41 +0200 |
wenzelm |
just one ProofGeneral module;
|
file |
diff |
annotate
|
Tue, 02 Apr 2013 10:58:51 +0200 |
blanchet |
got rid of legacy smartness
|
file |
diff |
annotate
|
Wed, 27 Mar 2013 17:58:07 +0100 |
wenzelm |
more robust access Toplevel.proof_of -- prefer warning via Toplevel.unknown_proof over hard crash (notably for skipped proofs);
|
file |
diff |
annotate
|
Fri, 16 Mar 2012 18:20:12 +0100 |
wenzelm |
outer syntax command definitions based on formal command_spec derived from theory header declarations;
|
file |
diff |
annotate
|
Mon, 30 May 2011 17:00:38 +0200 |
blanchet |
make SML/NJ happy
|
file |
diff |
annotate
|
Fri, 27 May 2011 10:30:08 +0200 |
blanchet |
repaired theory merging and defined/used helpers
|
file |
diff |
annotate
|
Fri, 27 May 2011 10:30:08 +0200 |
blanchet |
prioritize try and auto try's tools, with fast ones first, with a slight preference for provers vs. counterexample generators
|
file |
diff |
annotate
|
Fri, 27 May 2011 10:30:08 +0200 |
blanchet |
handle non-auto try case of Sledgehammer better
|
file |
diff |
annotate
|
Fri, 27 May 2011 10:30:08 +0200 |
blanchet |
added "try" command, to launch Solve Direct, Quickcheck, Nitpick, Sledgehammer, and Try Methods
|
file |
diff |
annotate
|
Fri, 27 May 2011 10:30:08 +0200 |
blanchet |
renamed "Auto_Tools" "Try"
|
file |
diff |
annotate
| base
|