src/HOL/List.thy
Sun, 13 Sep 2015 22:56:52 +0200 wenzelm tuned proofs -- less legacy;
Tue, 01 Sep 2015 22:32:58 +0200 wenzelm eliminated \<Colon>;
Thu, 27 Aug 2015 21:19:48 +0200 haftmann standardized some occurences of ancient "split" alias
Thu, 27 Aug 2015 13:07:45 +0200 haftmann more lemmas on sorting and multisets (due to Thomas Sewell)
Sat, 18 Jul 2015 22:58:50 +0200 wenzelm isabelle update_cartouches;
Sat, 18 Jul 2015 20:47:08 +0200 wenzelm prefer tactics with explicit context;
Thu, 25 Jun 2015 23:33:47 +0200 wenzelm tuned proofs;
Mon, 22 Jun 2015 11:15:23 +0200 nipkow modernized name
Thu, 30 Apr 2015 16:07:43 +0200 wenzelm more formal source, more PIDE markup;
Thu, 30 Apr 2015 15:58:15 +0200 wenzelm tuned -- avoid odd rebinding of "ctxt" and "context";
Thu, 30 Apr 2015 15:41:53 +0200 wenzelm tuned;
Wed, 29 Apr 2015 23:26:11 +0200 wenzelm tuned;
Tue, 17 Mar 2015 09:22:17 +0100 nipkow added lemmas
Wed, 04 Mar 2015 19:53:18 +0100 wenzelm tuned signature -- prefer qualified names;
Wed, 11 Feb 2015 13:58:51 +0100 Andreas Lochbihler add parametricity rules for monotone, fun_lub, and fun_ord
Mon, 29 Dec 2014 21:02:49 +0100 wenzelm tuned;
Tue, 11 Nov 2014 14:46:26 +0100 noschinl added lemma
Mon, 10 Nov 2014 10:29:19 +0100 traytel dropped redundant transfer rules (now proved and registered by datatype and plugins)
Sun, 09 Nov 2014 14:08:00 +0100 wenzelm proper context for compose_tac, Splitter.split_tac (relevant for unify trace options);
Fri, 07 Nov 2014 11:28:37 +0100 traytel more complete fp_sugars for sum and prod;
Sun, 02 Nov 2014 18:21:45 +0100 wenzelm modernized header uniformly as section;
Wed, 29 Oct 2014 12:01:39 +0100 nipkow removed useless lemmas
Wed, 29 Oct 2014 11:03:23 +0100 nipkow tuned layout and proofs
Wed, 24 Sep 2014 19:11:21 +0200 haftmann added lemmas
Thu, 11 Sep 2014 19:32:36 +0200 blanchet updated news
Tue, 09 Sep 2014 17:50:54 +0200 nipkow enamed drop_Suc_conv_tl and nth_drop' to Cons_nth_drop_Suc
Sat, 06 Sep 2014 20:12:32 +0200 haftmann added various facts
Tue, 02 Sep 2014 09:28:23 +0200 traytel silenced nonexhaustive primrec warnings
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
less more (0) -300 -100 -60 tip