| Wed, 18 Mar 2009 22:41:14 +0100 |
wenzelm |
more precise type Symbol_Pos.text;
|
file |
diff |
annotate
|
| Tue, 17 Mar 2009 19:06:04 +0100 |
wenzelm |
close/all_assm_tac: finish all subgoals from left to right (cf. Proof.goal_tac a28d83e903ce) -- NB: ALLGOALS/THEN_ALL_NEW operate from right to left;
|
file |
diff |
annotate
|
| Mon, 16 Mar 2009 17:46:49 +0100 |
wenzelm |
adapted 'method_setup' command to Method.setup;
|
file |
diff |
annotate
|
| Sun, 15 Mar 2009 20:19:14 +0100 |
wenzelm |
export section, sections;
|
file |
diff |
annotate
|
| Fri, 13 Mar 2009 23:50:05 +0100 |
wenzelm |
simplified method setup;
|
file |
diff |
annotate
|
| Fri, 13 Mar 2009 21:24:21 +0100 |
wenzelm |
added simplified setup;
|
file |
diff |
annotate
|
| Fri, 13 Mar 2009 19:10:46 +0100 |
wenzelm |
tuned Method exports: non-pervasive type method (cf. Proof.method), pervasive METHOD combinators;
|
file |
diff |
annotate
|
| Thu, 12 Mar 2009 11:10:02 +0100 |
wenzelm |
renamed NameSpace.bind to NameSpace.define;
|
file |
diff |
annotate
|
| Wed, 04 Mar 2009 11:05:29 +0100 |
blanchet |
Merge.
|
file |
diff |
annotate
|
| Wed, 04 Mar 2009 10:45:52 +0100 |
blanchet |
Merge.
|
file |
diff |
annotate
|
| Wed, 04 Mar 2009 00:05:20 +0100 |
wenzelm |
renamed Method.assumption_tac back to Method.assm_tac -- as assumption_tac it would have to be exactly the tactic behind the assumption method (with facts);
|
file |
diff |
annotate
|
| Sun, 01 Mar 2009 23:36:12 +0100 |
wenzelm |
use long names for old-style fold combinators;
|
file |
diff |
annotate
|
| Sat, 28 Feb 2009 14:52:21 +0100 |
wenzelm |
moved generic intuitionistic prover to src/Tools/intuitionistic.ML;
|
file |
diff |
annotate
|
| Wed, 11 Feb 2009 14:48:14 +1100 |
kleing |
FindTheorems: add solves feature; tidy up const name subsettin; patch by Timothy Bourke
|
file |
diff |
annotate
|
| Thu, 01 Jan 2009 22:57:42 +0100 |
wenzelm |
assumption/close: discontinued implicit prems;
|
file |
diff |
annotate
|
| Fri, 05 Dec 2008 18:42:37 +0100 |
haftmann |
removed Table.extend, NameSpace.extend_table
|
file |
diff |
annotate
|
| Sat, 09 Aug 2008 22:43:55 +0200 |
wenzelm |
unified Args.T with OuterLex.token, renamed some operations;
|
file |
diff |
annotate
|
| Wed, 06 Aug 2008 00:10:22 +0200 |
wenzelm |
report markup;
|
file |
diff |
annotate
|
| Mon, 04 Aug 2008 20:27:39 +0200 |
wenzelm |
tuned signature;
|
file |
diff |
annotate
|
| Sat, 28 Jun 2008 21:21:17 +0200 |
wenzelm |
replaced simple_text by fully-featured parse_args;
|
file |
diff |
annotate
|
| Mon, 16 Jun 2008 22:13:52 +0200 |
wenzelm |
renamed rename_params_tac to rename_tac;
|
file |
diff |
annotate
|
| Mon, 16 Jun 2008 17:54:49 +0200 |
wenzelm |
ML tactic: do not abstract over context again;
|
file |
diff |
annotate
|
| Wed, 14 May 2008 20:30:29 +0200 |
wenzelm |
added intern, defined;
|
file |
diff |
annotate
|
| Tue, 29 Apr 2008 19:55:02 +0200 |
haftmann |
added lemma antiquotation
|
file |
diff |
annotate
|
| Fri, 28 Mar 2008 22:39:43 +0100 |
wenzelm |
ml_tactic: non-critical version via proof data and thread data;
|
file |
diff |
annotate
|
| Fri, 28 Mar 2008 20:02:04 +0100 |
wenzelm |
Context.>> : operate on Context.generic;
|
file |
diff |
annotate
|
| Fri, 28 Mar 2008 00:02:54 +0100 |
wenzelm |
reorganized signature of ML_Context;
|
file |
diff |
annotate
|
| Thu, 27 Mar 2008 15:32:15 +0100 |
wenzelm |
eliminated delayed theory setup
|
file |
diff |
annotate
|
| Wed, 26 Mar 2008 22:40:07 +0100 |
wenzelm |
adapted to Context.thread_data interface;
|
file |
diff |
annotate
|
| Mon, 24 Mar 2008 23:34:24 +0100 |
wenzelm |
ML runtime compilation: pass position, tuned signature;
|
file |
diff |
annotate
|
| Sat, 15 Mar 2008 22:07:32 +0100 |
wenzelm |
tuned messages;
|
file |
diff |
annotate
|
| Thu, 24 Jan 2008 23:51:18 +0100 |
wenzelm |
improved apply: handle thread position, apply to context here;
|
file |
diff |
annotate
|
| Tue, 18 Dec 2007 19:54:33 +0100 |
wenzelm |
named some critical sections;
|
file |
diff |
annotate
|
| Fri, 02 Nov 2007 18:53:01 +0100 |
haftmann |
generic tactic Method.intros_tac
|
file |
diff |
annotate
|
| Wed, 01 Aug 2007 16:55:44 +0200 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
| Sat, 28 Jul 2007 20:40:27 +0200 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
| Fri, 27 Jul 2007 21:55:20 +0200 |
wenzelm |
method section scanners: added [[declaration]] syntax, ignore sid-effects of thms;
|
file |
diff |
annotate
|
| Mon, 23 Jul 2007 19:45:44 +0200 |
wenzelm |
eliminated transform_failure (to avoid critical section for main transactions);
|
file |
diff |
annotate
|
| Mon, 23 Jul 2007 14:06:12 +0200 |
wenzelm |
marked some CRITICAL sections (for multithreading);
|
file |
diff |
annotate
|
| Sun, 08 Jul 2007 19:51:58 +0200 |
wenzelm |
replaced exception TableFun/GraphFun.DUPS by TableFun/GraphFun.DUP;
|
file |
diff |
annotate
|
| Thu, 05 Jul 2007 20:01:26 +0200 |
wenzelm |
renamed ObjectLogic.atomize_tac to ObjectLogic.atomize_prems_tac;
|
file |
diff |
annotate
|
| Thu, 05 Jul 2007 00:06:14 +0200 |
wenzelm |
avoid polymorphic equality;
|
file |
diff |
annotate
|
| Tue, 19 Jun 2007 23:15:57 +0200 |
wenzelm |
added raw_tactic;
|
file |
diff |
annotate
|
| Thu, 14 Jun 2007 23:04:40 +0200 |
wenzelm |
method assumption: uniform treatment of prems as legacy feature;
|
file |
diff |
annotate
|
| Wed, 13 Jun 2007 00:01:38 +0200 |
wenzelm |
Basic text: include position;
|
file |
diff |
annotate
|
| Thu, 31 May 2007 23:47:36 +0200 |
wenzelm |
simplified/unified list fold;
|
file |
diff |
annotate
|
| Thu, 24 May 2007 08:37:37 +0200 |
haftmann |
tuned Pure/General/name_space.ML
|
file |
diff |
annotate
|
| Mon, 07 May 2007 00:49:59 +0200 |
wenzelm |
simplified DataFun interfaces;
|
file |
diff |
annotate
|
| Wed, 04 Apr 2007 00:11:18 +0200 |
wenzelm |
tuned comment;
|
file |
diff |
annotate
|
| Sat, 20 Jan 2007 14:09:19 +0100 |
wenzelm |
ML tactic: proper context for compile and runtime;
|
file |
diff |
annotate
|
| Fri, 19 Jan 2007 22:08:27 +0100 |
wenzelm |
removed obsolete Method;
|
file |
diff |
annotate
|
| Fri, 19 Jan 2007 13:09:33 +0100 |
wenzelm |
adapted ML context operations;
|
file |
diff |
annotate
|
| Sat, 30 Dec 2006 16:08:00 +0100 |
wenzelm |
removed conditional combinator;
|
file |
diff |
annotate
|
| Mon, 18 Dec 2006 08:21:35 +0100 |
haftmann |
switched argument order in *.syntax lifters
|
file |
diff |
annotate
|
| Thu, 07 Dec 2006 00:42:04 +0100 |
wenzelm |
reorganized structure Goal vs. Tactic;
|
file |
diff |
annotate
|
| Wed, 29 Nov 2006 15:44:59 +0100 |
wenzelm |
renamed SIMPLE_METHOD' to SIMPLE_METHOD'';
|
file |
diff |
annotate
|
| Wed, 29 Nov 2006 04:11:12 +0100 |
wenzelm |
COMP_INCR;
|
file |
diff |
annotate
|
| Thu, 03 Aug 2006 17:30:43 +0200 |
wenzelm |
moved bires_inst_tac etc. to rule_insts.ML;
|
file |
diff |
annotate
|
| Wed, 02 Aug 2006 22:26:41 +0200 |
wenzelm |
normalized Proof.context/method type aliases;
|
file |
diff |
annotate
|
| Thu, 27 Jul 2006 13:43:01 +0200 |
wenzelm |
moved basic assumption operations from structure ProofContext to Assumption;
|
file |
diff |
annotate
|
| Wed, 12 Jul 2006 21:19:24 +0200 |
wenzelm |
removed duplicate of Tactic.make_elim_preserve;
|
file |
diff |
annotate
|
| Thu, 06 Jul 2006 17:47:34 +0200 |
wenzelm |
added method_i and Source_i;
|
file |
diff |
annotate
|
| Mon, 05 Jun 2006 21:54:24 +0200 |
wenzelm |
assm_tac: try rule termI;
|
file |
diff |
annotate
|
| Thu, 27 Apr 2006 15:06:35 +0200 |
wenzelm |
tuned basic list operators (flat, maps, map_filter);
|
file |
diff |
annotate
|
| Tue, 21 Mar 2006 12:18:18 +0100 |
wenzelm |
moved gen_eq_set to library.ML;
|
file |
diff |
annotate
|
| Sat, 04 Mar 2006 21:10:10 +0100 |
wenzelm |
text: added SelectGoals;
|
file |
diff |
annotate
|
| Wed, 15 Feb 2006 21:34:55 +0100 |
wenzelm |
removed distinct, renamed gen_distinct to distinct;
|
file |
diff |
annotate
|
| Fri, 10 Feb 2006 02:22:43 +0100 |
wenzelm |
syntax: Context.generic;
|
file |
diff |
annotate
|
| Mon, 06 Feb 2006 20:59:06 +0100 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
| Fri, 03 Feb 2006 23:12:28 +0100 |
wenzelm |
canonical member/insert/merge;
|
file |
diff |
annotate
|
| Tue, 31 Jan 2006 18:19:32 +0100 |
wenzelm |
(un)fold: removed '(raw)' option;
|
file |
diff |
annotate
|
| Sun, 29 Jan 2006 19:23:48 +0100 |
wenzelm |
method (un)folded: option '(raw)';
|
file |
diff |
annotate
|
| Sat, 28 Jan 2006 17:28:58 +0100 |
wenzelm |
(un)fold: support object-level rewrites;
|
file |
diff |
annotate
|
| Sat, 21 Jan 2006 23:02:14 +0100 |
wenzelm |
simplified type attribute;
|
file |
diff |
annotate
|
| Thu, 19 Jan 2006 21:22:08 +0100 |
wenzelm |
setup: theory -> theory;
|
file |
diff |
annotate
|
| Tue, 10 Jan 2006 19:33:39 +0100 |
wenzelm |
generic attributes;
|
file |
diff |
annotate
|
| Thu, 22 Dec 2005 00:29:06 +0100 |
wenzelm |
conjunction_tac: single goal;
|
file |
diff |
annotate
|
| Fri, 16 Dec 2005 09:00:11 +0100 |
haftmann |
re-arranged tuples (theory * 'a) to ('a * theory) in Pure
|
file |
diff |
annotate
|
| Wed, 30 Nov 2005 22:52:49 +0100 |
wenzelm |
method 'fact': SIMPLE_METHOD, i.e. insert facts;
|
file |
diff |
annotate
|
| Tue, 22 Nov 2005 19:34:47 +0100 |
wenzelm |
moved multi_resolve(s) to drule.ML;
|
file |
diff |
annotate
|
| Thu, 10 Nov 2005 20:57:11 +0100 |
wenzelm |
renamed Thm.cgoal_of to Thm.cprem_of;
|
file |
diff |
annotate
|
| Fri, 28 Oct 2005 22:28:11 +0200 |
wenzelm |
added fact method;
|
file |
diff |
annotate
|
| Sat, 15 Oct 2005 00:08:06 +0200 |
wenzelm |
added primitive_text, succeed_text;
|
file |
diff |
annotate
|
| Tue, 04 Oct 2005 19:01:37 +0200 |
wenzelm |
minor tweaks for Poplog/ML;
|
file |
diff |
annotate
|
| Thu, 22 Sep 2005 23:43:55 +0200 |
nipkow |
renamed "rules" to "iprover"
|
file |
diff |
annotate
|
| Tue, 20 Sep 2005 08:21:49 +0200 |
haftmann |
slight adaptions to library changes
|
file |
diff |
annotate
|
| Thu, 15 Sep 2005 17:16:56 +0200 |
wenzelm |
TableFun/Symtab: curried lookup and update;
|
file |
diff |
annotate
|
| Tue, 13 Sep 2005 22:19:40 +0200 |
wenzelm |
added cheating, sorry_text (from skip_proofs.ML);
|
file |
diff |
annotate
|
| Thu, 08 Sep 2005 16:09:23 +0200 |
haftmann |
introduces some modern-style AList operations
|
file |
diff |
annotate
|
| Thu, 01 Sep 2005 18:48:50 +0200 |
wenzelm |
curried_lookup/update;
|
file |
diff |
annotate
|
| Thu, 18 Aug 2005 11:17:45 +0200 |
wenzelm |
moved before proof.ML;
|
file |
diff |
annotate
|
| Tue, 19 Jul 2005 17:21:47 +0200 |
wenzelm |
Logic.incr_tvar;
|
file |
diff |
annotate
|
| Mon, 20 Jun 2005 22:14:14 +0200 |
wenzelm |
refl_tac: avoid failure of unification, i.e. confusing trace msg;
|
file |
diff |
annotate
|
| Fri, 17 Jun 2005 18:33:33 +0200 |
wenzelm |
(RAW_)METHOD_CASES: RuleCases.tactic;
|
file |
diff |
annotate
|
| Thu, 09 Jun 2005 12:03:34 +0200 |
wenzelm |
meths: NameSpace.table;
|
file |
diff |
annotate
|
| Tue, 31 May 2005 11:53:36 +0200 |
wenzelm |
renamed cond_extern to extern;
|
file |
diff |
annotate
|
| Tue, 17 May 2005 10:19:44 +0200 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
| Sat, 23 Apr 2005 19:50:40 +0200 |
wenzelm |
removed structure PureIsar;
|
file |
diff |
annotate
|
| Thu, 21 Apr 2005 22:02:06 +0200 |
wenzelm |
superceded by Pure.thy and CPure.thy;
|
file |
diff |
annotate
|
| Thu, 21 Apr 2005 19:13:03 +0200 |
berghofe |
Adapted to new interface of instantiation and unification / matching functions.
|
file |
diff |
annotate
|
| Wed, 13 Apr 2005 18:46:52 +0200 |
wenzelm |
*** MESSAGE REFERS TO PREVIOUS VERSION ***
|
file |
diff |
annotate
|
| Wed, 13 Apr 2005 18:34:22 +0200 |
wenzelm |
*** empty log message ***
|
file |
diff |
annotate
|
| Fri, 04 Mar 2005 15:07:34 +0100 |
skalberg |
Removed practically all references to Library.foldr.
|
file |
diff |
annotate
|
| Thu, 03 Mar 2005 12:43:01 +0100 |
skalberg |
Move towards standard functions.
|
file |
diff |
annotate
|
| Sun, 13 Feb 2005 17:15:14 +0100 |
skalberg |
Deleted Library.option type.
|
file |
diff |
annotate
|
| Mon, 24 Jan 2005 17:56:18 +0100 |
berghofe |
Specific theorems in a named list of theorems can now be referred to
|
file |
diff |
annotate
|
| Mon, 21 Jun 2004 10:25:57 +0200 |
kleing |
Merged in license change from Isabelle2004
|
file |
diff |
annotate
|
| Fri, 07 May 2004 20:33:14 +0200 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
| Fri, 02 Apr 2004 14:08:30 +0200 |
ballarin |
Experimental command for instantiation of locales in proof contexts:
|
file |
diff |
annotate
|
| Tue, 30 Sep 2003 15:13:02 +0200 |
ballarin |
Improvements to Isar/Locales: premises generated by "includes" elements
|
file |
diff |
annotate
|
| Fri, 29 Aug 2003 15:19:02 +0200 |
ballarin |
Methods rule_tac etc support static (Isar) contexts.
|
file |
diff |
annotate
|
| Thu, 17 Oct 2002 10:52:59 +0200 |
paulson |
fixing the cut_tac method to work when there are no instantiations and the
|
file |
diff |
annotate
|
| Mon, 21 Jan 2002 16:15:16 +0100 |
wenzelm |
full_atomize;
|
file |
diff |
annotate
|
| Thu, 06 Dec 2001 00:40:19 +0100 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
| Wed, 05 Dec 2001 03:17:34 +0100 |
wenzelm |
simple version of 'intro' and 'elim' method;
|
file |
diff |
annotate
|
| Tue, 04 Dec 2001 14:26:22 +0100 |
wenzelm |
rules_tac: SELECT_GOAL!!;
|
file |
diff |
annotate
|
| Mon, 03 Dec 2001 21:31:55 +0100 |
wenzelm |
renamed rule_context.ML to context_rules.ML;
|
file |
diff |
annotate
|
| Mon, 03 Dec 2001 21:02:08 +0100 |
wenzelm |
added "rules" method;
|
file |
diff |
annotate
|
| Thu, 29 Nov 2001 01:50:50 +0100 |
wenzelm |
rule context and attributes moved to rule_context.ML;
|
file |
diff |
annotate
|
| Wed, 28 Nov 2001 00:46:26 +0100 |
wenzelm |
theory data: removed obsolete finish method;
|
file |
diff |
annotate
|