src/HOL/Library/Library.thy
Thu, 08 Jan 2009 17:10:41 +0100 split of Imperative_HOL theories from HOL-Library
Mon, 29 Dec 2008 14:08:08 +0100 adapted HOL source structure to distribution layout
Wed, 10 Dec 2008 10:23:47 +0100 moved ContNotDenum into Library
Wed, 03 Dec 2008 15:58:44 +0100 made repository layout more coherent with logical distribution structure; stripped some $Id$s
Thu, 23 Oct 2008 00:24:31 +0200 fixed and reactivated HOL/Library/Pocklington.thy -- by Mark Hillebrand;
Tue, 16 Sep 2008 09:21:24 +0200 evaluation using code generator
Tue, 02 Sep 2008 22:37:20 +0200 Replaced Library/NatPair by Nat_Int_Bij.
Fri, 18 Jul 2008 18:25:56 +0200 refined code generator setup for rational numbers; more simplification rules for rational numbers
Thu, 03 Jul 2008 18:16:40 +0200 add Infinite_Set and Zorn back in (since they are no longer included in main HOL image)
Thu, 26 Jun 2008 10:07:01 +0200 established Plain theory and image
Fri, 20 Jun 2008 21:00:16 +0200 moved Float.thy to Library
Thu, 20 Mar 2008 12:01:10 +0100 added theory Library/Enum.thy
Fri, 14 Mar 2008 19:57:32 +0100 Added Order_Relation
Fri, 07 Mar 2008 13:53:01 +0100 canonical order on option type
Mon, 03 Mar 2008 14:03:19 +0100 new theory of red-black trees, an efficient implementation of finite maps.
Thu, 28 Feb 2008 00:11:28 +0100 renamed ListSpace to ListVector;
Wed, 27 Feb 2008 21:41:08 +0100 added theories for imperative HOL
Wed, 27 Feb 2008 14:39:51 +0100 Loads Dense_Linear_Order.thy
Mon, 25 Feb 2008 11:27:08 +0100 Uses Univ_Poly.thy
Mon, 14 Jan 2008 11:45:57 +0100 *** empty log message ***
Tue, 06 Nov 2007 20:27:33 +0100 removed dependencies on Size_Change_Termination from HOL-Library;
Fri, 12 Oct 2007 08:21:09 +0200 consolidated naming conventions for code generator theories
Tue, 18 Sep 2007 07:46:00 +0200 introduced generic concepts for theory interpretators
Tue, 18 Sep 2007 05:42:46 +0200 Added function package to PreList
Thu, 06 Sep 2007 11:32:28 +0200 Integrated Executable_Rat and Executable_Real theories into
Mon, 20 Aug 2007 00:22:18 +0200 boolean algebras as locales and numbers as types by Brian Huffman
Wed, 15 Aug 2007 08:57:40 +0200 added Eval_Witness theory
Thu, 09 Aug 2007 15:52:49 +0200 proper implementation of rational numbers
Thu, 19 Jul 2007 21:47:39 +0200 uniform naming conventions for CG theories
Fri, 01 Jun 2007 22:09:16 +0200 Moved list comprehension into List
Fri, 25 May 2007 18:08:34 +0200 Added List_Comprehension
Tue, 15 May 2007 18:28:02 +0200 A verified theory for rational numbers representation and simple calculations;
Thu, 26 Apr 2007 13:32:59 +0200 moved code generation pretty integers and characters to separate theories
Mon, 26 Mar 2007 14:53:02 +0200 importing Eval theory
Mon, 26 Feb 2007 21:34:16 +0100 Added formalization of size-change principle (experimental).
Mon, 04 Dec 2006 15:15:59 +0100 added Ramsey.thy to Library imports, to include it in the daily builds
Wed, 08 Nov 2006 23:11:13 +0100 moved theories Parity, GCD, Binomial to Library;
Mon, 06 Nov 2006 16:28:33 +0100 added state monad to HOL library
Sun, 01 Oct 2006 18:29:26 +0200 moved theory Infinite_Set to Library;
Mon, 21 Aug 2006 11:02:39 +0200 added some codegen examples/applications
Tue, 09 May 2006 10:13:09 +0200 added ExecutableRat.thy
Fri, 05 May 2006 17:17:21 +0200 First usable version of the new function definition package (HOL/function_packake/...).
Wed, 26 Apr 2006 07:01:33 +0200 moved arithmetic series to geometric series in SetInterval
Fri, 07 Apr 2006 03:20:34 +0200 renamed ASeries to Arithmetic_Series, removed the ^M
Fri, 10 Mar 2006 16:05:34 +0100 Added Library/AssocList.thy
Sun, 19 Feb 2006 13:21:32 +0100 * added Library/ASeries (sum of arithmetic series with instantiation to nat and int)
Tue, 13 Dec 2005 19:32:04 +0100 added HOL/Library/Coinductive_List.thy;
Sun, 25 Sep 2005 20:12:59 +0200 Added ExecutableSet.
Tue, 20 Sep 2005 14:10:29 +0200 added Commutative_Ring (from Main HOL);
Mon, 01 Aug 2005 11:39:33 +0200 1. changed configuration variables for linear programming (Cplex_tools):
Mon, 25 Jul 2005 18:54:49 +0200 Added two new theories to HOL/Library: SetsAndFunctions.thy and BigO.thy
Sun, 29 May 2005 12:41:40 +0200 Removes an inconsistent definition from Library.thy ,
Thu, 14 Apr 2005 17:57:04 +0200 Removed dir Orderings in Library
Wed, 26 Jan 2005 16:39:44 +0100 added OptionalSugar
Wed, 24 Nov 2004 10:30:19 +0100 Added EfficientNat
Wed, 18 Aug 2004 11:09:40 +0200 import -> imports
Mon, 16 Aug 2004 14:22:27 +0200 New theory header syntax.
Thu, 06 May 2004 14:14:18 +0200 tuned document;
Mon, 29 Mar 2004 15:35:04 +0200 Added bitvector library (Word) to HOL/Library and a theory using it (Adder)
Tue, 27 Jan 2004 15:39:51 +0100 replacing HOL/Real/PRat, PNat by the rational number development