src/HOL/Library/Library.thy
Wed, 07 Sep 2011 23:38:52 +0200 haftmann theory of saturated naturals contributed by Peter Gammie
Sun, 28 Aug 2011 08:13:30 +0200 haftmann avoid loading List_Cset and Dlist_Cet at the same time
Wed, 17 Aug 2011 13:14:20 +0200 wenzelm moved theory Nested_Environment to HOL-Unix (a bit too specific for HOL-Library);
Tue, 16 Aug 2011 07:06:54 -0700 huffman get Library/Permutations.thy compiled and working again
Tue, 02 Aug 2011 11:52:57 +0200 krauss moved recursion combinator to HOL/Library/Wfrec.thy -- it is so fundamental and well-known that it should survive recdef
Tue, 02 Aug 2011 10:36:50 +0200 krauss moved recdef package to HOL/Library/Old_Recdef.thy
Tue, 26 Jul 2011 10:49:34 +0200 Andreas Lochbihler Add theory for setting up monad syntax for Cset
Mon, 25 Jul 2011 10:43:14 +0200 bulwahn removing SML_Quickcheck
Tue, 19 Jul 2011 14:35:44 +0200 hoelzl rename Nat_Infinity (inat) to Extended_Nat (enat)
Tue, 07 Jun 2011 11:12:05 +0200 bulwahn splitting Cset into Cset and List_Cset
Thu, 02 Jun 2011 08:55:08 +0200 bulwahn splitting Dlist theory in Dlist and Dlist_Cset
Wed, 01 Jun 2011 09:10:13 +0200 bulwahn splitting RBT theory into RBT and RBT_Mapping
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.
less more (0) -100 -60 tip