Sun, 18 Aug 2024 15:29:03 +0200 |
wenzelm |
tuned: more antiquotations;
|
file |
diff |
annotate
|
Tue, 13 Aug 2024 18:53:24 +0200 |
wenzelm |
tuned: prefer canonical argument order;
|
file |
diff |
annotate
|
Sat, 21 Oct 2023 11:24:34 +0200 |
wenzelm |
more standard simproc_setup using ML antiquotation;
|
file |
diff |
annotate
|
Sat, 22 Jun 2019 07:18:55 +0000 |
haftmann |
streamlined setup for linear algebra, particularly removed redundant rule declarations
|
file |
diff |
annotate
|
Fri, 04 Jan 2019 23:22:53 +0100 |
wenzelm |
isabelle update -u control_cartouches;
|
file |
diff |
annotate
|
Wed, 06 Dec 2017 20:43:09 +0100 |
wenzelm |
prefer control symbol antiquotations;
|
file |
diff |
annotate
|
Sat, 02 Dec 2017 16:50:53 +0000 |
haftmann |
cleaned up and tuned
|
file |
diff |
annotate
|
Fri, 08 Apr 2016 20:15:20 +0200 |
wenzelm |
eliminated unused simproc identifier;
|
file |
diff |
annotate
|
Wed, 09 Sep 2015 20:57:21 +0200 |
wenzelm |
simplified simproc programming interfaces;
|
file |
diff |
annotate
|
Mon, 27 Jul 2015 17:44:55 +0200 |
wenzelm |
tuned signature;
|
file |
diff |
annotate
|
Fri, 10 Apr 2015 11:31:10 +0200 |
wenzelm |
tuned signature;
|
file |
diff |
annotate
|
Fri, 06 Mar 2015 15:58:56 +0100 |
wenzelm |
Thm.cterm_of and Thm.ctyp_of operate on local context;
|
file |
diff |
annotate
|
Wed, 04 Mar 2015 22:05:01 +0100 |
wenzelm |
clarified signature;
|
file |
diff |
annotate
|
Wed, 04 Mar 2015 19:53:18 +0100 |
wenzelm |
tuned signature -- prefer qualified names;
|
file |
diff |
annotate
|
Mon, 04 Nov 2013 20:10:06 +0100 |
haftmann |
streamlined setup of linear arithmetic
|
file |
diff |
annotate
|
Thu, 18 Apr 2013 17:07:01 +0200 |
wenzelm |
simplifier uses proper Proof.context instead of historic type simpset;
|
file |
diff |
annotate
|
Fri, 30 Mar 2012 09:08:29 +0200 |
huffman |
add constant pred_numeral k = numeral k - (1::nat);
|
file |
diff |
annotate
|
Sun, 25 Mar 2012 20:15:39 +0200 |
huffman |
merged fork with new numeral representation (see NEWS)
|
file |
diff |
annotate
|
Wed, 29 Jun 2011 18:12:34 +0200 |
wenzelm |
modernized some simproc setup;
|
file |
diff |
annotate
|
Fri, 13 May 2011 23:58:40 +0200 |
wenzelm |
clarified map_simpset versus Simplifier.map_simpset_global;
|
file |
diff |
annotate
|
Sat, 28 Aug 2010 16:14:32 +0200 |
haftmann |
formerly unnamed infix equality now named HOL.eq
|
file |
diff |
annotate
|
Thu, 26 Aug 2010 20:42:09 +0200 |
wenzelm |
Fast_Lin_Arith.number_of: more conventional merge that prefers the left side -- note that former ordering wrt. serial numbers makes it depend on accidental load order;
|
file |
diff |
annotate
|
Wed, 25 Aug 2010 18:36:22 +0200 |
wenzelm |
renamed Simplifier.simproc(_i) to Simplifier.simproc_global(_i) to emphasize that this is not the real thing;
|
file |
diff |
annotate
|
Sat, 15 May 2010 21:50:05 +0200 |
wenzelm |
less pervasive names from structure Thm;
|
file |
diff |
annotate
|
Fri, 19 Feb 2010 14:47:01 +0100 |
haftmann |
moved remaning class operations from Algebras.thy to Groups.thy
|
file |
diff |
annotate
|
Wed, 10 Feb 2010 14:12:04 +0100 |
haftmann |
moved less_eq, less to Orderings.thy; moved abs, sgn to Groups.thy
|
file |
diff |
annotate
|
Fri, 05 Feb 2010 14:33:50 +0100 |
haftmann |
more consistent naming of type classes involving orderings (and lattices) -- c.f. NEWS
|
file |
diff |
annotate
|
Thu, 28 Jan 2010 11:48:49 +0100 |
haftmann |
new theory Algebras.thy for generic algebraic structures
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 19:09:47 +0100 |
haftmann |
moved theory Divides after theory Nat_Numeral; tuned some proof texts
|
file |
diff |
annotate
|
Fri, 18 Sep 2009 09:07:50 +0200 |
haftmann |
tuned const_name antiquotations
|
file |
diff |
annotate
|
Mon, 08 Jun 2009 22:29:37 +0200 |
boehmes |
fast_lin_arith uses proper multiplication instead of unfolding to additions
|
file |
diff |
annotate
|
Mon, 11 May 2009 15:57:29 +0200 |
haftmann |
qualified names for Lin_Arith tactics and simprocs
|
file |
diff |
annotate
|
Mon, 11 May 2009 15:18:32 +0200 |
haftmann |
tuned interface of Lin_Arith
|
file |
diff |
annotate
|
Sat, 09 May 2009 09:17:29 +0200 |
haftmann |
interface changes in linarith.ML
|
file |
diff |
annotate
|
Fri, 08 May 2009 09:48:07 +0200 |
haftmann |
modules numeral_simprocs, nat_numeral_simprocs; proper structures for numeral simprocs
|
file |
diff |
annotate
|
Wed, 29 Apr 2009 17:15:01 -0700 |
huffman |
reimplement reorientation simproc using theory data
|
file |
diff |
annotate
|
Mon, 30 Mar 2009 12:07:59 -0700 |
huffman |
simplify theorem references
|
file |
diff |
annotate
|
Thu, 26 Mar 2009 11:33:50 -0700 |
huffman |
parameterize assoc_fold with is_numeral predicate
|
file |
diff |
annotate
|
Mon, 23 Mar 2009 19:01:15 +0100 |
haftmann |
structure LinArith now named Lin_Arith
|
file |
diff |
annotate
|
Fri, 13 Mar 2009 19:17:57 +0100 |
haftmann |
moved some generic nonsense to arith_data.ML
|
file |
diff |
annotate
|
Thu, 12 Mar 2009 18:01:26 +0100 |
haftmann |
vague cleanup in arith proof tools setup: deleted dead code, more proper structures, clearer arrangement
|
file |
diff |
annotate
|
Wed, 31 Dec 2008 15:30:10 +0100 |
wenzelm |
moved term order operations to structure TermOrd (cf. Pure/term_ord.ML);
|
file |
diff |
annotate
|
Wed, 03 Dec 2008 15:58:44 +0100 |
haftmann |
made repository layout more coherent with logical distribution structure; stripped some $Id$s
|
file |
diff |
annotate
| base
|