src/HOL/List.thy
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
Thu, 18 Feb 2010 14:21:44 -0800 huffman get rid of many duplicate simp rule warnings
Thu, 18 Feb 2010 16:08:26 +0100 nipkow added lemma
Wed, 17 Feb 2010 16:49:38 +0100 haftmann more lemmas about sort(_key)
Thu, 11 Feb 2010 23:00:22 +0100 wenzelm modernized translations;
Fri, 05 Feb 2010 14:33:50 +0100 haftmann more consistent naming of type classes involving orderings (and lattices) -- c.f. NEWS
Sun, 31 Jan 2010 14:51:32 +0100 haftmann canonical insert operation; generalized lemma foldl_apply_inv to foldl_apply
Thu, 21 Jan 2010 09:27:57 +0100 haftmann merged
Sat, 16 Jan 2010 17:15:28 +0100 haftmann dropped some old primrecs and some constdefs
Tue, 19 Jan 2010 17:53:11 +0100 hoelzl Added transpose_rectangle, when the input list is rectangular.
Tue, 19 Jan 2010 16:52:01 +0100 hoelzl Add transpose to the List-theory.
Fri, 15 Jan 2010 14:43:00 +0100 berghofe merged
Sun, 10 Jan 2010 18:09:11 +0100 berghofe same_append_eq / append_same_eq are now used for simplifying induction rules.
Wed, 13 Jan 2010 08:56:15 +0100 haftmann some syntax setup for Scala
Fri, 11 Dec 2009 14:43:55 +0100 haftmann avoid dependency on implicit dest rule predicate1D in proofs
Sat, 05 Dec 2009 20:02:21 +0100 haftmann tuned lattices theory fragements; generlized some lemmas from sets to lattices
Fri, 04 Dec 2009 12:22:09 +0100 haftmann merged
Mon, 30 Nov 2009 11:42:49 +0100 haftmann modernized structures and tuned headers of datatype package modules; joined former datatype.ML and datatype_rep_proofs.ML
Fri, 04 Dec 2009 08:26:25 +0100 nipkow added remdups_filter lemma
Thu, 12 Nov 2009 17:21:51 +0100 hoelzl Remove map_compose, replaced by map_map
Thu, 12 Nov 2009 17:21:48 +0100 hoelzl New list theorems; added map_map to simpset, this is the prefered direction; allow sorting by a key
Tue, 10 Nov 2009 16:11:37 +0100 haftmann tuned imports
Thu, 29 Oct 2009 11:41:36 +0100 haftmann moved Nat_Transfer before Divides; distributed Nat_Transfer setup accordingly
Sat, 17 Oct 2009 14:43:18 +0200 wenzelm eliminated hard tabulators, guessing at each author's individual tab-width;
Thu, 24 Sep 2009 18:29:29 +0200 haftmann lemma relating fold1 and foldl; code_unfold rules for Inf_fin, Sup_fin, Min, Max, Inf, Sup
Thu, 27 Aug 2009 11:41:07 +0200 nipkow code generator: quantifiers over {_.._::int} and {_..<_::nat}
Thu, 27 Aug 2009 09:28:52 +0200 nipkow tuned code generation for lists
Wed, 26 Aug 2009 19:54:01 +0200 nipkow got rid of complicated class finite_intvl_succ and defined "upto" directly on int, the only instance of the class.
Mon, 20 Jul 2009 09:52:09 +0200 haftmann merged
Wed, 15 Jul 2009 16:00:06 +0200 haftmann merged
Mon, 20 Jul 2009 08:32:07 +0200 haftmann merged
Tue, 14 Jul 2009 16:27:32 +0200 haftmann prefer code_inline over code_unfold; use code_unfold_post where appropriate
Wed, 15 Jul 2009 23:48:21 +0200 wenzelm more antiquotations;
Wed, 15 Jul 2009 20:34:58 +0200 nipkow Made "prime" executable
Wed, 15 Jul 2009 12:44:41 +0200 nipkow made upt/upto executable on nat/int by simp
Tue, 14 Jul 2009 10:54:04 +0200 haftmann code attributes use common underscore convention
Fri, 03 Jul 2009 08:44:13 +0200 haftmann lemma foldl_apply_inv
Tue, 23 Jun 2009 16:27:12 +0200 haftmann tuned interfaces of datatype module
Fri, 19 Jun 2009 17:23:21 +0200 haftmann discontinued ancient tradition to suffix certain ML module names with "_package"
Thu, 11 Jun 2009 23:24:28 +0200 nipkow two finiteness lemmas by Robert Himmelmann
Thu, 04 Jun 2009 15:28:59 +0200 haftmann lemma about List.foldl and Finite_Set.fold
Tue, 02 Jun 2009 13:59:32 +0200 hoelzl Added theorems about distinct & concat, map & replicate and concat & replicate
Wed, 27 May 2009 07:56:11 +0200 nipkow more lemmas
Tue, 26 May 2009 10:31:39 -0700 huffman listsum lemmas
less more (0) -300 -100 -60 tip