src/HOL/List.thy
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
Fri, 14 May 2010 22:46:41 +0200 nipkow added listsum lemmas
Thu, 13 May 2010 14:34:05 +0200 nipkow Multiset: renamed, added and tuned lemmas;
Wed, 12 May 2010 11:17:59 +0200 haftmann added lemmas concerning last, butlast, insort
Tue, 20 Apr 2010 17:58:34 +0200 hoelzl Generalize swap_inj_on; add simps for Times; add Ex_list_of_length, log_inj; Added missing locale edges for linordered semiring with 1.
Thu, 22 Apr 2010 09:30:39 +0200 haftmann lemmas concerning remdups
Mon, 19 Apr 2010 07:38:35 +0200 haftmann merged
Mon, 19 Apr 2010 07:38:08 +0200 haftmann more convenient equations for zip
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 16:55:12 +0200 Cezary Kaliszyk Respectfullness and preservation of list_rel
Thu, 18 Mar 2010 12:58:52 +0100 blanchet now use "Named_Thms" for "noatp", and renamed "noatp" to "no_atp"
Wed, 17 Mar 2010 19:37:44 +0100 blanchet renamed "ATP_Linkup" theory to "Sledgehammer"
Sat, 06 Mar 2010 09:58:33 +0100 haftmann added insort_insert
Fri, 05 Mar 2010 17:55:14 +0100 haftmann moved lemma map_sorted_distinct_set_unique
Tue, 02 Mar 2010 17:36:16 +0000 paulson Slightly generalised a theorem
Mon, 22 Feb 2010 09:24:20 +0100 haftmann merged
Sat, 20 Feb 2010 21:13:29 +0100 haftmann lemma distinct_insert
Mon, 22 Feb 2010 09:17:49 +0100 haftmann merged
Fri, 19 Feb 2010 14:47:01 +0100 haftmann moved remaning class operations from Algebras.thy to Groups.thy
Sun, 21 Feb 2010 21:10:01 +0100 wenzelm adapted to authentic syntax;
Sat, 20 Feb 2010 16:20:38 +0100 nipkow added lemma
Thu, 18 Feb 2010 14:28:26 -0800 huffman merged
less more (0) -300 -100 -60 tip