Wed, 27 Mar 2013 16:38:25 +0100 |
wenzelm |
more ambitious Goal.skip_proofs: covers Goal.prove forms as well, and do not insist in quick_and_dirty (for the sake of Isabelle/jEdit);
|
file |
diff |
annotate
|
Wed, 27 Mar 2013 14:19:18 +0100 |
wenzelm |
tuned signature and module arrangement;
|
file |
diff |
annotate
|
Sat, 09 Mar 2013 13:01:24 +0100 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
Mon, 04 Mar 2013 15:03:46 +0100 |
wenzelm |
refined parallel_proofs = 2: fork whole Isar sub-proofs, not just terminal ones;
|
file |
diff |
annotate
|
Thu, 28 Feb 2013 21:11:07 +0100 |
wenzelm |
simplified Proof.future_proof;
|
file |
diff |
annotate
|
Wed, 20 Feb 2013 11:40:30 +0100 |
wenzelm |
proper check of Proof.is_relevant (again, cf. c3e99efacb67 and df8fc0567a3d);
|
file |
diff |
annotate
|
Tue, 19 Feb 2013 17:55:26 +0100 |
wenzelm |
improved scheduling of forked proofs, based on elapsed time estimate (from last run via session log file);
|
file |
diff |
annotate
|
Fri, 25 Jan 2013 13:09:34 +0100 |
wenzelm |
clarified notion of Command.proper_range (according to Token.is_proper), especially relevant for Active.try_replace_command, to avoid loosing subsequent comments accidentally;
|
file |
diff |
annotate
|
Wed, 16 Jan 2013 18:43:59 +0100 |
wenzelm |
proper range position;
|
file |
diff |
annotate
|
Mon, 14 Jan 2013 13:59:43 +0100 |
wenzelm |
restrict "bad" markup to command keyword, notably excluding subsequent comments;
|
file |
diff |
annotate
|
Mon, 03 Dec 2012 14:44:00 +0100 |
wenzelm |
recovered error to finish proof (e.g. bad obtain export) from 223f18cfbb32;
|
file |
diff |
annotate
|
Sun, 25 Nov 2012 19:49:24 +0100 |
wenzelm |
Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
|
file |
diff |
annotate
|
Thu, 18 Oct 2012 14:15:46 +0200 |
wenzelm |
more robust future_proof result with specific error message (e.g. relevant for incomplete proof of non-registered theorem);
|
file |
diff |
annotate
|
Thu, 18 Oct 2012 13:26:49 +0200 |
wenzelm |
tuned message;
|
file |
diff |
annotate
|
Thu, 18 Oct 2012 12:26:30 +0200 |
wenzelm |
avoid spurious "bad" markup for show/test_proof;
|
file |
diff |
annotate
|
Wed, 17 Oct 2012 14:20:54 +0200 |
wenzelm |
skipped proofs appear as "bad" without counting as error;
|
file |
diff |
annotate
|
Wed, 17 Oct 2012 13:20:08 +0200 |
wenzelm |
more method position information, notably finished_pos after end of previous text;
|
file |
diff |
annotate
|
Tue, 16 Oct 2012 20:35:24 +0200 |
wenzelm |
tuned messages;
|
file |
diff |
annotate
|
Tue, 16 Oct 2012 20:23:00 +0200 |
wenzelm |
more proof method text position information;
|
file |
diff |
annotate
|
Tue, 16 Oct 2012 17:47:23 +0200 |
wenzelm |
clarified defer/prefer: more specific errors;
|
file |
diff |
annotate
|
Tue, 16 Oct 2012 15:14:12 +0200 |
wenzelm |
more informative errors for 'proof' and 'apply' steps;
|
file |
diff |
annotate
|
Tue, 16 Oct 2012 14:14:37 +0200 |
wenzelm |
more informative error for stand-alone 'qed';
|
file |
diff |
annotate
|
Tue, 16 Oct 2012 14:02:02 +0200 |
wenzelm |
further attempts to unify/simplify goal output;
|
file |
diff |
annotate
|
Tue, 16 Oct 2012 13:06:40 +0200 |
wenzelm |
more informative error messages of initial/terminal proof methods;
|
file |
diff |
annotate
|
Sat, 13 Oct 2012 21:09:20 +0200 |
wenzelm |
more informative error of initial/terminal proof steps;
|
file |
diff |
annotate
|
Sat, 13 Oct 2012 19:53:04 +0200 |
wenzelm |
some attempts to unify/simplify pretty_goal;
|
file |
diff |
annotate
|
Sat, 13 Oct 2012 18:04:11 +0200 |
wenzelm |
refined Proof.the_finished_goal with more informative error;
|
file |
diff |
annotate
|
Tue, 09 Oct 2012 20:05:17 +0200 |
wenzelm |
clarified Local_Defs.add_def(s): refrain from hard-wiring Thm.def_binding_optional;
|
file |
diff |
annotate
|
Sat, 01 Sep 2012 19:46:21 +0200 |
wenzelm |
removed unused material;
|
file |
diff |
annotate
|
Sat, 01 Sep 2012 19:43:18 +0200 |
wenzelm |
discontinued complicated/unreliable notion of recent proofs within context;
|
file |
diff |
annotate
|
Fri, 31 Aug 2012 16:35:30 +0200 |
wenzelm |
more precise register_proofs for local goals;
|
file |
diff |
annotate
|
Thu, 30 Aug 2012 21:50:49 +0200 |
wenzelm |
register proofs of Isar goals, to enable recovery from unstable command states after interactive cancellation;
|
file |
diff |
annotate
|
Thu, 30 Aug 2012 21:23:04 +0200 |
wenzelm |
refined treatment of forked proofs at transaction boundaries, including proof commands (see also 7ee000ce5390);
|
file |
diff |
annotate
|
Thu, 30 Aug 2012 19:18:49 +0200 |
wenzelm |
some support for registering forked proofs within Proof.state, using its bottom context;
|
file |
diff |
annotate
|
Fri, 27 Apr 2012 22:47:30 +0200 |
wenzelm |
clarified signature;
|
file |
diff |
annotate
|
Thu, 12 Apr 2012 11:34:50 +0200 |
wenzelm |
more precise declaration of goal_tfrees in forked proof state;
|
file |
diff |
annotate
|
Tue, 10 Apr 2012 21:31:05 +0200 |
wenzelm |
static relevance of proof via syntax keywords;
|
file |
diff |
annotate
|
Wed, 21 Mar 2012 21:24:13 +0100 |
wenzelm |
tuned signature;
|
file |
diff |
annotate
|
Wed, 21 Mar 2012 17:16:39 +0100 |
wenzelm |
tuned messages;
|
file |
diff |
annotate
|
Wed, 21 Mar 2012 11:00:34 +0100 |
wenzelm |
prefer explicitly qualified exception List.Empty;
|
file |
diff |
annotate
|
Sun, 18 Mar 2012 13:04:22 +0100 |
wenzelm |
maintain generic context naming in structure Name_Space (NB: empty = default_naming, init = local_naming);
|
file |
diff |
annotate
|
Tue, 28 Feb 2012 16:43:32 +0100 |
wenzelm |
display proof results as "state", to suppress odd squiggles in the Prover IDE (see also 9240be8c8c69);
|
file |
diff |
annotate
|
Tue, 14 Feb 2012 19:51:39 +0100 |
wenzelm |
tuned signature, according to actual usage of these operations;
|
file |
diff |
annotate
|
Mon, 28 Nov 2011 22:05:32 +0100 |
wenzelm |
separate module for concrete Isabelle markup;
|
file |
diff |
annotate
|
Sun, 20 Nov 2011 16:59:37 +0100 |
wenzelm |
uniform cert_vars/read_vars;
|
file |
diff |
annotate
|
Mon, 07 Nov 2011 17:00:23 +0100 |
wenzelm |
tuned signature -- avoid spurious Thm.mixed_attribute;
|
file |
diff |
annotate
|
Thu, 03 Nov 2011 22:23:41 +0100 |
wenzelm |
tuned signature -- canonical argument order;
|
file |
diff |
annotate
|
Mon, 01 Aug 2011 12:08:53 +0200 |
nipkow |
infrastructure for attaching names to hypothesis in cases; realised via the same tag mechanism as case names
|
file |
diff |
annotate
|
Mon, 11 Jul 2011 22:55:47 +0200 |
wenzelm |
tuned signature -- corresponding to Scala version;
|
file |
diff |
annotate
|
Thu, 12 May 2011 16:23:13 +0200 |
wenzelm |
proper configuration options Proof_Context.debug and Proof_Context.verbose;
|
file |
diff |
annotate
|
Wed, 27 Apr 2011 23:02:43 +0200 |
wenzelm |
more precise positions via binding;
|
file |
diff |
annotate
|
Sat, 16 Apr 2011 15:47:52 +0200 |
wenzelm |
modernized structure Proof_Context;
|
file |
diff |
annotate
|
Fri, 08 Apr 2011 14:20:57 +0200 |
wenzelm |
discontinued special treatment of structure Mixfix;
|
file |
diff |
annotate
|
Mon, 21 Mar 2011 20:15:03 +0100 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
Mon, 31 Jan 2011 23:53:07 +0100 |
wenzelm |
more specific Goal.fork_name;
|
file |
diff |
annotate
|
Wed, 15 Dec 2010 20:52:20 +0100 |
wenzelm |
show: display goal refinement rule as "state", to avoid odd Output.urgent_message and make its association with the goal more explicit;
|
file |
diff |
annotate
|
Sat, 04 Dec 2010 21:26:55 +0100 |
wenzelm |
formal notepad without any result;
|
file |
diff |
annotate
|
Mon, 22 Nov 2010 10:42:04 +0100 |
bulwahn |
added useful function map_context_result to signature
|
file |
diff |
annotate
|
Mon, 25 Oct 2010 21:06:56 +0200 |
wenzelm |
renamed Output.priority to Output.urgent_message to emphasize its special role more clearly;
|
file |
diff |
annotate
|
Wed, 22 Sep 2010 18:21:48 +0200 |
wenzelm |
renamed setmp_noncritical to Unsynchronized.setmp to emphasize its meaning;
|
file |
diff |
annotate
|