src/HOL/Library/RBT_Impl.thy
Fri, 13 Apr 2012 14:00:26 +0200 wenzelm updated headers;
Fri, 13 Apr 2012 11:45:30 +0200 Andreas Lochbihler move RBT implementation into type class contexts
Fri, 06 Apr 2012 18:17:16 +0200 haftmann no preference wrt. fold(l/r); prefer fold rather than foldr for iterating over lists in generated code
Fri, 06 Jan 2012 10:19:49 +0100 haftmann incorporated canonical fold combinator on lists into body of List theory; refactored passages on List.fold(l/r)
Mon, 26 Dec 2011 22:17:10 +0100 haftmann incorporated More_Set and More_List into the Main body -- to be consolidated later
Sun, 13 Mar 2011 22:55:50 +0100 wenzelm tuned headers;
Wed, 08 Dec 2010 13:34:50 +0100 haftmann hide popular names R and B
Mon, 13 Sep 2010 11:13:15 +0200 nipkow renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
Tue, 07 Sep 2010 10:05:19 +0200 nipkow expand_fun_eq -> ext_iff
Mon, 28 Jun 2010 15:03:07 +0200 haftmann merged constants "split" and "prod_case"
Fri, 18 Jun 2010 15:03:20 +0200 haftmann prefer fold over foldl
Fri, 16 Apr 2010 21:28:09 +0200 wenzelm replaced generic 'hide' command by more conventional 'hide_class', 'hide_type', 'hide_const', 'hide_fact' -- frees some popular keywords;
Thu, 15 Apr 2010 12:27:14 +0200 haftmann theory RBT with abstract type of red-black trees backed by implementation RBT_Impl
less more (0) tip