Tue, 13 Sep 2011 17:07:33 -0700 |
huffman |
tuned proofs
|
file |
diff |
annotate
|
Mon, 08 Aug 2011 17:23:15 +0200 |
wenzelm |
misc tuning -- eliminated old-fashioned rep_thm;
|
file |
diff |
annotate
|
Wed, 03 Aug 2011 23:21:52 +0200 |
haftmann |
tuned
|
file |
diff |
annotate
|
Sat, 16 Jul 2011 22:04:02 +0200 |
haftmann |
consolidated bot and top classes, tuned notation
|
file |
diff |
annotate
|
Wed, 13 Jul 2011 23:49:56 +0200 |
haftmann |
uniqueness lemmas for bot and top
|
file |
diff |
annotate
|
Wed, 13 Jul 2011 19:43:12 +0200 |
haftmann |
moved lemmas bot_less and less_top to classes bot and top respectively
|
file |
diff |
annotate
|
Wed, 13 Jul 2011 19:40:18 +0200 |
haftmann |
tightened specification of classes bot and top: uniqueness of top and bot elements
|
file |
diff |
annotate
|
Wed, 29 Jun 2011 21:34:16 +0200 |
wenzelm |
tuned signature;
|
file |
diff |
annotate
|
Wed, 29 Jun 2011 20:39:41 +0200 |
wenzelm |
simplified/unified Simplifier.mk_solver;
|
file |
diff |
annotate
|
Fri, 13 May 2011 23:58:40 +0200 |
wenzelm |
clarified map_simpset versus Simplifier.map_simpset_global;
|
file |
diff |
annotate
|
Fri, 08 Apr 2011 14:20:57 +0200 |
wenzelm |
discontinued special treatment of structure Mixfix;
|
file |
diff |
annotate
|
Fri, 08 Apr 2011 13:31:16 +0200 |
wenzelm |
explicit structure Syntax_Trans;
|
file |
diff |
annotate
|
Wed, 08 Dec 2010 15:05:46 +0100 |
haftmann |
bot comes before top, inf before sup etc.
|
file |
diff |
annotate
|
Wed, 08 Dec 2010 14:52:23 +0100 |
haftmann |
nice syntax for lattice INFI, SUPR;
|
file |
diff |
annotate
|
Wed, 08 Dec 2010 13:34:50 +0100 |
haftmann |
primitive definitions of bot/top/inf/sup for bool and fun are named with canonical suffix `_def` rather than `_eq`
|
file |
diff |
annotate
|
Fri, 27 Aug 2010 10:56:46 +0200 |
haftmann |
formerly unnamed infix conjunction and disjunction now named HOL.conj and HOL.disj
|
file |
diff |
annotate
|
Thu, 26 Aug 2010 20:51:17 +0200 |
haftmann |
formerly unnamed infix impliciation now named HOL.implies
|
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
|
Tue, 24 Aug 2010 14:41:37 +0200 |
hoelzl |
moved generic lemmas in Probability to HOL
|
file |
diff |
annotate
|
Mon, 23 Aug 2010 14:21:57 +0200 |
blanchet |
"no_atp" fact that leads to unsound proofs in Sledgehammer
|
file |
diff |
annotate
|
Mon, 12 Jul 2010 10:48:37 +0200 |
haftmann |
dropped superfluous [code del]s
|
file |
diff |
annotate
|
Mon, 17 May 2010 23:54:15 +0200 |
wenzelm |
prefer structure Keyword, Parse, Parse_Spec, Outer_Syntax;
|
file |
diff |
annotate
|
Tue, 04 May 2010 08:55:43 +0200 |
haftmann |
locale predicates of classes carry a mandatory "class" prefix
|
file |
diff |
annotate
|
Thu, 18 Mar 2010 12:58:52 +0100 |
blanchet |
now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
|
file |
diff |
annotate
|
Thu, 04 Mar 2010 18:42:39 +0100 |
hoelzl |
Add dense_le, dense_le_bounded, field_le_mult_one_interval.
|
file |
diff |
annotate
|
Thu, 25 Feb 2010 22:32:09 +0100 |
wenzelm |
more antiquotations;
|
file |
diff |
annotate
|
Mon, 22 Feb 2010 15:53:18 +0100 |
haftmann |
distributed theory Algebras to theories Groups and Lattices
|
file |
diff |
annotate
|
Thu, 11 Feb 2010 23:00:22 +0100 |
wenzelm |
modernized translations;
|
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
|
Mon, 04 Jan 2010 16:00:23 +0100 |
haftmann |
moved name duplicates to end of theory; reduced warning noise
|
file |
diff |
annotate
|
Fri, 11 Dec 2009 14:43:56 +0100 |
haftmann |
moved predicate rules to Predicate.thy; weakened default dest rule predicate1D (is not that reliable wrt. sets)
|
file |
diff |
annotate
|
Sun, 08 Nov 2009 16:30:41 +0100 |
wenzelm |
adapted Generic_Data, Proof_Data;
|
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
|
Fri, 09 Oct 2009 13:34:34 +0200 |
haftmann |
tuned order of lemmas
|
file |
diff |
annotate
|
Wed, 07 Oct 2009 14:01:26 +0200 |
haftmann |
added bot_boolE, top_boolI
|
file |
diff |
annotate
|
Sun, 26 Jul 2009 22:28:31 +0200 |
wenzelm |
replaced old METAHYPS by FOCUS;
|
file |
diff |
annotate
|
Tue, 14 Jul 2009 10:54:04 +0200 |
haftmann |
code attributes use common underscore convention
|
file |
diff |
annotate
|
Wed, 15 Apr 2009 15:52:37 +0200 |
haftmann |
code generator bootstrap theory src/Tools/Code_Generator.thy
|
file |
diff |
annotate
|
Mon, 30 Mar 2009 22:48:15 +0200 |
wenzelm |
simplified 'print_orders' command;
|
file |
diff |
annotate
|
Thu, 26 Mar 2009 14:14:02 +0100 |
wenzelm |
simplified attribute and method setup: eliminating bottom-up styles makes it easier to keep things in one place, and also SML/NJ happy;
|
file |
diff |
annotate
|
Sun, 15 Mar 2009 15:59:44 +0100 |
wenzelm |
simplified attribute setup;
|
file |
diff |
annotate
|
Fri, 13 Mar 2009 23:50:05 +0100 |
wenzelm |
simplified method setup;
|
file |
diff |
annotate
|
Fri, 13 Mar 2009 19:58:26 +0100 |
wenzelm |
unified type Proof.method and pervasive METHOD combinators;
|
file |
diff |
annotate
|
Fri, 06 Mar 2009 14:33:19 +0100 |
haftmann |
added strict_mono predicate
|
file |
diff |
annotate
|
Thu, 26 Feb 2009 16:32:46 +0100 |
berghofe |
Fixed nonexhaustive match problem in decomp, to make it fail more gracefully
|
file |
diff |
annotate
|
Fri, 06 Feb 2009 15:15:32 +0100 |
haftmann |
session Reflecion renamed to Decision_Procs, moved Dense_Linear_Order there
|
file |
diff |
annotate
|
Wed, 21 Jan 2009 16:47:31 +0100 |
haftmann |
dropped ID
|
file |
diff |
annotate
|
Mon, 17 Nov 2008 17:00:55 +0100 |
haftmann |
tuned unfold_locales invocation
|
file |
diff |
annotate
|
Fri, 24 Oct 2008 17:48:37 +0200 |
haftmann |
new classes "top" and "bot"
|
file |
diff |
annotate
|
Fri, 10 Oct 2008 06:45:53 +0200 |
haftmann |
`code func` now just `code`
|
file |
diff |
annotate
|
Tue, 07 Oct 2008 16:07:21 +0200 |
haftmann |
tuned min/max code generation
|
file |
diff |
annotate
|
Mon, 11 Aug 2008 14:49:53 +0200 |
haftmann |
moved class wellorder to theory Orderings
|
file |
diff |
annotate
|
Tue, 29 Jul 2008 08:15:38 +0200 |
haftmann |
declare
|
file |
diff |
annotate
|
Fri, 25 Jul 2008 12:03:34 +0200 |
haftmann |
added class preorder
|
file |
diff |
annotate
|
Fri, 20 Jun 2008 21:00:21 +0200 |
haftmann |
streamlined definitions
|
file |
diff |
annotate
|
Tue, 10 Jun 2008 15:30:58 +0200 |
haftmann |
localized Least in Orderings.thy
|
file |
diff |
annotate
|
Wed, 07 May 2008 10:56:38 +0200 |
berghofe |
- Now imports Code_Setup, rather than Set and Fun, since the theorems
|
file |
diff |
annotate
|
Sat, 29 Mar 2008 22:55:49 +0100 |
wenzelm |
purely functional setup of claset/simpset/clasimpset;
|
file |
diff |
annotate
|
Wed, 19 Mar 2008 07:20:28 +0100 |
haftmann |
whitespace tuning
|
file |
diff |
annotate
|
Mon, 17 Mar 2008 18:37:00 +0100 |
wenzelm |
removed duplicate lemmas;
|
file |
diff |
annotate
|
Wed, 30 Jan 2008 10:57:46 +0100 |
haftmann |
dual orders and dual lattices
|
file |
diff |
annotate
|
Thu, 13 Dec 2007 07:09:02 +0100 |
haftmann |
clarified heading
|
file |
diff |
annotate
|
Fri, 30 Nov 2007 20:13:03 +0100 |
haftmann |
adjustions to due to instance target
|
file |
diff |
annotate
|
Thu, 29 Nov 2007 17:08:26 +0100 |
haftmann |
instance command as rudimentary class target
|
file |
diff |
annotate
|
Sat, 10 Nov 2007 18:36:06 +0100 |
wenzelm |
Orderings.min/max: no need to qualify consts;
|
file |
diff |
annotate
|
Fri, 26 Oct 2007 21:22:18 +0200 |
haftmann |
dropped square syntax
|
file |
diff |
annotate
|
Thu, 25 Oct 2007 19:27:50 +0200 |
haftmann |
various localizations
|
file |
diff |
annotate
|
Fri, 19 Oct 2007 19:45:31 +0200 |
haftmann |
tuned
|
file |
diff |
annotate
|
Thu, 18 Oct 2007 09:20:55 +0200 |
haftmann |
localized mono predicate
|
file |
diff |
annotate
|
Tue, 16 Oct 2007 23:12:45 +0200 |
haftmann |
global class syntax
|
file |
diff |
annotate
|
Tue, 09 Oct 2007 00:20:13 +0200 |
wenzelm |
generic Syntax.pretty/string_of operations;
|
file |
diff |
annotate
|
Sat, 06 Oct 2007 16:50:04 +0200 |
wenzelm |
simplified interfaces for outer syntax;
|
file |
diff |
annotate
|
Sat, 29 Sep 2007 08:58:51 +0200 |
haftmann |
proper syntax during class specification
|
file |
diff |
annotate
|
Thu, 27 Sep 2007 17:28:05 +0200 |
ballarin |
Fixed setup of transitivity reasoner (function decomp).
|
file |
diff |
annotate
|
Tue, 25 Sep 2007 12:56:27 +0200 |
ballarin |
Transitivity reasoner gets additional argument of premises to improve integration with simplifier.
|
file |
diff |
annotate
|
Tue, 18 Sep 2007 18:53:12 +0200 |
ballarin |
Transitivity reasoner set up for locales order and linorder.
|
file |
diff |
annotate
|
Fri, 24 Aug 2007 14:14:18 +0200 |
haftmann |
moved class dense_linear_order to Orderings.thy
|
file |
diff |
annotate
|
Wed, 15 Aug 2007 12:52:56 +0200 |
paulson |
ATP blacklisting is now in theory data, attribute noatp
|
file |
diff |
annotate
|
Tue, 24 Jul 2007 15:20:45 +0200 |
haftmann |
using class target
|
file |
diff |
annotate
|
Fri, 20 Jul 2007 14:28:25 +0200 |
haftmann |
moved class ord from Orderings.thy to HOL.thy
|
file |
diff |
annotate
|
Tue, 19 Jun 2007 23:15:23 +0200 |
wenzelm |
tuned;
|
file |
diff |
annotate
|
Tue, 05 Jun 2007 19:23:09 +0200 |
haftmann |
tuned boostrap
|
file |
diff |
annotate
|
Tue, 05 Jun 2007 15:16:08 +0200 |
haftmann |
merged Code_Generator.thy into HOL.thy
|
file |
diff |
annotate
|
Sun, 03 Jun 2007 16:57:51 +0200 |
nipkow |
tuned list comprehension, added lemma
|
file |
diff |
annotate
|
Fri, 01 Jun 2007 10:44:28 +0200 |
haftmann |
dropped superfluous name bindings
|
file |
diff |
annotate
|
Thu, 24 May 2007 08:37:39 +0200 |
haftmann |
rudimentary class target implementation
|
file |
diff |
annotate
|
Sat, 19 May 2007 14:05:05 +0200 |
nipkow |
unfold min/max in Stefans code generator
|
file |
diff |
annotate
|
Sat, 19 May 2007 11:33:22 +0200 |
haftmann |
no special treatment in naming of locale predicates stemming form classes
|
file |
diff |
annotate
|
Thu, 17 May 2007 19:49:40 +0200 |
haftmann |
canonical prefixing of class constants
|
file |
diff |
annotate
|
Thu, 10 May 2007 10:21:44 +0200 |
haftmann |
tuned
|
file |
diff |
annotate
|
Wed, 09 May 2007 07:53:06 +0200 |
haftmann |
moved recfun_codegen.ML to Code_Generator.thy
|
file |
diff |
annotate
|
Sun, 06 May 2007 21:49:27 +0200 |
haftmann |
dropped preorders, unified syntax
|
file |
diff |
annotate
|
Fri, 20 Apr 2007 11:21:36 +0200 |
haftmann |
shifted min/max to class order
|
file |
diff |
annotate
|
Thu, 29 Mar 2007 14:21:45 +0200 |
haftmann |
dropped legacy ML bindings
|
file |
diff |
annotate
|
Tue, 20 Mar 2007 08:27:15 +0100 |
haftmann |
explizit "type" superclass
|
file |
diff |
annotate
|
Fri, 09 Mar 2007 08:45:55 +0100 |
haftmann |
*** empty log message ***
|
file |
diff |
annotate
|
Fri, 02 Mar 2007 15:43:15 +0100 |
haftmann |
prefix of class interpretation not mandatory any longer
|
file |
diff |
annotate
|
Wed, 28 Feb 2007 22:05:43 +0100 |
wenzelm |
tuned ML setup;
|
file |
diff |
annotate
|
Fri, 23 Feb 2007 08:39:21 +0100 |
haftmann |
adjusted code lemmas
|
file |
diff |
annotate
|
Wed, 21 Feb 2007 13:51:12 +0100 |
krauss |
Fixed print translations for quantifiers a la "ALL x>=t. P x". These used
|
file |
diff |
annotate
|
Wed, 14 Feb 2007 10:06:12 +0100 |
haftmann |
added class "preorder"
|
file |
diff |
annotate
|
Sat, 10 Feb 2007 09:26:14 +0100 |
haftmann |
changed name of interpretation linorder to order
|
file |
diff |
annotate
|
Tue, 30 Jan 2007 08:21:13 +0100 |
haftmann |
changed name of interpretation linorder to order
|
file |
diff |
annotate
|
Tue, 16 Jan 2007 08:06:57 +0100 |
haftmann |
renamed locale partial_order to order
|
file |
diff |
annotate
|
Wed, 13 Dec 2006 15:45:29 +0100 |
haftmann |
dropped superfluous header
|
file |
diff |
annotate
|
Sun, 10 Dec 2006 15:30:34 +0100 |
wenzelm |
hide const linorder.less_eq_less.max linorder.less_eq_less.min;
|
file |
diff |
annotate
|
Wed, 06 Dec 2006 01:12:51 +0100 |
wenzelm |
added basic ML bindings;
|
file |
diff |
annotate
|
Tue, 05 Dec 2006 22:14:39 +0100 |
wenzelm |
restored notation for less/less_eq (observe proper order of mixfix annotations!);
|
file |
diff |
annotate
|
Fri, 01 Dec 2006 17:22:30 +0100 |
haftmann |
some syntax cleanup
|
file |
diff |
annotate
|
Mon, 27 Nov 2006 13:42:33 +0100 |
haftmann |
removed HOL structure
|
file |
diff |
annotate
|
Sun, 26 Nov 2006 18:07:16 +0100 |
wenzelm |
updated (binder) syntax/notation;
|
file |
diff |
annotate
|
Sat, 18 Nov 2006 00:20:19 +0100 |
haftmann |
re-eliminated thm trichotomy
|
file |
diff |
annotate
|
Fri, 17 Nov 2006 02:20:03 +0100 |
wenzelm |
more robust syntax for definition/abbreviation/notation;
|
file |
diff |
annotate
|
Wed, 15 Nov 2006 17:05:42 +0100 |
haftmann |
added transitivity rules, reworking of min/max lemmas
|
file |
diff |
annotate
|
Mon, 13 Nov 2006 15:43:06 +0100 |
haftmann |
introduces preorders
|
file |
diff |
annotate
|
Thu, 09 Nov 2006 11:58:13 +0100 |
wenzelm |
modified less/less_eq syntax to avoid "x < y < z" etc.;
|
file |
diff |
annotate
|
Wed, 08 Nov 2006 19:46:10 +0100 |
haftmann |
abstract ordering theories
|
file |
diff |
annotate
|
Tue, 07 Nov 2006 14:03:06 +0100 |
haftmann |
made locale partial_order compatible with axclass order; changed import order; consecutive changes
|
file |
diff |
annotate
|