src/HOL/List.thy
Sun, 31 Aug 2014 09:10:42 +0200 haftmann separated listsum material
Mon, 25 Aug 2014 16:06:41 +0200 nipkow added lemmas
Thu, 07 Aug 2014 12:17:41 +0200 blanchet no need for 'set_simps' now that 'datatype_new' generates the desired 'set' property
Mon, 21 Jul 2014 17:51:29 +0200 Andreas Lochbihler add parametricity lemmas
Sat, 19 Jul 2014 18:30:43 +0200 haftmann reverse induction over nonempty lists
Wed, 09 Jul 2014 11:48:21 +0200 nipkow added lemmas
Sat, 05 Jul 2014 11:01:53 +0200 haftmann prefer ac_simps collections over separate name bindings for add and mult
Fri, 04 Jul 2014 20:18:47 +0200 haftmann reduced name variants for assoc and commute on plus and mult
Sat, 28 Jun 2014 09:16:42 +0200 haftmann fact consolidation
Tue, 24 Jun 2014 15:05:58 +0200 Andreas Lochbihler add lemma
Thu, 12 Jun 2014 18:47:27 +0200 nipkow merged
Thu, 12 Jun 2014 18:47:16 +0200 nipkow added [simp]
Thu, 12 Jun 2014 17:02:03 +0200 blanchet reintroduced vital 'Thm.transfer'
Thu, 12 Jun 2014 01:00:49 +0200 blanchet reduces Sledgehammer dependencies
Tue, 10 Jun 2014 21:15:57 +0200 blanchet changed syntax of map: and rel: arguments to BNF-based datatypes
Tue, 10 Jun 2014 12:16:22 +0200 blanchet use 'where' clause for selector default value syntax
Mon, 09 Jun 2014 16:08:30 +0200 nipkow added List.union
Fri, 30 May 2014 12:27:51 +0200 blanchet tuned whitespace, to make datatype definitions slightly less intimidating
Mon, 26 May 2014 16:32:55 +0200 blanchet got rid of '=:' squiggly
Wed, 14 May 2014 11:33:38 +0200 nipkow added lemma
Tue, 29 Apr 2014 16:02:02 +0200 wenzelm prefer plain ASCII / latex over not-so-universal Unicode;
Wed, 23 Apr 2014 10:23:27 +0200 blanchet move size hooks together, with new one preceding old one and sharing same theory data
Sat, 12 Apr 2014 11:27:36 +0200 haftmann more operations and lemmas
Thu, 10 Apr 2014 17:48:54 +0200 kuncar make list_all an abbreviation of pred_list - prevent duplication
Thu, 10 Apr 2014 17:48:32 +0200 kuncar simplify and fix theories thanks to 356a5efdb278
Thu, 10 Apr 2014 17:48:15 +0200 kuncar abstract Domainp in relator_domain rules => more natural statement of the rule
Thu, 10 Apr 2014 17:48:15 +0200 kuncar more appropriate name (Lifting.invariant -> eq_onp)
Thu, 10 Apr 2014 17:48:14 +0200 kuncar left_total and left_unique rules are now transfer rules (cleaner solution, reflexvity_rule attribute not needed anymore)
Fri, 21 Mar 2014 11:42:32 +0100 wenzelm more qualified names;
Wed, 19 Mar 2014 18:47:22 +0100 haftmann elongated INFI and SUPR, to reduced risk of confusing theorems names in the future while still being consistent with INTER and UNION
Sun, 16 Mar 2014 18:09:04 +0100 haftmann normalising simp rules for compound operators
Thu, 13 Mar 2014 13:18:13 +0100 blanchet killed a few 'metis' calls
Thu, 06 Mar 2014 15:40:33 +0100 blanchet renamed 'fun_rel' to 'rel_fun'
Thu, 06 Mar 2014 15:29:18 +0100 blanchet renamed 'prod_rel' to 'rel_prod'
Thu, 06 Mar 2014 14:57:14 +0100 blanchet renamed 'set_rel' to 'rel_set'
Thu, 06 Mar 2014 13:36:48 +0100 blanchet renamed 'map_pair' to 'map_prod'
Fri, 28 Feb 2014 17:54:52 +0100 traytel load Metis a little later
Fri, 28 Feb 2014 18:09:37 +0100 nipkow added function "List.extract"
Fri, 21 Feb 2014 00:09:56 +0100 blanchet adapted to renaming of datatype 'cases' and 'recs' to 'case' and 'rec'
Wed, 19 Feb 2014 16:32:37 +0100 blanchet merged 'List.set' with BNF-generated 'set'
Tue, 18 Feb 2014 23:03:49 +0100 kuncar delete or move now not necessary reflexivity rules due to 1726f46d2aa8
Mon, 17 Feb 2014 13:31:42 +0100 blanchet renamed 'datatype_new_compat' to 'datatype_compat'
Sun, 16 Feb 2014 21:33:28 +0100 blanchet folded 'rel_option' into 'option_rel'
Sun, 16 Feb 2014 21:33:28 +0100 blanchet folded 'list_all2' with the relator generated by 'datatype_new'
Fri, 14 Feb 2014 07:53:46 +0100 blanchet hide 'rel' name -- this one is waiting to be merged with 'list_all2'
Fri, 14 Feb 2014 07:53:46 +0100 blanchet renamed 'enriched_type' to more informative 'functor' (following the renaming of enriched type constructors to bounded natural functors)
Fri, 14 Feb 2014 07:53:46 +0100 blanchet merged 'Option.map' and 'Option.map_option'
Fri, 14 Feb 2014 07:53:45 +0100 blanchet merged 'List.map' and 'List.list.map'
Wed, 12 Feb 2014 17:35:59 +0100 blanchet tuning
Wed, 12 Feb 2014 08:37:06 +0100 blanchet adapted to 'xxx_{case,rec}' renaming, to new theorem names, and to new variable names in theorems
Wed, 12 Feb 2014 08:35:57 +0100 blanchet renamed 'nat_{case,rec}' to '{case,rec}_nat'
Wed, 12 Feb 2014 08:35:56 +0100 blanchet compatibility names
Wed, 12 Feb 2014 08:35:56 +0100 blanchet use new selector support to define 'the', 'hd', 'tl'
Wed, 12 Feb 2014 08:35:56 +0100 blanchet transformed 'option' and 'list' into new-style datatypes (but register them as old-style as well)
Sat, 25 Jan 2014 23:50:49 +0100 haftmann avoid (now superfluous) indirect passing of constant names
Sat, 25 Jan 2014 23:50:49 +0100 haftmann prefer explicit code symbol type over ad-hoc name mangling
Fri, 24 Jan 2014 11:51:45 +0100 blanchet killed 'More_BNFs' by moving its various bits where they (now) belong
Wed, 01 Jan 2014 01:05:48 +0100 haftmann fundamental treatment of undefined vs. universally partial replaces code_abort
Tue, 31 Dec 2013 22:18:31 +0100 haftmann more abstract declaration of code attributes
Fri, 27 Dec 2013 14:35:14 +0100 haftmann prefer target-style syntaxx for sublocale
Wed, 25 Dec 2013 17:39:06 +0100 haftmann prefer more canonical names for lemmas on min/max
Wed, 27 Nov 2013 11:08:55 +0100 Andreas Lochbihler remove junk
Wed, 27 Nov 2013 10:43:51 +0100 Andreas Lochbihler merged
Wed, 20 Nov 2013 10:59:12 +0100 Andreas Lochbihler add predicate version of lexicographic order on lists
Thu, 21 Nov 2013 21:33:34 +0100 blanchet rationalize imports
Tue, 19 Nov 2013 17:07:52 +0100 hoelzl merged
Mon, 18 Nov 2013 17:14:01 +0100 hoelzl add lemmas Suc_funpow and id_funpow to simpset; add lemma map_add_upt
Tue, 19 Nov 2013 10:05:53 +0100 haftmann eliminiated neg_numeral in favour of - (numeral _)
Tue, 12 Nov 2013 13:47:24 +0100 blanchet port list comprehension simproc to 'Ctr_Sugar' abstraction
Sun, 10 Nov 2013 15:05:06 +0100 haftmann qualifed popular user space names
Fri, 18 Oct 2013 10:43:20 +0200 blanchet killed most "no_atp", to make Sledgehammer more complete
Fri, 27 Sep 2013 15:38:23 +0200 nipkow added code eqns for bounded LEAST operator
Thu, 26 Sep 2013 13:37:33 +0200 lammich Added symmetric code_unfold-lemmas for null and is_none
Wed, 18 Sep 2013 18:11:32 +0200 traytel added two functions to List (one contributed by Manuel Eberl)
Wed, 18 Sep 2013 12:16:10 +0200 nipkow added and tuned lemmas
Thu, 05 Sep 2013 11:10:51 +0200 traytel list_to_set_comprehension: don't crash in case distinctions on datatypes with even number of constructors
Tue, 03 Sep 2013 01:12:40 +0200 wenzelm tuned proofs -- clarified flow of facts wrt. calculation;
Tue, 13 Aug 2013 17:45:22 +0200 wenzelm merged
Tue, 13 Aug 2013 16:25:47 +0200 wenzelm standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;
Tue, 13 Aug 2013 15:59:22 +0200 kuncar move Lifting/Transfer relevant parts of Library/Quotient_* to Main
Sun, 23 Jun 2013 21:16:07 +0200 haftmann migration from code_(const|type|class|instance) to code_printing and from code_module to code_identifier
Sat, 15 Jun 2013 17:19:23 +0200 haftmann lifting for primitive definitions;
Sat, 15 Jun 2013 17:19:23 +0200 haftmann selection operator smallest_prime_beyond
Sat, 25 May 2013 18:30:38 +0200 wenzelm merged
Sat, 25 May 2013 15:37:53 +0200 wenzelm syntax translations always depend on context;
Sat, 25 May 2013 15:44:29 +0200 haftmann weaker precendence of syntax for big intersection and union on sets
Fri, 24 May 2013 17:00:46 +0200 wenzelm tuned signature;
Thu, 23 May 2013 14:22:49 +0200 noschinl more lemmas for sorted_list_of_set
Mon, 06 May 2013 02:48:18 +0200 nipkow tail recursive version of map, for code generation, optionally
Tue, 23 Apr 2013 11:14:51 +0200 haftmann tuned: unnamed contexts, interpretation and sublocale in locale target;
Thu, 18 Apr 2013 17:07:01 +0200 wenzelm simplifier uses proper Proof.context instead of historic type simpset;
Fri, 05 Apr 2013 22:08:42 +0200 traytel allow redundant cases in the list comprehension translation
Tue, 22 Jan 2013 14:33:45 +0100 traytel separate data used for case translation from the datatype package
Tue, 22 Jan 2013 13:32:41 +0100 berghofe case translations performed in a separate check phase (with adjustments by traytel)
Wed, 27 Mar 2013 10:55:05 +0100 haftmann centralized various multiset operations in theory multiset;
Tue, 26 Mar 2013 20:49:57 +0100 haftmann explicit sublocale dependency for Min/Max yields more appropriate Min/Max prefix for a couple of facts
Sat, 23 Mar 2013 20:50:39 +0100 haftmann fundamental revision of big operators on sets
Thu, 28 Feb 2013 17:14:55 +0100 wenzelm provide common HOLogic.conj_conv and HOLogic.eq_conv;
Thu, 28 Feb 2013 16:54:52 +0100 wenzelm just one HOLogic.Trueprop_conv, with regular exception CTERM;
Mon, 25 Feb 2013 12:17:50 +0100 wenzelm prefer stateless 'ML_val' for tests;
Sun, 17 Feb 2013 21:29:30 +0100 haftmann Sieve of Eratosthenes
Sun, 17 Feb 2013 11:34:40 +0100 haftmann simplified construction of upto_aux
Sat, 16 Feb 2013 15:27:10 +0100 nipkow tail recursive code for function "upto"
Fri, 15 Feb 2013 11:47:33 +0100 haftmann systematic conversions between nat and nibble/char;
Thu, 14 Feb 2013 12:24:42 +0100 haftmann abandoned theory Plain
Wed, 13 Feb 2013 13:38:52 +0100 haftmann combinator List.those;
Fri, 14 Dec 2012 19:51:20 +0100 nipkow unified layout of defs
Fri, 07 Dec 2012 16:25:33 +0100 wenzelm avoid ML_file in large theory files to improve performance of dependency discovery of main HOL (approx. 1s CPU time) -- relevant for any application using it, e.g. small paper sessions;
Tue, 20 Nov 2012 18:59:35 +0100 hoelzl add Countable_Set theory
Thu, 08 Nov 2012 11:59:48 +0100 bulwahn adjusting proofs as the set_comprehension_pointfree simproc breaks some existing proofs
Sun, 21 Oct 2012 17:04:13 +0200 webertj merged
Fri, 19 Oct 2012 15:12:52 +0200 webertj Renamed {left,right}_distrib to distrib_{right,left}.
Sat, 20 Oct 2012 09:12:16 +0200 haftmann moved quite generic material from theory Enum to more appropriate places
Wed, 10 Oct 2012 15:16:44 +0200 Andreas Lochbihler tail-recursive implementation for length
Tue, 09 Oct 2012 16:57:58 +0200 kuncar rename Set.project to Set.filter - more appropriate name
Mon, 08 Oct 2012 12:03:49 +0200 haftmann consolidated names of theorems on composition;
Wed, 22 Aug 2012 22:55:41 +0200 wenzelm prefer ML_file over old uses;
Thu, 16 Aug 2012 14:07:32 +0200 haftmann prefer eta-expanded code equations for fold, to accomodate tail recursion optimisation in Scala
Tue, 31 Jul 2012 13:55:39 +0200 kuncar more set operations expressed by Finite_Set.fold
Mon, 30 Apr 2012 12:14:53 +0200 bulwahn making sorted_list_of_set executable
less more (0) -120 tip