| Tue, 01 Jun 2021 19:46:34 +0200 | 
nipkow | 
More general fold function for maps
 | 
file |
diff |
annotate
 | 
| Thu, 02 Jun 2016 08:34:23 +0200 | 
Manuel Eberl | 
Hid RBT.filter
 | 
file |
diff |
annotate
 | 
| Tue, 31 May 2016 13:02:44 +0200 | 
eberlm | 
Added code generation for PMFs
 | 
file |
diff |
annotate
 | 
| Thu, 24 Sep 2015 13:33:42 +0200 | 
wenzelm | 
explicit indication of overloaded typedefs;
 | 
file |
diff |
annotate
 | 
| Tue, 01 Sep 2015 22:32:58 +0200 | 
wenzelm | 
eliminated \<Colon>;
 | 
file |
diff |
annotate
 | 
| Wed, 17 Jun 2015 11:03:05 +0200 | 
wenzelm | 
isabelle update_cartouches;
 | 
file |
diff |
annotate
 | 
| Sun, 02 Nov 2014 17:20:45 +0100 | 
wenzelm | 
modernized header;
 | 
file |
diff |
annotate
 | 
| Mon, 10 Mar 2014 17:14:57 +0100 | 
kuncar | 
hide implementation details
 | 
file |
diff |
annotate
 | 
| Tue, 18 Feb 2014 23:03:50 +0100 | 
kuncar | 
simplify proofs because of the stronger reflexivity prover
 | 
file |
diff |
annotate
 | 
| Fri, 14 Feb 2014 07:53:46 +0100 | 
blanchet | 
merged 'Option.map' and 'Option.map_option'
 | 
file |
diff |
annotate
 | 
| Wed, 12 Feb 2014 08:35:57 +0100 | 
blanchet | 
renamed '{prod,sum,bool,unit}_case' to 'case_...'
 | 
file |
diff |
annotate
 | 
| Tue, 13 Aug 2013 15:59:22 +0200 | 
kuncar | 
remove unnecessary dependencies on Library/Quotient_*
 | 
file |
diff |
annotate
 | 
| Fri, 08 Mar 2013 13:21:06 +0100 | 
kuncar | 
patch Isabelle ditribution to conform to changes regarding the parametricity
 | 
file |
diff |
annotate
 | 
| Fri, 19 Oct 2012 17:54:16 +0200 | 
kuncar | 
don't include Quotient_Option - workaround to a transfer bug
 | 
file |
diff |
annotate
 | 
| Thu, 18 Oct 2012 15:52:31 +0200 | 
kuncar | 
new theorem
 | 
file |
diff |
annotate
 | 
| Fri, 12 Oct 2012 18:58:20 +0200 | 
wenzelm | 
discontinued obsolete typedef (open) syntax;
 | 
file |
diff |
annotate
 | 
| Tue, 31 Jul 2012 13:55:39 +0200 | 
kuncar | 
use lifting/transfer formalization of RBT from Lift_RBT
 | 
file |
diff |
annotate
 | 
| Fri, 13 Apr 2012 11:45:30 +0200 | 
Andreas Lochbihler | 
move RBT implementation into type class contexts
 | 
file |
diff |
annotate
 | 
| Tue, 21 Feb 2012 12:20:33 +0100 | 
bulwahn | 
subtype preprocessing in Quickcheck;
 | 
file |
diff |
annotate
 | 
| 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)
 | 
file |
diff |
annotate
 | 
| Tue, 20 Dec 2011 17:40:18 +0100 | 
bulwahn | 
adding quickcheck generators in some HOL-Library theories
 | 
file |
diff |
annotate
 | 
| Wed, 30 Nov 2011 16:27:10 +0100 | 
wenzelm | 
prefer typedef without extra definition and alternative name;
 | 
file |
diff |
annotate
 | 
| Wed, 01 Jun 2011 09:10:13 +0200 | 
bulwahn | 
splitting RBT theory into RBT and RBT_Mapping
 | 
file |
diff |
annotate
 | 
| Thu, 18 Nov 2010 18:53:36 +0100 | 
haftmann | 
proper qualification needed due to shadowing on theory merge
 | 
file |
diff |
annotate
 | 
| Mon, 13 Sep 2010 16:43:23 +0200 | 
haftmann | 
established emerging canonical names *_eqI and *_eq_iff
 | 
file |
diff |
annotate
 | 
| 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
 | 
file |
diff |
annotate
 | 
| Tue, 07 Sep 2010 10:05:19 +0200 | 
nipkow | 
expand_fun_eq -> ext_iff
 | 
file |
diff |
annotate
 | 
| Fri, 27 Aug 2010 19:34:23 +0200 | 
haftmann | 
renamed class/constant eq to equal; tuned some instantiations
 | 
file |
diff |
annotate
 | 
| Fri, 18 Jun 2010 15:26:02 +0200 | 
haftmann | 
prefer fold over foldl
 | 
file |
diff |
annotate
 | 
| Fri, 21 May 2010 15:22:37 +0200 | 
haftmann | 
tuned
 | 
file |
diff |
annotate
 | 
| Thu, 20 May 2010 17:29:43 +0200 | 
haftmann | 
implement Mapping.map_entry
 | 
file |
diff |
annotate
 | 
| Wed, 21 Apr 2010 11:23:04 +0200 | 
hoelzl | 
merged
 | 
file |
diff |
annotate
 | 
| 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;
 | 
file |
diff |
annotate
 | 
| Thu, 15 Apr 2010 12:27:14 +0200 | 
haftmann | 
theory RBT with abstract type of red-black trees backed by implementation RBT_Impl
 | 
file |
diff |
annotate
| base
 | 
| Sat, 06 Mar 2010 15:31:30 +0100 | 
haftmann | 
some lemma refinements
 | 
file |
diff |
annotate
 | 
| Sat, 06 Mar 2010 09:58:28 +0100 | 
haftmann | 
added bulkload; tuned document
 | 
file |
diff |
annotate
 | 
| Fri, 05 Mar 2010 17:55:14 +0100 | 
haftmann | 
moved lemma map_sorted_distinct_set_unique
 | 
file |
diff |
annotate
 | 
| Fri, 05 Mar 2010 17:51:29 +0100 | 
haftmann | 
various refinements
 | 
file |
diff |
annotate
 | 
| Wed, 03 Mar 2010 17:21:45 +0100 | 
haftmann | 
restructured RBT theory
 | 
file |
diff |
annotate
 | 
| Wed, 03 Mar 2010 08:28:33 +0100 | 
haftmann | 
more explicit naming scheme
 | 
file |
diff |
annotate
 | 
| Tue, 28 Jul 2009 08:49:03 +0200 | 
krauss | 
tuned
 | 
file |
diff |
annotate
 | 
| Mon, 27 Jul 2009 22:50:04 +0200 | 
krauss | 
added missing proof of RBT.map_of_alist_of (contributed by Peter Lammich)
 | 
file |
diff |
annotate
 | 
| Fri, 27 Mar 2009 10:05:11 +0100 | 
haftmann | 
normalized imports
 | 
file |
diff |
annotate
 | 
| Wed, 04 Mar 2009 10:47:20 +0100 | 
nipkow | 
Made Option a separate theory and renamed option_map to Option.map
 | 
file |
diff |
annotate
 | 
| Thu, 26 Jun 2008 10:07:01 +0200 | 
haftmann | 
established Plain theory and image
 | 
file |
diff |
annotate
 | 
| Mon, 03 Mar 2008 14:03:19 +0100 | 
krauss | 
new theory of red-black trees, an efficient implementation of finite maps.
 | 
file |
diff |
annotate
 |