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
Sat, 21 Apr 2012 06:49:04 +0200 huffman strengthen rule list_all2_induct
Thu, 12 Apr 2012 11:01:15 +0200 bulwahn merged
Tue, 03 Apr 2012 17:26:30 +0900 griff renamed "rel_comp" to "relcomp" (to be consistent with, e.g., "relpow")
Fri, 06 Apr 2012 19:23:51 +0200 haftmann abandoned almost redundant *_foldr lemmas
Fri, 06 Apr 2012 19:18:00 +0200 haftmann tuned
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
Mon, 26 Mar 2012 21:00:23 +0200 nipkow reverted to canonical name
Mon, 26 Mar 2012 18:54:41 +0200 nipkow Functions and lemmas by Christian Sternagel
Sun, 25 Mar 2012 20:15:39 +0200 huffman merged fork with new numeral representation (see NEWS)
Tue, 13 Mar 2012 13:31:26 +0100 wenzelm tuned proofs -- eliminated pointless chaining of facts after 'interpret';
Mon, 12 Mar 2012 21:41:11 +0100 noschinl tuned proofs
Mon, 27 Feb 2012 09:01:49 +0100 nipkow converting "set [...]" to "{...}" in evaluation results
Sat, 25 Feb 2012 09:07:37 +0100 bulwahn one general list_all2_update_cong instead of two special ones
Fri, 24 Feb 2012 22:46:44 +0100 haftmann moved predicate relations and conversion rules between set and predicate relations from Predicate.thy to Relation.thy; moved Predicate.thy upwards in theory hierarchy
Fri, 24 Feb 2012 09:40:02 +0100 haftmann given up disfruitful branch
Thu, 23 Feb 2012 21:25:59 +0100 haftmann moved predicate relations and conversion rules between set and predicate relations from Predicate.thy to Relation.thy; moved Predicate.thy upwards in theory hierarchy
Thu, 16 Feb 2012 09:18:23 +0100 bulwahn removing unnecessary premises in theorems of List theory
Fri, 10 Feb 2012 09:47:59 +0100 Cezary Kaliszyk more specification of the quotient package in IsarRef
Wed, 08 Feb 2012 01:49:33 +0100 blanchet use 'primrec' to define "rotate1", for uniformity (and to help first-order tools that rely on "Spec_Rules")
Wed, 08 Feb 2012 00:55:06 +0100 blanchet removed fact that confuses SPASS -- better rely on "rev_rev_ident", which is stronger and more ATP friendly
Sun, 05 Feb 2012 10:43:52 +0100 bulwahn adding code equation for Relation.image; adding map_project as correspondence to map_filter on lists
Sun, 05 Feb 2012 08:24:39 +0100 bulwahn another try to improve code generation of set equality (cf. da32cf32c0c7)
Thu, 02 Feb 2012 10:12:30 +0100 bulwahn adding a minimally refined equality on sets for code generation
Tue, 31 Jan 2012 15:39:45 +0100 bulwahn adding code equation for setsum
Mon, 23 Jan 2012 17:29:19 +0100 huffman generalize type of List.listrel
Mon, 23 Jan 2012 14:07:36 +0100 bulwahn adding code generation for some list relations
Tue, 10 Jan 2012 18:12:03 +0100 berghofe pred_subset/equals_eq are now standard pred_set_conv rules
Sat, 07 Jan 2012 20:44:23 +0100 haftmann massaging of code setup for sets
Sat, 07 Jan 2012 11:45:53 +0100 haftmann corrected slip
Sat, 07 Jan 2012 09:32:01 +0100 haftmann restore convenient code_abbrev declarations (particulary important if List.set is not the formal constructor for sets)
Fri, 06 Jan 2012 22:16:01 +0100 haftmann moved lemmas about List.set and set operations to List theory
Fri, 06 Jan 2012 20:39:50 +0100 haftmann farewell to theory More_List
Fri, 06 Jan 2012 17:44:42 +0100 wenzelm improved list comprehension syntax: more careful treatment of position constraints, which enables PIDE markup;
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)
Thu, 05 Jan 2012 18:18:39 +0100 wenzelm improved case syntax: more careful treatment of position constraints, which enables PIDE markup;
Thu, 29 Dec 2011 13:42:21 +0100 haftmann qualified Finite_Set.fold
Thu, 29 Dec 2011 10:47:55 +0100 haftmann attribute code_abbrev superseedes code_unfold_post; tuned text
Tue, 27 Dec 2011 09:15:26 +0100 haftmann dropped fact whose names clash with corresponding facts on canonical fold
Sat, 24 Dec 2011 15:53:10 +0100 haftmann dropped obsolete lemma member_set
Mon, 19 Dec 2011 14:41:08 +0100 noschinl add lemmas
Thu, 15 Dec 2011 18:08:40 +0100 wenzelm clarified module dependencies: Datatype_Data, Datatype_Case, Rep_Datatype;
Tue, 13 Dec 2011 22:44:16 +0100 noschinl added lemmas
Fri, 09 Dec 2011 13:42:16 +0100 huffman add induction rule for list_all2
Thu, 08 Dec 2011 13:53:27 +0100 bulwahn removing special code generator setup for hd and last function because this causes problems with quickcheck narrowing as the Haskell Prelude functions throw errors that cannot be caught instead of PatternFail exceptions
Thu, 01 Dec 2011 15:41:58 +0100 hoelzl cardinality of sets of lists
Sun, 20 Nov 2011 21:07:10 +0100 wenzelm eliminated obsolete "standard";
Wed, 19 Oct 2011 08:37:27 +0200 bulwahn removing old code generator setup for lists
Mon, 03 Oct 2011 14:43:12 +0200 bulwahn adding lemma to List library for executable equation of the (refl) transitive closure
Wed, 14 Sep 2011 10:08:52 -0400 hoelzl renamed Complete_Lattices lemmas, removed legacy names
Tue, 13 Sep 2011 17:07:33 -0700 huffman tuned proofs
Tue, 13 Sep 2011 12:14:29 +0200 bulwahn added lemma motivated by a more specific lemma in the AFP-KBPs theories
Mon, 12 Sep 2011 07:55:43 +0200 nipkow new fastforce replacing fastsimp - less confusing name
Thu, 01 Sep 2011 13:18:27 +0200 blanchet added two lemmas about "distinct" to help Sledgehammer
Tue, 30 Aug 2011 20:10:48 +0200 bulwahn adding list_size_append (thanks to Rene Thiemann)
Tue, 30 Aug 2011 20:10:47 +0200 bulwahn strengthening list_size_pointwise (thanks to Rene Thiemann)
Fri, 26 Aug 2011 11:22:47 +0200 nipkow added lemma
Tue, 02 Aug 2011 10:36:50 +0200 krauss moved recdef package to HOL/Library/Old_Recdef.thy
Wed, 29 Jun 2011 17:35:46 +0200 wenzelm modernized some simproc setup;
Mon, 27 Jun 2011 17:04:04 +0200 krauss new Datatype.info_of_constr with strict behaviour wrt. to overloaded constructors -- side effect: function package correctly identifies 0::int as a non-constructor;
Thu, 09 Jun 2011 16:34:49 +0200 wenzelm discontinued Name.variant to emphasize that this is old-style / indirect;
Fri, 20 May 2011 11:44:16 +0200 haftmann names of fold_set locales resemble name of characteristic property more closely
Sat, 14 May 2011 18:26:25 +0200 haftmann use pointfree characterisation for fold_set locale
Mon, 09 May 2011 16:11:20 +0200 noschinl add a lemma about commutative append to List.thy
Mon, 09 May 2011 12:26:25 +0200 noschinl removed assumption from lemma List.take_add
Tue, 19 Apr 2011 23:57:28 +0200 wenzelm eliminated Codegen.mode in favour of explicit argument;
Sat, 16 Apr 2011 16:15:37 +0200 wenzelm modernized structure Proof_Context;
Sat, 16 Apr 2011 15:25:25 +0200 wenzelm prefer local name spaces;
Wed, 06 Apr 2011 23:04:00 +0200 wenzelm separate structure Term_Position;
Wed, 30 Mar 2011 20:19:21 +0200 wenzelm actually check list comprehension examples;
Mon, 28 Mar 2011 23:49:53 +0200 wenzelm list comprehension: strip positions where the translation cannot handle them right now;
Tue, 22 Mar 2011 20:44:47 +0100 wenzelm more selective strip_positions in case patterns -- reactivate translations based on "case _ of _" in HOL and special patterns in HOLCF;
Tue, 15 Mar 2011 22:04:02 +0100 nipkow added lemma
Fri, 25 Feb 2011 14:25:41 +0100 nipkow added simp lemma nth_Cons_pos to List
Thu, 03 Feb 2011 18:57:42 +0100 wenzelm explicit is better than implicit;
Tue, 11 Jan 2011 14:12:37 +0100 haftmann "enriched_type" replaces less specific "type_lifting"
Fri, 07 Jan 2011 18:10:35 +0100 bulwahn adding simproc to rewrite list comprehensions to set comprehensions; adopting proofs
Tue, 21 Dec 2010 17:52:23 +0100 haftmann tuned type_lifting declarations
Fri, 17 Dec 2010 17:43:54 +0100 wenzelm replaced command 'nonterminals' by slightly modernized version 'nonterminal';
Wed, 08 Dec 2010 13:34:50 +0100 haftmann primitive definitions of bot/top/inf/sup for bool and fun are named with canonical suffix `_def` rather than `_eq`
Mon, 06 Dec 2010 09:19:10 +0100 haftmann replace `type_mapper` by the more adequate `type_lifting`
Sun, 28 Nov 2010 15:20:51 +0100 nipkow gave more standard finite set rules simp and intro attribute
Mon, 22 Nov 2010 11:34:58 +0100 bulwahn adding code equations for EX1 on finite types
Thu, 18 Nov 2010 17:01:16 +0100 haftmann mapper for list type; map_pair replaces prod_fun
Wed, 17 Nov 2010 21:35:23 +0100 nipkow code eqn for slice was missing; redefined splice with fun
Fri, 05 Nov 2010 08:16:34 +0100 bulwahn added two lemmas about injectivity of concat to the list theory
Tue, 02 Nov 2010 16:31:57 +0100 haftmann lemmas sorted_map_same, sorted_same
Thu, 28 Oct 2010 17:54:09 +0200 nipkow added lemmas about listrel(1)
Wed, 27 Oct 2010 16:40:31 +0200 haftmann sorting: avoid _key suffix if lemma applies both to simple and generalized variant; generalized insort_insert to insort_insert_key; additional lemmas
Tue, 26 Oct 2010 16:39:21 +0200 haftmann include ATP in theory List -- avoid theory edge by-passing the prominent list theory
Mon, 25 Oct 2010 13:34:58 +0200 haftmann dropped (almost) redundant distinct.induct rule; distinct_simps again named distinct.simps
Sun, 24 Oct 2010 20:19:00 +0200 nipkow nat_number -> eval_nat_numeral
Wed, 06 Oct 2010 17:44:21 +0200 blanchet merged
Mon, 04 Oct 2010 22:45:09 +0200 blanchet move Metis into Plain
Mon, 04 Oct 2010 12:22:58 +0200 haftmann turned distinct and sorted into inductive predicates: yields nice induction principles for free; more elegant proofs
Tue, 28 Sep 2010 15:21:45 +0200 haftmann localized listsum
Mon, 27 Sep 2010 14:13:22 +0200 haftmann lemma remdups_map_remdups
Wed, 22 Sep 2010 16:52:09 +0200 nipkow more lists lemmas
Tue, 21 Sep 2010 02:03:40 +0200 nipkow new lemma
Fri, 17 Sep 2010 20:53:50 +0200 haftmann generalized lemma insort_remove1 to insort_key_remove1
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
Fri, 10 Sep 2010 10:21:25 +0200 haftmann Haskell == is infix, not infixl
Tue, 07 Sep 2010 10:05:19 +0200 nipkow expand_fun_eq -> ext_iff
Thu, 02 Sep 2010 10:18:15 +0200 hoelzl Add filter_remove1
Fri, 27 Aug 2010 19:34:23 +0200 haftmann renamed class/constant eq to equal; tuned some instantiations
Wed, 25 Aug 2010 18:36:22 +0200 wenzelm renamed Simplifier.simproc(_i) to Simplifier.simproc_global(_i) to emphasize that this is not the real thing;
Mon, 19 Jul 2010 11:55:43 +0200 haftmann Scala: subtle difference in printing strings vs. complex mixfix syntax
Mon, 12 Jul 2010 10:48:37 +0200 haftmann dropped superfluous [code del]s
Mon, 28 Jun 2010 15:32:26 +0200 haftmann put section on distinctness before listsum; refined code generation operations; dropped ancient infix mem
Fri, 18 Jun 2010 21:22:05 +0200 haftmann merged
Fri, 18 Jun 2010 09:21:41 +0200 haftmann made List.thy a join point in the theory graph
Fri, 18 Jun 2010 20:22:06 +0200 nipkow tuned set_replicate lemmas
Fri, 18 Jun 2010 14:14:42 +0200 nipkow merged
Fri, 18 Jun 2010 14:14:29 +0200 nipkow added lemmas
Thu, 17 Jun 2010 16:15:15 +0200 haftmann rev is reverse in Haskell
Mon, 14 Jun 2010 12:01:30 +0200 haftmann use various predefined Haskell operations when generating code
Sat, 12 Jun 2010 15:47:50 +0200 haftmann declare lexn.simps [code del]
Wed, 02 Jun 2010 15:35:14 +0200 haftmann induction over non-empty lists
Wed, 26 May 2010 11:59:06 +0200 haftmann more convenient order of code equations
Mon, 24 May 2010 13:48:57 +0200 haftmann more lemmas
Thu, 20 May 2010 16:35:52 +0200 haftmann turned old-style mem into an input abbreviation
less more (0) -240 tip