Thu, 31 May 2007 20:55:29 +0200 |
wenzelm |
moved IsaPlanner from Provers to Tools;
|
file |
diff |
annotate
|
Thu, 31 May 2007 18:16:51 +0200 |
wenzelm |
proper loading of ML files;
|
file |
diff |
annotate
|
Sat, 19 May 2007 19:08:42 +0200 |
chaieb |
added a set of NNF normalization lemmas and nnf_conv
|
file |
diff |
annotate
|
Thu, 17 May 2007 19:49:16 +0200 |
haftmann |
tuned
|
file |
diff |
annotate
|
Sun, 06 May 2007 21:49:24 +0200 |
haftmann |
dropped HOL.ML
|
file |
diff |
annotate
|
Fri, 20 Apr 2007 11:21:42 +0200 |
haftmann |
Isar definitions are now added explicitly to code theorem table
|
file |
diff |
annotate
|
Tue, 20 Mar 2007 15:52:38 +0100 |
haftmann |
added class "default" and expansion axioms for undefined
|
file |
diff |
annotate
|
Tue, 20 Mar 2007 08:27:15 +0100 |
haftmann |
explizit "type" superclass
|
file |
diff |
annotate
|
Sun, 18 Mar 2007 01:50:05 +0100 |
dixon |
TrueElim and notTrueElim tested and added as safe elim rules.
|
file |
diff |
annotate
|
Fri, 16 Mar 2007 16:40:49 +0100 |
dixon |
removed safe elim flag of trueElim and notFalseElim for testing.
|
file |
diff |
annotate
|
Fri, 16 Mar 2007 16:37:52 +0100 |
dixon |
added safe intro rules for removing "True" subgoals as well as "~ False" ones.
|
file |
diff |
annotate
|
Wed, 28 Feb 2007 22:05:43 +0100 |
wenzelm |
tuned ML setup;
|
file |
diff |
annotate
|
Wed, 31 Jan 2007 16:05:10 +0100 |
haftmann |
dropped lemma duplicates in HOL.thy
|
file |
diff |
annotate
|
Sat, 20 Jan 2007 14:09:12 +0100 |
wenzelm |
tuned ML setup;
|
file |
diff |
annotate
|
Wed, 06 Dec 2006 01:12:42 +0100 |
wenzelm |
removed legacy ML bindings;
|
file |
diff |
annotate
|
Mon, 27 Nov 2006 13:42:39 +0100 |
haftmann |
moved order arities for fun and bool to Fun/Orderings
|
file |
diff |
annotate
|
Sun, 26 Nov 2006 18:07:16 +0100 |
wenzelm |
updated (binder) syntax/notation;
|
file |
diff |
annotate
|
Thu, 23 Nov 2006 22:38:28 +0100 |
wenzelm |
tuned proofs;
|
file |
diff |
annotate
|
Thu, 23 Nov 2006 20:34:21 +0100 |
wenzelm |
prefer antiquotations over LaTeX macros;
|
file |
diff |
annotate
|
Thu, 23 Nov 2006 13:32:19 +0100 |
webertj |
typo in comment fixed
|
file |
diff |
annotate
|
Sat, 18 Nov 2006 00:20:17 +0100 |
haftmann |
tuned
|
file |
diff |
annotate
|
Fri, 17 Nov 2006 02:20:03 +0100 |
wenzelm |
more robust syntax for definition/abbreviation/notation;
|
file |
diff |
annotate
|
Wed, 08 Nov 2006 19:48:35 +0100 |
haftmann |
moved lemma eq_neq_eq_imp_neq to HOL
|
file |
diff |
annotate
|
Tue, 07 Nov 2006 14:29:57 +0100 |
wenzelm |
tuned hypsubst setup;
|
file |
diff |
annotate
|
Tue, 07 Nov 2006 11:47:57 +0100 |
wenzelm |
renamed 'const_syntax' to 'notation';
|
file |
diff |
annotate
|
Sun, 05 Nov 2006 21:44:32 +0100 |
wenzelm |
Sign.const_syntax_name;
|
file |
diff |
annotate
|
Fri, 03 Nov 2006 14:22:37 +0100 |
haftmann |
simplified reasoning tools setup
|
file |
diff |
annotate
|
Tue, 31 Oct 2006 09:28:55 +0100 |
haftmann |
added Equals_conv
|
file |
diff |
annotate
|
Mon, 16 Oct 2006 14:07:31 +0200 |
haftmann |
moved HOL code generator setup to Code_Generator
|
file |
diff |
annotate
|
Fri, 13 Oct 2006 12:32:44 +0200 |
haftmann |
lifted claset setup from ML to Isar level
|
file |
diff |
annotate
|
Wed, 11 Oct 2006 14:51:24 +0200 |
haftmann |
cleaned up HOL bootstrap
|
file |
diff |
annotate
|
Tue, 10 Oct 2006 10:35:24 +0200 |
haftmann |
cleanup basic HOL bootstrap
|
file |
diff |
annotate
|
Mon, 02 Oct 2006 23:00:49 +0200 |
haftmann |
improved serialization for arbitrary
|
file |
diff |
annotate
|
Thu, 28 Sep 2006 23:42:30 +0200 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
Wed, 27 Sep 2006 21:49:34 +0200 |
wenzelm |
proper const_syntax for uminus, abs;
|
file |
diff |
annotate
|
Tue, 26 Sep 2006 13:34:16 +0200 |
haftmann |
renamed 0 and 1 to HOL.zero and HOL.one respectivly; introduced corresponding syntactic classes
|
file |
diff |
annotate
|
Mon, 25 Sep 2006 17:04:14 +0200 |
haftmann |
added 'undefined' serializer
|
file |
diff |
annotate
|
Tue, 19 Sep 2006 15:21:44 +0200 |
haftmann |
introduced syntactic classes; moved some setup to Pure/codegen, Pure/nbe or OperationalEquality.thy
|
file |
diff |
annotate
|
Fri, 01 Sep 2006 08:36:51 +0200 |
haftmann |
final syntax for some Isar code generator keywords
|
file |
diff |
annotate
|
Mon, 14 Aug 2006 13:46:06 +0200 |
haftmann |
simplified code generator setup
|
file |
diff |
annotate
|
Thu, 27 Jul 2006 13:43:00 +0200 |
wenzelm |
tuned proofs;
|
file |
diff |
annotate
|
Fri, 21 Jul 2006 11:34:01 +0200 |
berghofe |
- Added new "undefined" constant
|
file |
diff |
annotate
|
Fri, 07 Jul 2006 09:31:57 +0200 |
nipkow |
made evaluation_conv and normalization_conv visible.
|
file |
diff |
annotate
|
Wed, 05 Jul 2006 16:24:28 +0200 |
paulson |
removed the "tagging" feature
|
file |
diff |
annotate
|
Fri, 30 Jun 2006 18:26:22 +0200 |
nipkow |
normalization uses refl now
|
file |
diff |
annotate
|
Thu, 29 Jun 2006 13:52:28 +0200 |
nipkow |
new method "normalization"
|
file |
diff |
annotate
|
Wed, 14 Jun 2006 12:14:42 +0200 |
haftmann |
slight adaption for code generator
|
file |
diff |
annotate
|
Tue, 06 Jun 2006 20:42:25 +0200 |
wenzelm |
quoted "if";
|
file |
diff |
annotate
|
Tue, 16 May 2006 21:33:01 +0200 |
wenzelm |
tuned concrete syntax -- abbreviation/const_syntax;
|
file |
diff |
annotate
|
Tue, 09 May 2006 14:18:40 +0200 |
haftmann |
introduced characters for code generator; some improved code lemmas for some list functions
|
file |
diff |
annotate
|
Tue, 09 May 2006 10:09:17 +0200 |
haftmann |
different object logic setup for CodegenTheorems
|
file |
diff |
annotate
|
Tue, 02 May 2006 20:42:32 +0200 |
wenzelm |
replaced syntax/translations by abbreviation;
|
file |
diff |
annotate
|
Thu, 06 Apr 2006 16:11:30 +0200 |
haftmann |
adapted for definitional code generation
|
file |
diff |
annotate
|
Fri, 10 Mar 2006 15:33:48 +0100 |
haftmann |
renamed HOL + - * etc. to HOL.plus HOL.minus HOL.times etc.
|
file |
diff |
annotate
|
Thu, 02 Mar 2006 18:49:13 +0100 |
paulson |
moved the "use" directive
|
file |
diff |
annotate
|
Wed, 01 Mar 2006 06:08:12 +0100 |
mengj |
Added setup for "atpset" (a rule set for ATPs).
|
file |
diff |
annotate
|
Sat, 25 Feb 2006 15:19:47 +0100 |
haftmann |
improved codegen bootstrap
|
file |
diff |
annotate
|
Wed, 22 Feb 2006 22:18:32 +0100 |
wenzelm |
simplified Pure conjunction;
|
file |
diff |
annotate
|
Tue, 14 Feb 2006 17:07:48 +0100 |
haftmann |
added theory of executable rational numbers
|
file |
diff |
annotate
|
Wed, 01 Feb 2006 19:19:32 +0100 |
berghofe |
Added "evaluation" method and oracle.
|
file |
diff |
annotate
|
Tue, 31 Jan 2006 16:26:18 +0100 |
haftmann |
added serialization for arbitrary
|
file |
diff |
annotate
|
Sun, 29 Jan 2006 19:23:38 +0100 |
wenzelm |
declare 'defn' rules;
|
file |
diff |
annotate
|
Mon, 23 Jan 2006 14:07:52 +0100 |
haftmann |
removed problematic keyword 'atom'
|
file |
diff |
annotate
|
Thu, 19 Jan 2006 21:22:08 +0100 |
wenzelm |
setup: theory -> theory;
|
file |
diff |
annotate
|
Tue, 17 Jan 2006 16:36:57 +0100 |
haftmann |
substantial improvements in code generator
|
file |
diff |
annotate
|
Mon, 16 Jan 2006 21:55:14 +0100 |
wenzelm |
declare the1_equality [elim?];
|
file |
diff |
annotate
|
Sun, 15 Jan 2006 19:58:51 +0100 |
wenzelm |
prefer ex1I over ex_ex1I in single-step reasoning;
|
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:36 +0100 |
wenzelm |
structure ProjectRule;
|
file |
diff |
annotate
|
Thu, 27 Oct 2005 13:54:38 +0200 |
wenzelm |
alternative iff syntax for equality on booleans, with print_mode 'iff';
|
file |
diff |
annotate
|
Sun, 25 Sep 2005 20:19:31 +0200 |
berghofe |
eq_codegen now ensures that code for bool type is generated.
|
file |
diff |
annotate
|
Thu, 22 Sep 2005 23:56:15 +0200 |
nipkow |
renamed rules to iprover
|
file |
diff |
annotate
|
Sat, 17 Sep 2005 18:11:19 +0200 |
wenzelm |
added code generator setup (from Main.thy);
|
file |
diff |
annotate
|
Thu, 15 Sep 2005 11:15:52 +0200 |
paulson |
the experimental tagging system, and the usual tidying
|
file |
diff |
annotate
|
Tue, 06 Sep 2005 16:59:48 +0200 |
wenzelm |
axclass: name space prefix is now "c_class" instead of just "c";
|
file |
diff |
annotate
|
Wed, 31 Aug 2005 15:46:34 +0200 |
wenzelm |
simp_implies: proper named infix;
|
file |
diff |
annotate
|
Tue, 02 Aug 2005 16:50:55 +0200 |
ballarin |
Turned simp_implies into binary operator.
|
file |
diff |
annotate
|
Tue, 12 Jul 2005 17:56:03 +0200 |
avigad |
added lemmas to OrderedGroup.thy (reasoning about signs, absolute value, triangle inequalities)
|
file |
diff |
annotate
|
Fri, 01 Jul 2005 13:54:12 +0200 |
berghofe |
Implemented trick (due to Tobias Nipkow) for fine-tuning simplification
|
file |
diff |
annotate
|
Tue, 28 Jun 2005 15:27:45 +0200 |
paulson |
Constant "If" is now local
|
file |
diff |
annotate
|
Fri, 17 Jun 2005 16:12:49 +0200 |
haftmann |
migrated theory headers to new format
|
file |
diff |
annotate
|
Tue, 31 May 2005 11:53:12 +0200 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
Sun, 22 May 2005 16:51:07 +0200 |
wenzelm |
Simplifier already setup in Pure;
|
file |
diff |
annotate
|
Thu, 21 Apr 2005 22:02:06 +0200 |
wenzelm |
superceded by Pure.thy and CPure.thy;
|
file |
diff |
annotate
|
Thu, 07 Apr 2005 13:29:41 +0200 |
paulson |
new meta-level rules
|
file |
diff |
annotate
|
Tue, 05 Apr 2005 13:05:20 +0200 |
paulson |
arg_cong2 by Norbert Voelker
|
file |
diff |
annotate
|
Thu, 03 Mar 2005 12:43:01 +0100 |
skalberg |
Move towards standard functions.
|
file |
diff |
annotate
|
Thu, 10 Feb 2005 18:51:12 +0100 |
nipkow |
Moved oderings from HOL into the new Orderings.thy
|
file |
diff |
annotate
|
Tue, 01 Feb 2005 18:01:57 +0100 |
paulson |
the new subst tactic, by Lucas Dixon
|
file |
diff |
annotate
|
Sat, 18 Dec 2004 17:14:33 +0100 |
schirmer |
added simproc for Let
|
file |
diff |
annotate
|
Wed, 15 Dec 2004 10:19:01 +0100 |
paulson |
removal of HOL_Lemmas
|
file |
diff |
annotate
|
Tue, 07 Dec 2004 16:15:05 +0100 |
paulson |
proof of subst by S Merz
|
file |
diff |
annotate
|
Thu, 02 Dec 2004 12:28:09 +0100 |
nipkow |
Fixed print translation for ALL x > y etc
|
file |
diff |
annotate
|
Thu, 02 Dec 2004 11:59:34 +0100 |
nipkow |
added ALL print-translation for > and >=.
|
file |
diff |
annotate
|
Thu, 02 Dec 2004 11:42:01 +0100 |
nipkow |
Added "ALL x > y" and relatives.
|
file |
diff |
annotate
|
Wed, 01 Dec 2004 18:11:13 +0100 |
nipkow |
Added > and >= sugar
|
file |
diff |
annotate
|
Mon, 15 Nov 2004 18:21:34 +0100 |
paulson |
removed a "clone" (duplicate code)
|
file |
diff |
annotate
|
Fri, 10 Sep 2004 20:04:14 +0200 |
nipkow |
Added antisymmetry simproc
|
file |
diff |
annotate
|
Wed, 18 Aug 2004 11:09:40 +0200 |
nipkow |
import -> imports
|
file |
diff |
annotate
|
Mon, 16 Aug 2004 14:22:27 +0200 |
nipkow |
New theory header syntax.
|
file |
diff |
annotate
|
Tue, 03 Aug 2004 14:47:51 +0200 |
ballarin |
New transitivity reasoners for transitivity only and quasi orders.
|
file |
diff |
annotate
|
Wed, 28 Jul 2004 10:49:29 +0200 |
paulson |
conversion of Hyperreal/MacLaurin_lemmas to Isar script
|
file |
diff |
annotate
|
Mon, 21 Jun 2004 10:25:57 +0200 |
kleing |
Merged in license change from Isabelle2004
|
file |
diff |
annotate
|
Tue, 01 Jun 2004 12:33:50 +0200 |
wenzelm |
removed obsolete sort 'logic';
|
file |
diff |
annotate
|
Fri, 14 May 2004 16:53:15 +0200 |
paulson |
new atomize theorem
|
file |
diff |
annotate
|
Sat, 01 May 2004 21:59:12 +0200 |
wenzelm |
_index1: accomodate improved indexed syntax;
|
file |
diff |
annotate
|
Fri, 16 Apr 2004 13:52:43 +0200 |
wenzelm |
simplified ML code for setsubgoaler;
|
file |
diff |
annotate
|
Wed, 14 Apr 2004 14:13:05 +0200 |
kleing |
use more symbols in HTML output
|
file |
diff |
annotate
|
Mon, 08 Mar 2004 12:16:57 +0100 |
ballarin |
Added documentation for transitivity solver setup.
|
file |
diff |
annotate
|
Thu, 04 Mar 2004 12:06:07 +0100 |
paulson |
new material from Avigad, and simplified treatment of division by 0
|
file |
diff |
annotate
|
Thu, 19 Feb 2004 15:57:34 +0100 |
ballarin |
Efficient, graph-based reasoner for linear and partial orders.
|
file |
diff |
annotate
|
Tue, 27 Jan 2004 15:39:51 +0100 |
paulson |
replacing HOL/Real/PRat, PNat by the rational number development
|
file |
diff |
annotate
|
Mon, 26 Jan 2004 10:34:02 +0100 |
schirmer |
* Support for raw latex output in control symbols: \<^raw...>
|
file |
diff |
annotate
|
Wed, 14 Jan 2004 07:53:27 +0100 |
kleing |
print translation for ALL x <= n. P x
|
file |
diff |
annotate
|
Mon, 15 Dec 2003 16:38:25 +0100 |
paulson |
more general lemmas for Ring_and_Field
|
file |
diff |
annotate
|
Wed, 29 Oct 2003 11:50:26 +0100 |
berghofe |
Tuned proof of choice_eq.
|
file |
diff |
annotate
|