src/HOL/Library/Library.thy
Sat, 08 Jan 2011 17:39:51 +0100 wenzelm renamed Sum_Of_Squares to Sum_of_Squares;
Mon, 22 Nov 2010 17:49:12 +0100 haftmann merged
Mon, 22 Nov 2010 17:46:51 +0100 haftmann replaced misleading Fset/fset name -- these do not stand for finite sets
Mon, 22 Nov 2010 11:34:56 +0100 bulwahn adding Enum to HOL-Main image and removing it from HOL-Library
Wed, 03 Nov 2010 12:20:33 +0100 haftmann moved theory Quicksort from Library/ to ex/
Fri, 20 Aug 2010 17:48:30 +0200 haftmann split and enriched theory SetsAndFunctions
Wed, 14 Jul 2010 14:16:12 +0200 haftmann load cache_io before code generator; moved adhoc-overloading to generic tools
Tue, 13 Jul 2010 00:15:37 +0200 krauss uniform do notation for monads
Tue, 13 Jul 2010 00:15:37 +0200 krauss generic ad-hoc overloading via check/uncheck
Fri, 02 Jul 2010 14:23:17 +0200 haftmann remove codegeneration-related theories from big library theory
Thu, 01 Jul 2010 11:48:42 +0200 hoelzl Add theory for indicator function.
Thu, 20 May 2010 16:35:54 +0200 haftmann added theory More_List
Mon, 17 May 2010 10:58:31 +0200 haftmann dropped old Library/Word.thy and toy example ex/Adder.thy
Tue, 04 May 2010 18:05:22 +0200 hoelzl Add Convex to Library build
Thu, 15 Apr 2010 12:27:14 +0200 haftmann theory RBT with abstract type of red-black trees backed by implementation RBT_Impl
Sat, 13 Mar 2010 17:19:12 +0100 wenzelm removed obsolete HOL/Library/Coinductive_List.thy, superceded by thys/Coinductive/Coinductive_List.thy in AFP/f2f5727b77d0;
Sat, 06 Mar 2010 15:31:30 +0100 haftmann added Table.thy
Mon, 22 Feb 2010 15:53:18 +0100 haftmann added Dlist
Fri, 19 Feb 2010 13:54:19 +0100 Cezary Kaliszyk Initial version of HOL quotient package.
Wed, 10 Feb 2010 19:37:34 +0100 wenzelm renamed Library/Quotient.thy to Library/Quotient_Type.thy to avoid clash with new theory Quotient in Main HOL;
Wed, 10 Feb 2010 14:12:02 +0100 haftmann revert uninspired Structure_Syntax experiment
Mon, 08 Feb 2010 14:08:32 +0100 haftmann merged
Mon, 08 Feb 2010 14:06:41 +0100 haftmann separate library theory for type classes combining lattices with various algebraic structures
Mon, 08 Feb 2010 10:36:02 +0100 haftmann separate theory for index structures
Mon, 07 Dec 2009 14:54:01 +0100 haftmann merged Crude_Executable_Set into Executable_Set
Wed, 02 Dec 2009 17:53:34 +0100 haftmann added Crude_Executable_Set.thy
Thu, 12 Nov 2009 20:38:57 +0100 bulwahn added a tabled implementation of the reflexive transitive closure
Fri, 30 Oct 2009 13:59:49 +0100 haftmann moved Commutative_Ring into session Decision_Procs
Mon, 26 Oct 2009 11:19:24 +0100 haftmann re-moved theory Fin_Fun to AFP
Mon, 26 Oct 2009 09:03:57 +0100 haftmann merged
Fri, 23 Oct 2009 13:23:18 +0200 himmelma distinguished session for multivariate analysis
Fri, 23 Oct 2009 17:12:36 +0200 haftmann turned off old quickcheck
Tue, 01 Sep 2009 15:39:33 +0200 haftmann some reorganization of number theory
Fri, 10 Jul 2009 09:24:50 +0200 krauss move Kleene_Algebra to Library
Mon, 29 Jun 2009 12:18:55 +0200 haftmann renamed theory Code_Set to Fset
Thu, 25 Jun 2009 17:07:18 +0200 haftmann added List_Set and Code_Set theories
Tue, 23 Jun 2009 10:22:11 +0200 chaieb Added Library/Fraction_Field.thy: The fraction field of any integral
Tue, 02 Jun 2009 15:53:34 +0200 haftmann added Fin_Fun theory
Tue, 02 Jun 2009 10:00:29 +0200 berghofe Added Convex_Euclidean_Space.thy again.
Thu, 28 May 2009 18:59:51 +0200 himmelma Removed Convex_Euclidean_Space.thy from Library.
Thu, 28 May 2009 13:56:50 +0200 himmelma Added Convex_Euclidean_Space to Library.thy and Library/IsaMakefile
Sat, 16 May 2009 20:16:49 +0200 haftmann experimental move of Quickcheck and related theories to HOL image
Tue, 12 May 2009 17:32:49 +0100 chaieb Added files Sum_Of_Squares.thy, positivstellensatz.ML and sum_of_squares.ML to Library
Thu, 07 May 2009 12:17:17 +0200 haftmann added theory for explicit equivalence relation in preorders
Fri, 06 Mar 2009 20:30:16 +0100 haftmann constructive version of Cantor's first diagonalization argument
Wed, 04 Mar 2009 19:21:55 +0000 chaieb Added Libray dependency on Topology_Euclidean_Space
Wed, 04 Mar 2009 11:05:29 +0100 blanchet Merge.
Wed, 04 Mar 2009 10:45:52 +0100 blanchet Merge.
Fri, 20 Feb 2009 08:02:11 -0800 huffman add theory of products as real vector spaces to Library
Fri, 20 Feb 2009 07:41:41 -0800 huffman add new theory Product_plus.thy to Library
Thu, 19 Feb 2009 12:03:31 -0800 huffman add formalization of a type of integers mod 2 to Library
Thu, 19 Feb 2009 09:42:23 -0800 huffman new theory of real inner product spaces
Wed, 18 Feb 2009 20:14:45 -0800 huffman move Polynomial.thy to Library
Wed, 18 Feb 2009 19:51:39 -0800 huffman move FrechetDeriv.thy to Library
Wed, 18 Feb 2009 19:32:26 -0800 huffman split polynomial-related stuff from Deriv.thy into Library/Poly_Deriv.thy
Thu, 12 Feb 2009 18:14:43 +0100 nipkow Moved FTA into Lib and cleaned it up a little.
Mon, 09 Feb 2009 17:21:46 +0000 chaieb added Determinants to Library
Mon, 09 Feb 2009 17:09:18 +0000 chaieb added Euclidean_Space and Glbs to Library
Mon, 09 Feb 2009 11:15:13 +0000 chaieb Added HOL/Library/Finite_Cartesian_Product.thy to Library
Fri, 06 Feb 2009 15:15:32 +0100 haftmann session Reflecion renamed to Decision_Procs, moved Dense_Linear_Order there
Fri, 06 Feb 2009 00:10:58 +0000 chaieb fixed Proofs and dependencies ; Theory Dense_Linear_Order moved to Library
Thu, 05 Feb 2009 14:14:02 +0100 haftmann moved Random.thy to Library
Mon, 02 Feb 2009 13:56:22 +0100 haftmann added Mapping.thy to Library
Thu, 29 Jan 2009 14:56:29 +0000 chaieb Added Formal_Power_Series in imports
Wed, 28 Jan 2009 11:04:10 +0100 haftmann Reflection.thy now in HOL/Library
Fri, 16 Jan 2009 08:28:53 +0100 haftmann moved Univ_Poly to Library
Thu, 08 Jan 2009 17:10:41 +0100 haftmann split of Imperative_HOL theories from HOL-Library
Mon, 29 Dec 2008 14:08:08 +0100 haftmann adapted HOL source structure to distribution layout
Wed, 10 Dec 2008 10:23:47 +0100 nipkow moved ContNotDenum into Library
Wed, 03 Dec 2008 15:58:44 +0100 haftmann made repository layout more coherent with logical distribution structure; stripped some $Id$s
Thu, 23 Oct 2008 00:24:31 +0200 wenzelm fixed and reactivated HOL/Library/Pocklington.thy -- by Mark Hillebrand;
Tue, 16 Sep 2008 09:21:24 +0200 haftmann evaluation using code generator
Tue, 02 Sep 2008 22:37:20 +0200 nipkow Replaced Library/NatPair by Nat_Int_Bij.
Fri, 18 Jul 2008 18:25:56 +0200 haftmann refined code generator setup for rational numbers; more simplification rules for rational numbers
Thu, 03 Jul 2008 18:16:40 +0200 huffman 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 haftmann established Plain theory and image
Fri, 20 Jun 2008 21:00:16 +0200 haftmann moved Float.thy to Library
Thu, 20 Mar 2008 12:01:10 +0100 haftmann added theory Library/Enum.thy
Fri, 14 Mar 2008 19:57:32 +0100 nipkow Added Order_Relation
Fri, 07 Mar 2008 13:53:01 +0100 haftmann canonical order on option type
Mon, 03 Mar 2008 14:03:19 +0100 krauss new theory of red-black trees, an efficient implementation of finite maps.
Thu, 28 Feb 2008 00:11:28 +0100 wenzelm renamed ListSpace to ListVector;
Wed, 27 Feb 2008 21:41:08 +0100 haftmann added theories for imperative HOL
Wed, 27 Feb 2008 14:39:51 +0100 chaieb Loads Dense_Linear_Order.thy
Mon, 25 Feb 2008 11:27:08 +0100 chaieb Uses Univ_Poly.thy
Mon, 14 Jan 2008 11:45:57 +0100 nipkow *** empty log message ***
Tue, 06 Nov 2007 20:27:33 +0100 wenzelm removed dependencies on Size_Change_Termination from HOL-Library;
Fri, 12 Oct 2007 08:21:09 +0200 haftmann consolidated naming conventions for code generator theories
Tue, 18 Sep 2007 07:46:00 +0200 haftmann introduced generic concepts for theory interpretators
Tue, 18 Sep 2007 05:42:46 +0200 nipkow Added function package to PreList
Thu, 06 Sep 2007 11:32:28 +0200 berghofe Integrated Executable_Rat and Executable_Real theories into
Mon, 20 Aug 2007 00:22:18 +0200 kleing boolean algebras as locales and numbers as types by Brian Huffman
Wed, 15 Aug 2007 08:57:40 +0200 haftmann added Eval_Witness theory
Thu, 09 Aug 2007 15:52:49 +0200 haftmann proper implementation of rational numbers
Thu, 19 Jul 2007 21:47:39 +0200 haftmann uniform naming conventions for CG theories
Fri, 01 Jun 2007 22:09:16 +0200 nipkow Moved list comprehension into List
Fri, 25 May 2007 18:08:34 +0200 nipkow Added List_Comprehension
Tue, 15 May 2007 18:28:02 +0200 chaieb A verified theory for rational numbers representation and simple calculations;
Thu, 26 Apr 2007 13:32:59 +0200 haftmann moved code generation pretty integers and characters to separate theories
Mon, 26 Mar 2007 14:53:02 +0200 haftmann importing Eval theory
Mon, 26 Feb 2007 21:34:16 +0100 krauss Added formalization of size-change principle (experimental).
Mon, 04 Dec 2006 15:15:59 +0100 krauss added Ramsey.thy to Library imports, to include it in the daily builds
Wed, 08 Nov 2006 23:11:13 +0100 wenzelm moved theories Parity, GCD, Binomial to Library;
Mon, 06 Nov 2006 16:28:33 +0100 haftmann added state monad to HOL library
Sun, 01 Oct 2006 18:29:26 +0200 wenzelm moved theory Infinite_Set to Library;
Mon, 21 Aug 2006 11:02:39 +0200 haftmann added some codegen examples/applications
Tue, 09 May 2006 10:13:09 +0200 haftmann added ExecutableRat.thy
Fri, 05 May 2006 17:17:21 +0200 krauss First usable version of the new function definition package (HOL/function_packake/...).
Wed, 26 Apr 2006 07:01:33 +0200 kleing moved arithmetic series to geometric series in SetInterval
Fri, 07 Apr 2006 03:20:34 +0200 kleing renamed ASeries to Arithmetic_Series, removed the ^M
Fri, 10 Mar 2006 16:05:34 +0100 schirmer Added Library/AssocList.thy
Sun, 19 Feb 2006 13:21:32 +0100 kleing * added Library/ASeries (sum of arithmetic series with instantiation to nat and int)
Tue, 13 Dec 2005 19:32:04 +0100 wenzelm added HOL/Library/Coinductive_List.thy;
Sun, 25 Sep 2005 20:12:59 +0200 berghofe Added ExecutableSet.
Tue, 20 Sep 2005 14:10:29 +0200 wenzelm added Commutative_Ring (from Main HOL);
Mon, 01 Aug 2005 11:39:33 +0200 obua 1. changed configuration variables for linear programming (Cplex_tools):
Mon, 25 Jul 2005 18:54:49 +0200 avigad Added two new theories to HOL/Library: SetsAndFunctions.thy and BigO.thy
Sun, 29 May 2005 12:41:40 +0200 obua Removes an inconsistent definition from Library.thy ,
Thu, 14 Apr 2005 17:57:04 +0200 nipkow Removed dir Orderings in Library
Wed, 26 Jan 2005 16:39:44 +0100 nipkow added OptionalSugar
less more (0) -120 tip