src/HOL/List.thy
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
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
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
less more (0) -120 tip