Sat, 11 Aug 2012 22:17:46 +0200 |
wenzelm |
faster compilation of ML with antiquotations: static ML_context is bound once in auxiliary structure Isabelle;
|
file |
diff |
annotate
|
Thu, 15 Mar 2012 22:08:53 +0100 |
wenzelm |
declare command keywords via theory header, including strict checking outside Pure;
|
file |
diff |
annotate
|
Sun, 27 Nov 2011 23:10:19 +0100 |
wenzelm |
more antiquotations;
|
file |
diff |
annotate
|
Wed, 23 Nov 2011 22:59:39 +0100 |
wenzelm |
modernized some old-style infix operations, which were left over from the time of ML proof scripts;
|
file |
diff |
annotate
|
Sun, 20 Nov 2011 13:29:12 +0100 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
Mon, 27 Jun 2011 16:53:31 +0200 |
wenzelm |
ML antiquotations are managed as theory data, with proper name space and entity markup;
|
file |
diff |
annotate
|
Sun, 15 May 2011 17:45:53 +0200 |
wenzelm |
simplified/unified method_setup/attribute_setup;
|
file |
diff |
annotate
|
Sat, 14 May 2011 13:32:33 +0200 |
wenzelm |
simplified BLAST_DATA;
|
file |
diff |
annotate
|
Sat, 14 May 2011 11:42:43 +0200 |
wenzelm |
modernized functor names;
|
file |
diff |
annotate
|
Fri, 13 May 2011 23:58:40 +0200 |
wenzelm |
clarified map_simpset versus Simplifier.map_simpset_global;
|
file |
diff |
annotate
|
Fri, 13 May 2011 22:55:00 +0200 |
wenzelm |
proper Proof.context for classical tactics;
|
file |
diff |
annotate
|
Tue, 26 Apr 2011 21:27:01 +0200 |
wenzelm |
simplified Blast setup;
|
file |
diff |
annotate
|
Fri, 22 Apr 2011 15:05:04 +0200 |
wenzelm |
misc tuning and simplification;
|
file |
diff |
annotate
|
Fri, 22 Apr 2011 14:30:32 +0200 |
wenzelm |
proper context for Quantifier1 simprocs (avoid bad ProofContext.init_global from abc655166d61);
|
file |
diff |
annotate
|
Fri, 22 Apr 2011 13:58:13 +0200 |
wenzelm |
modernized Quantifier1 simproc setup;
|
file |
diff |
annotate
|
Fri, 22 Apr 2011 12:46:48 +0200 |
wenzelm |
clarified simpset setup;
|
file |
diff |
annotate
|
Wed, 23 Feb 2011 11:23:26 +0100 |
noschinl |
setup case_product attribute in HOL and FOL
|
file |
diff |
annotate
|
Fri, 18 Feb 2011 17:03:30 +0100 |
wenzelm |
modernized specifications;
|
file |
diff |
annotate
|
Mon, 20 Dec 2010 16:44:33 +0100 |
wenzelm |
proper identifiers for consts and types;
|
file |
diff |
annotate
|
Wed, 12 May 2010 16:44:49 +0200 |
wenzelm |
modernized specifications;
|
file |
diff |
annotate
|
Fri, 16 Apr 2010 21:28:09 +0200 |
wenzelm |
replaced generic 'hide' command by more conventional 'hide_class', 'hide_type', 'hide_const', 'hide_fact' -- frees some popular keywords;
|
file |
diff |
annotate
|
Sat, 30 Jan 2010 17:01:01 +0100 |
berghofe |
Adapted to changes in setup of cases method.
|
file |
diff |
annotate
|
Sun, 10 Jan 2010 18:41:07 +0100 |
berghofe |
Adapted to changes in setup of induct method.
|
file |
diff |
annotate
|
Sat, 17 Oct 2009 14:43:18 +0200 |
wenzelm |
eliminated hard tabulators, guessing at each author's individual tab-width;
|
file |
diff |
annotate
|
Wed, 29 Jul 2009 00:09:14 +0200 |
wenzelm |
removed old global get_claset/map_claset;
|
file |
diff |
annotate
|
Fri, 24 Jul 2009 21:21:45 +0200 |
wenzelm |
renamed functor BlastFun to Blast, require explicit theory;
|
file |
diff |
annotate
|
Fri, 24 Jul 2009 12:33:00 +0200 |
wenzelm |
renamed functor InductFun to Induct;
|
file |
diff |
annotate
|
Thu, 09 Jul 2009 22:09:58 +0200 |
wenzelm |
removed obsolete CVS Ids;
|
file |
diff |
annotate
|
Mon, 16 Mar 2009 18:24:30 +0100 |
wenzelm |
simplified method setup;
|
file |
diff |
annotate
|
Thu, 20 Nov 2008 00:03:47 +0100 |
wenzelm |
Pure syntax: more coherent treatment of aprop, permanent TERM and &&&;
|
file |
diff |
annotate
|
Tue, 28 Oct 2008 11:03:07 +0100 |
ballarin |
Removed 'includes meta_term_syntax' and 'includes meta_conjunction_syntax'.
|
file |
diff |
annotate
|
Fri, 15 Aug 2008 15:50:44 +0200 |
wenzelm |
Args.name_source(_position) for proper position information;
|
file |
diff |
annotate
|
Wed, 13 Aug 2008 20:57:18 +0200 |
wenzelm |
tuned document;
|
file |
diff |
annotate
|
Mon, 16 Jun 2008 22:13:39 +0200 |
wenzelm |
pervasive RuleInsts;
|
file |
diff |
annotate
|
Sat, 14 Jun 2008 23:20:02 +0200 |
wenzelm |
removed unused excluded_middle_tac;
|
file |
diff |
annotate
|
Tue, 10 Jun 2008 16:43:01 +0200 |
wenzelm |
eliminated obsolete case_split_thm -- use case_split;
|
file |
diff |
annotate
|
Sat, 29 Mar 2008 22:55:49 +0100 |
wenzelm |
purely functional setup of claset/simpset/clasimpset;
|
file |
diff |
annotate
|
Wed, 26 Mar 2008 22:40:01 +0100 |
wenzelm |
pass imp_elim, swap to classical prover;
|
file |
diff |
annotate
|
Sat, 15 Mar 2008 22:07:25 +0100 |
wenzelm |
added lemmas from simpdata.ML;
|
file |
diff |
annotate
|
Thu, 04 Oct 2007 14:42:47 +0200 |
wenzelm |
moved Pure/Isar/induct_attrib.ML and Provers/induct_method.ML to Tools/induct.ML;
|
file |
diff |
annotate
|
Tue, 31 Jul 2007 21:19:18 +0200 |
wenzelm |
moved classical tools from theory IFOL to FOL;
|
file |
diff |
annotate
|
Thu, 31 May 2007 14:34:05 +0200 |
wenzelm |
tuned header;
|
file |
diff |
annotate
|
Sat, 20 Jan 2007 14:09:27 +0100 |
wenzelm |
tuned ML setup;
|
file |
diff |
annotate
|
Sun, 26 Nov 2006 23:43:53 +0100 |
wenzelm |
converted legacy ML scripts;
|
file |
diff |
annotate
|
Thu, 27 Jul 2006 13:43:00 +0200 |
wenzelm |
tuned proofs;
|
file |
diff |
annotate
|
Sat, 28 Jan 2006 17:28:50 +0100 |
wenzelm |
tuned proofs;
|
file |
diff |
annotate
|
Fri, 06 Jan 2006 18:18:13 +0100 |
wenzelm |
simplified EqSubst setup;
|
file |
diff |
annotate
|
Fri, 06 Jan 2006 15:18:20 +0100 |
wenzelm |
tuned EqSubst setup;
|
file |
diff |
annotate
|
Sat, 31 Dec 2005 21:49:39 +0100 |
wenzelm |
removed obsolete cla_dist_concl;
|
file |
diff |
annotate
|
Fri, 30 Dec 2005 16:56:56 +0100 |
wenzelm |
provide cla_dist_concl;
|
file |
diff |
annotate
|
Fri, 23 Dec 2005 18:36:26 +0100 |
wenzelm |
removed obsolete induct_atomize_old;
|
file |
diff |
annotate
|
Thu, 22 Dec 2005 00:28:34 +0100 |
wenzelm |
updated auxiliary facts for induct method;
|
file |
diff |
annotate
|
Fri, 17 Jun 2005 16:12:49 +0200 |
haftmann |
migrated theory headers to new format
|
file |
diff |
annotate
|
Tue, 01 Feb 2005 18:01:57 +0100 |
paulson |
the new subst tactic, by Lucas Dixon
|
file |
diff |
annotate
|
Thu, 08 Jul 2004 19:32:46 +0200 |
wenzelm |
removed obsolete dependency;
|
file |
diff |
annotate
|
Wed, 20 Aug 2003 11:04:17 +0200 |
paulson |
new case_tac method
|
file |
diff |
annotate
|
Tue, 01 Jul 2003 10:50:26 +0200 |
paulson |
moved some lemmas here from ZF
|
file |
diff |
annotate
|
Fri, 30 Aug 2002 16:42:45 +0200 |
paulson |
removal of blast.overloaded
|
file |
diff |
annotate
|
Wed, 05 Dec 2001 02:59:49 +0100 |
wenzelm |
removed declaration of disjI1, disjI2 (already done in IFOL);
|
file |
diff |
annotate
|
Wed, 28 Nov 2001 00:37:08 +0100 |
wenzelm |
tuned;
|
file |
diff |
annotate
|