src/HOL/Orderings.thy
Sat, 06 Oct 2007 16:50:04 +0200 simplified interfaces for outer syntax;
Sat, 29 Sep 2007 08:58:51 +0200 proper syntax during class specification
Thu, 27 Sep 2007 17:28:05 +0200 Fixed setup of transitivity reasoner (function decomp).
Tue, 25 Sep 2007 12:56:27 +0200 Transitivity reasoner gets additional argument of premises to improve integration with simplifier.
Tue, 18 Sep 2007 18:53:12 +0200 Transitivity reasoner set up for locales order and linorder.
Fri, 24 Aug 2007 14:14:18 +0200 moved class dense_linear_order to Orderings.thy
Wed, 15 Aug 2007 12:52:56 +0200 ATP blacklisting is now in theory data, attribute noatp
Tue, 24 Jul 2007 15:20:45 +0200 using class target
Fri, 20 Jul 2007 14:28:25 +0200 moved class ord from Orderings.thy to HOL.thy
Tue, 19 Jun 2007 23:15:23 +0200 tuned;
Tue, 05 Jun 2007 19:23:09 +0200 tuned boostrap
Tue, 05 Jun 2007 15:16:08 +0200 merged Code_Generator.thy into HOL.thy
Sun, 03 Jun 2007 16:57:51 +0200 tuned list comprehension, added lemma
Fri, 01 Jun 2007 10:44:28 +0200 dropped superfluous name bindings
Thu, 24 May 2007 08:37:39 +0200 rudimentary class target implementation
Sat, 19 May 2007 14:05:05 +0200 unfold min/max in Stefans code generator
Sat, 19 May 2007 11:33:22 +0200 no special treatment in naming of locale predicates stemming form classes
Thu, 17 May 2007 19:49:40 +0200 canonical prefixing of class constants
Thu, 10 May 2007 10:21:44 +0200 tuned
Wed, 09 May 2007 07:53:06 +0200 moved recfun_codegen.ML to Code_Generator.thy
Sun, 06 May 2007 21:49:27 +0200 dropped preorders, unified syntax
Fri, 20 Apr 2007 11:21:36 +0200 shifted min/max to class order
Thu, 29 Mar 2007 14:21:45 +0200 dropped legacy ML bindings
Tue, 20 Mar 2007 08:27:15 +0100 explizit "type" superclass
Fri, 09 Mar 2007 08:45:55 +0100 *** empty log message ***
Fri, 02 Mar 2007 15:43:15 +0100 prefix of class interpretation not mandatory any longer
Wed, 28 Feb 2007 22:05:43 +0100 tuned ML setup;
Fri, 23 Feb 2007 08:39:21 +0100 adjusted code lemmas
Wed, 21 Feb 2007 13:51:12 +0100 Fixed print translations for quantifiers a la "ALL x>=t. P x". These used
Wed, 14 Feb 2007 10:06:12 +0100 added class "preorder"
Sat, 10 Feb 2007 09:26:14 +0100 changed name of interpretation linorder to order
Tue, 30 Jan 2007 08:21:13 +0100 changed name of interpretation linorder to order
Tue, 16 Jan 2007 08:06:57 +0100 renamed locale partial_order to order
Wed, 13 Dec 2006 15:45:29 +0100 dropped superfluous header
Sun, 10 Dec 2006 15:30:34 +0100 hide const linorder.less_eq_less.max linorder.less_eq_less.min;
Wed, 06 Dec 2006 01:12:51 +0100 added basic ML bindings;
Tue, 05 Dec 2006 22:14:39 +0100 restored notation for less/less_eq (observe proper order of mixfix annotations!);
Fri, 01 Dec 2006 17:22:30 +0100 some syntax cleanup
Mon, 27 Nov 2006 13:42:33 +0100 removed HOL structure
Sun, 26 Nov 2006 18:07:16 +0100 updated (binder) syntax/notation;
Sat, 18 Nov 2006 00:20:19 +0100 re-eliminated thm trichotomy
Fri, 17 Nov 2006 02:20:03 +0100 more robust syntax for definition/abbreviation/notation;
Wed, 15 Nov 2006 17:05:42 +0100 added transitivity rules, reworking of min/max lemmas
Mon, 13 Nov 2006 15:43:06 +0100 introduces preorders
Thu, 09 Nov 2006 11:58:13 +0100 modified less/less_eq syntax to avoid "x < y < z" etc.;
Wed, 08 Nov 2006 19:46:10 +0100 abstract ordering theories
Tue, 07 Nov 2006 14:03:06 +0100 made locale partial_order compatible with axclass order; changed import order; consecutive changes
Tue, 07 Nov 2006 11:46:46 +0100 renamed 'const_syntax' to 'notation';
Mon, 06 Nov 2006 16:28:35 +0100 removed dependency of ord on eq
Sun, 05 Nov 2006 21:44:33 +0100 fixed print_translation for ALL/EX and <, <=, etc.; tuned syntax names;
Mon, 23 Oct 2006 11:05:07 +0200 cleanup in ML setup code
Fri, 20 Oct 2006 18:20:22 +0200 cleaned up
Mon, 16 Oct 2006 14:07:20 +0200 fixed print translations for bounded quantification
Tue, 26 Sep 2006 13:34:17 +0200 tuned syntax for <= <
Tue, 19 Sep 2006 15:21:42 +0200 added operational equality
Tue, 04 Jul 2006 14:47:01 +0200 Method intro_locales replaced by intro_locales and unfold_locales.
Tue, 20 Jun 2006 15:53:44 +0200 Restructured locales with predicates: import is now an interpretation.
Tue, 16 May 2006 21:33:01 +0200 tuned concrete syntax -- abbreviation/const_syntax;
Sat, 13 May 2006 21:13:25 +0200 reactivated translations for less/less_eq;
Tue, 02 May 2006 20:42:32 +0200 replaced syntax/translations by abbreviation;