Mon, 02 Nov 2009 20:57:48 +0100 |
wenzelm |
modernized structure Proof_Display;
|
file |
diff |
annotate
|
Mon, 02 Nov 2009 20:45:23 +0100 |
wenzelm |
modernized structure AutoBind;
|
file |
diff |
annotate
|
Sun, 01 Nov 2009 15:24:45 +0100 |
wenzelm |
modernized structure Rule_Cases;
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 22:01:05 +0100 |
wenzelm |
replaced slightly odd get_goal/flat_goal by explicit goal views that correspond to the usual method categories;
|
file |
diff |
annotate
|
Sun, 25 Oct 2009 19:17:42 +0100 |
wenzelm |
more direct access to naming;
|
file |
diff |
annotate
|
Tue, 20 Oct 2009 21:26:45 +0200 |
wenzelm |
backpatching of structure Proof and ProofContext -- avoid odd aliases;
|
file |
diff |
annotate
|
Fri, 02 Oct 2009 21:39:06 +0200 |
wenzelm |
clarified Proof.refine_insert -- always "refine" to apply standard method treatment (of conjunctions);
|
file |
diff |
annotate
|
Wed, 30 Sep 2009 22:25:50 +0200 |
wenzelm |
eliminated dead code;
|
file |
diff |
annotate
|
Wed, 30 Sep 2009 00:57:28 +0200 |
wenzelm |
replaced chained_goal by slightly more appropriate flat_goal;
|
file |
diff |
annotate
|
Wed, 30 Sep 2009 00:17:06 +0200 |
wenzelm |
added chained_goal, which presents the goal thm as seen by semi-structured methods;
|
file |
diff |
annotate
|
Tue, 29 Sep 2009 11:49:22 +0200 |
wenzelm |
explicit indication of Unsynchronized.ref;
|
file |
diff |
annotate
|
Sat, 25 Jul 2009 18:02:43 +0200 |
wenzelm |
basic method application: avoid Position.setmp_thread_data_seq, which destroys transaction context;
|
file |
diff |
annotate
|
Sat, 25 Jul 2009 10:31:27 +0200 |
wenzelm |
renamed structure Display_Goal to Goal_Display;
|
file |
diff |
annotate
|
Fri, 24 Jul 2009 11:50:35 +0200 |
wenzelm |
Display_Goal.pretty_goals: always Markup.subgoal, clarified options;
|
file |
diff |
annotate
|
Thu, 23 Jul 2009 16:52:16 +0200 |
wenzelm |
clarified pretty_goals, pretty_thm_aux: plain context;
|
file |
diff |
annotate
|
Tue, 21 Jul 2009 01:03:18 +0200 |
wenzelm |
proper context for Display.pretty_thm etc. or old-style versions Display.pretty_thm_global, Display.pretty_thm_without_context etc.;
|
file |
diff |
annotate
|
Mon, 20 Jul 2009 21:20:09 +0200 |
wenzelm |
moved pretty_goals etc. to Display_Goal (required by tracing tacticals);
|
file |
diff |
annotate
|
Mon, 20 Jul 2009 00:37:39 +0200 |
wenzelm |
Proof.future_proof: declare all assumptions as well;
|
file |
diff |
annotate
|
Sun, 19 Jul 2009 19:24:04 +0200 |
wenzelm |
parallel_proofs: more fine-grained control with optional parallel checking of nested Isar proofs;
|
file |
diff |
annotate
|
Sun, 19 Jul 2009 18:02:40 +0200 |
wenzelm |
more abstract Future.is_worker;
|
file |
diff |
annotate
|
Sat, 28 Mar 2009 17:53:33 +0100 |
wenzelm |
renamed ProofContext.add_fixes_i to ProofContext.add_fixes, eliminated obsolete external version;
|
file |
diff |
annotate
|
Sat, 28 Mar 2009 17:21:11 +0100 |
wenzelm |
renamed ProofContext.note_thmss_i to ProofContext.note_thmss, eliminated obsolete external version;
|
file |
diff |
annotate
|
Sat, 28 Mar 2009 17:10:43 +0100 |
wenzelm |
simplified references to facts, eliminated external note_thmss;
|
file |
diff |
annotate
|
Sat, 28 Mar 2009 16:31:16 +0100 |
wenzelm |
replaced add_binds(_i) by bind_terms -- internal version only;
|
file |
diff |
annotate
|
Tue, 17 Mar 2009 13:33:21 +0100 |
wenzelm |
goal_tac: finish marked assumptions from left to right -- corresponds better with the strategy of etac, with significant performance gains in some situations;
|
file |
diff |
annotate
|
Fri, 13 Mar 2009 19:58:26 +0100 |
wenzelm |
unified type Proof.method and pervasive METHOD combinators;
|
file |
diff |
annotate
|
Tue, 10 Mar 2009 21:18:52 +0100 |
wenzelm |
invoke_case: proper qualification of name binding, avoiding old no_base_names;
|
file |
diff |
annotate
|
Thu, 05 Mar 2009 11:58:53 +0100 |
wenzelm |
eliminated obsolete ProofContext.full_bname;
|
file |
diff |
annotate
|
Tue, 03 Mar 2009 14:07:43 +0100 |
wenzelm |
Thm.binding;
|
file |
diff |
annotate
|
Wed, 21 Jan 2009 16:47:32 +0100 |
haftmann |
binding is alias for Binding.T
|
file |
diff |
annotate
|
Sun, 11 Jan 2009 18:18:35 +0100 |
wenzelm |
added Goal.future_enabled abstraction -- now also checks that this is already
|
file |
diff |
annotate
|
Sat, 10 Jan 2009 21:32:30 +0100 |
wenzelm |
added parallel_proofs flag (default true, cf. usedir option -Q), which can be disabled in low-memory situations;
|
file |
diff |
annotate
|
Thu, 08 Jan 2009 13:18:34 +0100 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
Thu, 08 Jan 2009 08:06:11 +0100 |
haftmann |
made SML/NJ happy
|
file |
diff |
annotate
|
Wed, 07 Jan 2009 20:27:05 +0100 |
wenzelm |
future_proof: refined version covers local_future_proof and global_future_proof;
|
file |
diff |
annotate
|
Wed, 07 Jan 2009 16:22:10 +0100 |
wenzelm |
qed/after_qed: singleton result;
|
file |
diff |
annotate
|
Wed, 07 Jan 2009 12:09:39 +0100 |
wenzelm |
future_terminal_proof: no fork for interactive mode, assert_backward;
|
file |
diff |
annotate
|
Tue, 06 Jan 2009 13:36:42 +0100 |
wenzelm |
future_terminal_proof: check Future.enabled;
|
file |
diff |
annotate
|
Mon, 05 Jan 2009 14:22:40 +0100 |
wenzelm |
added future_terminal_proof;
|
file |
diff |
annotate
|
Sun, 04 Jan 2009 15:40:30 +0100 |
wenzelm |
more precise is_relevant: requires original main goal, not initial goal state;
|
file |
diff |
annotate
|
Fri, 12 Dec 2008 22:13:13 +0100 |
wenzelm |
global_qed: refrain from ProofContext.auto_bind_facts, to avoid
|
file |
diff |
annotate
|
Fri, 05 Dec 2008 00:23:37 +0100 |
wenzelm |
merged
|
file |
diff |
annotate
|
Thu, 04 Dec 2008 23:00:58 +0100 |
wenzelm |
future proofs: pass actual futures to facilitate composite computations;
|
file |
diff |
annotate
|
Thu, 04 Dec 2008 14:43:33 +0100 |
haftmann |
cleaned up binding module and related code
|
file |
diff |
annotate
|
Thu, 16 Oct 2008 22:44:36 +0200 |
wenzelm |
conclude_goal: precise goal context, include all sorts from context into statement, check shyps of result;
|
file |
diff |
annotate
|
Thu, 02 Oct 2008 14:22:40 +0200 |
wenzelm |
simplified Exn.EXCEPTIONS;
|
file |
diff |
annotate
|
Wed, 01 Oct 2008 22:33:24 +0200 |
wenzelm |
replaced can_defer by is_relevant (negation);
|
file |
diff |
annotate
|
Wed, 01 Oct 2008 18:16:14 +0200 |
wenzelm |
future_proof: protect conclusion of deferred proof state;
|
file |
diff |
annotate
|
Wed, 01 Oct 2008 12:18:18 +0200 |
wenzelm |
renamed promise to future, tuned related interfaces;
|
file |
diff |
annotate
|
Wed, 01 Oct 2008 12:00:02 +0200 |
wenzelm |
more robust treatment of Interrupt (cf. exn.ML);
|
file |
diff |
annotate
|
Tue, 30 Sep 2008 23:31:38 +0200 |
wenzelm |
promise_proof: proper statement with empty vars;
|
file |
diff |
annotate
|
Mon, 29 Sep 2008 21:26:32 +0200 |
wenzelm |
promise global proofs;
|
file |
diff |
annotate
|
Fri, 26 Sep 2008 19:07:56 +0200 |
wenzelm |
eliminated polymorphic equality;
|
file |
diff |
annotate
|
Thu, 18 Sep 2008 14:06:58 +0200 |
wenzelm |
show: non-critical testing;
|
file |
diff |
annotate
|
Wed, 17 Sep 2008 22:06:57 +0200 |
wenzelm |
added map_contexts;
|
file |
diff |
annotate
|
Tue, 02 Sep 2008 16:55:33 +0200 |
wenzelm |
type Attrib.binding abbreviates Name.binding without attributes;
|
file |
diff |
annotate
|
Tue, 02 Sep 2008 14:10:45 +0200 |
wenzelm |
explicit type Name.binding for higher-specification elements;
|
file |
diff |
annotate
|
Fri, 16 May 2008 21:53:27 +0200 |
wenzelm |
removed obsolete case rule_context;
|
file |
diff |
annotate
|
Wed, 19 Mar 2008 22:27:57 +0100 |
wenzelm |
renamed datatype thmref to Facts.ref, tuned interfaces;
|
file |
diff |
annotate
|
Tue, 11 Mar 2008 17:13:41 +0100 |
wenzelm |
put_facts: do_props, i.e. facts are indexed by proposition again;
|
file |
diff |
annotate
|