src/Pure/Isar/proof.ML
Fri, 09 May 2014 22:14:06 +0200 wenzelm more markup;
Fri, 09 May 2014 22:04:50 +0200 wenzelm more position markup to help locating the query context, e.g. from "Info" dockable;
Thu, 08 May 2014 16:15:20 +0200 wenzelm some position markup to help locating the query context, e.g. from "Info" dockable;
Wed, 07 May 2014 14:05:17 +0200 wenzelm tuned message: "step" goes back to TTY mode before Proof General, while "depth" is more informative but sometimes confusing due to implementation details;
Wed, 07 May 2014 13:55:16 +0200 wenzelm print results as "state", to avoid intrusion into the source text;
Sun, 09 Mar 2014 16:37:56 +0100 wenzelm tuned signature;
Sat, 08 Mar 2014 21:08:10 +0100 wenzelm modernized Attrib.check_name/check_src similar to methods (see also a989bdaf8121);
Thu, 06 Mar 2014 14:38:54 +0100 wenzelm eliminated odd type constraint for read_const (see also 79c1d2bbe5a9);
Thu, 06 Mar 2014 13:44:01 +0100 wenzelm more uniform check_const/read_const;
Wed, 26 Feb 2014 11:58:35 +0100 wenzelm markup for method combinators;
Tue, 25 Feb 2014 14:34:18 +0100 wenzelm modernized Method.check_name/check_source (with reports) vs. strict Method.the_method (without interning nor reports), e.g. relevant for semantic completion;
Mon, 24 Feb 2014 10:48:34 +0100 wenzelm clarified Token.range_of in accordance to Symbol_Pos.range;
Sat, 11 Jan 2014 20:06:31 +0100 wenzelm check_hyps for attribute application (still inactive, due to non-compliant tools);
Fri, 10 Jan 2014 21:37:28 +0100 wenzelm more elementary management of declared hyps, below structure Assumption;
Fri, 10 Jan 2014 16:20:06 +0100 wenzelm explicit check of background theory;
Sat, 14 Dec 2013 17:28:05 +0100 wenzelm proper context for basic Simplifier operations: rewrite_rule, rewrite_goals_rule, rewrite_goals_tac etc.;
Sat, 23 Nov 2013 17:15:44 +0100 wenzelm more uniform / rigid checking of Goal.prove_common vs. Proof.conclude_goal -- NB: Goal.prove_common cannot check hyps right now, e.g. due to undeclared Simplifier prems;
Tue, 03 Sep 2013 19:58:00 +0200 wenzelm cases: formal binding of 'assumes', with position provided via invoke_case;
Tue, 03 Sep 2013 13:09:15 +0200 wenzelm cases: more position information and PIDE markup;
Sun, 25 Aug 2013 20:32:26 +0200 wenzelm maintain goal forks as part of global execution;
Sun, 25 Aug 2013 16:03:12 +0200 wenzelm discontinued parallel_subproofs_saturation and related internal counters (superseded by parallel_subproofs_threshold and timing information);
Sat, 27 Jul 2013 16:35:51 +0200 wenzelm standardized aliases;
Sat, 13 Jul 2013 00:50:49 +0200 wenzelm hybrid "auto" tool setup, for TTY (within theory) and PIDE (global print function);
Wed, 26 Jun 2013 21:48:23 +0200 wenzelm less intrusive SELECT_GOAL: merely rearrange subgoals without detaching goal state, and thus preserve maxidx context;
Wed, 26 Jun 2013 11:54:45 +0200 wenzelm tuned signature;
Tue, 09 Apr 2013 20:16:52 +0200 wenzelm just one timing protocol function, with 3 implementations: TTY/PG, PIDE/document, build;
Wed, 03 Apr 2013 21:48:43 +0200 wenzelm additional timing status for implicitly forked terminal proofs -- proper accounting for interactive Timing dockable etc.;
Wed, 03 Apr 2013 21:30:32 +0200 wenzelm more explicit Goal.fork_params -- avoid implicit arguments via thread data;
Sat, 30 Mar 2013 13:40:19 +0100 wenzelm more item markup;
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);
Wed, 27 Mar 2013 14:19:18 +0100 wenzelm tuned signature and module arrangement;
Sat, 09 Mar 2013 13:01:24 +0100 wenzelm tuned;
Mon, 04 Mar 2013 15:03:46 +0100 wenzelm refined parallel_proofs = 2: fork whole Isar sub-proofs, not just terminal ones;
Thu, 28 Feb 2013 21:11:07 +0100 wenzelm simplified Proof.future_proof;
Wed, 20 Feb 2013 11:40:30 +0100 wenzelm proper check of Proof.is_relevant (again, cf. c3e99efacb67 and df8fc0567a3d);
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);
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;
Wed, 16 Jan 2013 18:43:59 +0100 wenzelm proper range position;
Mon, 14 Jan 2013 13:59:43 +0100 wenzelm restrict "bad" markup to command keyword, notably excluding subsequent comments;
Mon, 03 Dec 2012 14:44:00 +0100 wenzelm recovered error to finish proof (e.g. bad obtain export) from 223f18cfbb32;
Sun, 25 Nov 2012 19:49:24 +0100 wenzelm Isabelle-specific implementation of quasi-abstract markup elements -- back to module arrangement before d83797ef0d2d;
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);
Thu, 18 Oct 2012 13:26:49 +0200 wenzelm tuned message;
Thu, 18 Oct 2012 12:26:30 +0200 wenzelm avoid spurious "bad" markup for show/test_proof;
Wed, 17 Oct 2012 14:20:54 +0200 wenzelm skipped proofs appear as "bad" without counting as error;
Wed, 17 Oct 2012 13:20:08 +0200 wenzelm more method position information, notably finished_pos after end of previous text;
Tue, 16 Oct 2012 20:35:24 +0200 wenzelm tuned messages;
Tue, 16 Oct 2012 20:23:00 +0200 wenzelm more proof method text position information;
Tue, 16 Oct 2012 17:47:23 +0200 wenzelm clarified defer/prefer: more specific errors;
Tue, 16 Oct 2012 15:14:12 +0200 wenzelm more informative errors for 'proof' and 'apply' steps;
Tue, 16 Oct 2012 14:14:37 +0200 wenzelm more informative error for stand-alone 'qed';
Tue, 16 Oct 2012 14:02:02 +0200 wenzelm further attempts to unify/simplify goal output;
Tue, 16 Oct 2012 13:06:40 +0200 wenzelm more informative error messages of initial/terminal proof methods;
Sat, 13 Oct 2012 21:09:20 +0200 wenzelm more informative error of initial/terminal proof steps;
Sat, 13 Oct 2012 19:53:04 +0200 wenzelm some attempts to unify/simplify pretty_goal;
Sat, 13 Oct 2012 18:04:11 +0200 wenzelm refined Proof.the_finished_goal with more informative error;
Tue, 09 Oct 2012 20:05:17 +0200 wenzelm clarified Local_Defs.add_def(s): refrain from hard-wiring Thm.def_binding_optional;
Sat, 01 Sep 2012 19:46:21 +0200 wenzelm removed unused material;
Sat, 01 Sep 2012 19:43:18 +0200 wenzelm discontinued complicated/unreliable notion of recent proofs within context;
Fri, 31 Aug 2012 16:35:30 +0200 wenzelm more precise register_proofs for local goals;
less more (0) -300 -100 -60 tip