src/HOL/List.thy
Thu, 28 Apr 2005 12:04:34 +0200 more on rev
Thu, 28 Apr 2005 09:21:35 +0200 more about list_update
Mon, 11 Apr 2005 12:14:23 +0200 tuned Map, renamed lex stuff in List.
Tue, 05 Apr 2005 13:05:38 +0200 lexicographic order by Norbert Voelker
Thu, 03 Mar 2005 12:43:01 +0100 Move towards standard functions.
Sun, 13 Feb 2005 17:15:14 +0100 Deleted Library.option type.
Wed, 02 Feb 2005 18:19:43 +0100 Replaced application of subst by simplesubst in proof of rev_induct
Fri, 14 Jan 2005 12:00:27 +0100 made diff_less a simp rule
Tue, 04 Jan 2005 04:06:29 +0100 added list_all_rev
Wed, 22 Dec 2004 11:36:33 +0100 [ .. (] -> [ ..< ]
Thu, 09 Dec 2004 18:30:59 +0100 First step in reorganizing Finite_Set
Mon, 22 Nov 2004 13:52:27 +0100 indentation
Mon, 22 Nov 2004 11:53:56 +0100 added lemmas
Sun, 21 Nov 2004 18:39:25 +0100 Added more lemmas
Sun, 21 Nov 2004 15:44:20 +0100 added lemmas
Sun, 21 Nov 2004 12:52:03 +0100 Restructured List and added "rotate"
Sat, 13 Nov 2004 07:47:34 +0100 More lemmas
Tue, 19 Oct 2004 18:18:45 +0200 converted some induct_tac to induct
Fri, 15 Oct 2004 18:16:03 +0200 added and renamed
Thu, 14 Oct 2004 12:18:52 +0200 Added a few lemmas
Mon, 11 Oct 2004 07:42:22 +0200 Proofs needed to be updated because induction now preserves name of
Fri, 03 Sep 2004 10:26:39 +0200 listrel operator for lifting relations to lists
Wed, 01 Sep 2004 15:03:41 +0200 new functions for sets of lists
Wed, 18 Aug 2004 11:09:40 +0200 import -> imports
Mon, 16 Aug 2004 14:22:27 +0200 New theory header syntax.
Thu, 05 Aug 2004 10:50:58 +0200 some structured proofs
Wed, 04 Aug 2004 19:10:45 +0200 Added a number of new thms and the new function remove1
Thu, 22 Jul 2004 10:33:26 +0200 new material courtesy of Norbert Voelker
Mon, 19 Jul 2004 18:19:42 +0200 - Moved code generator setup for lists from Main.thy to List.thy
Thu, 15 Jul 2004 13:11:34 +0200 Moved to new m<..<n syntax for set intervals.
Mon, 21 Jun 2004 10:25:57 +0200 Merged in license change from Isabelle2004
Mon, 24 May 2004 18:35:34 +0200 added drop_take:thm
Fri, 21 May 2004 21:16:51 +0200 removed duplicate thms;
Fri, 16 Apr 2004 15:46:50 +0200 lemma drop_Suc_conv_tl added.
Fri, 16 Apr 2004 13:51:04 +0200 tuned document;
Wed, 14 Apr 2004 14:13:05 +0200 use more symbols in HTML output
Mon, 12 Apr 2004 19:54:32 +0200 removed o2l and fold_rel; moved postfix to Library/List_Prefix.thy
Tue, 30 Mar 2004 08:45:39 +0200 Added append_eq_append_conv2
Fri, 20 Feb 2004 01:32:59 +0100 moved lemmas from MicroJava/Comp/AuxLemmas.thy to List.thy
Thu, 19 Feb 2004 10:40:28 +0100 new theorem
Mon, 16 Feb 2004 03:25:52 +0100 lemmas about card (set xs)
Wed, 07 Jan 2004 07:52:12 +0100 map_idI
Mon, 05 Jan 2004 23:10:32 +0100 *** empty log message ***
Mon, 05 Jan 2004 22:43:03 +0100 *** empty log message ***
Wed, 24 Dec 2003 08:54:30 +0100 list_all2_nthD no good as [intro?]
Tue, 23 Dec 2003 23:40:16 +0100 list_all2_mono should not be [trans]
Tue, 23 Dec 2003 06:35:41 +0100 added some [intro?] and [trans] for list_all2 lemmas
Fri, 19 Dec 2003 04:28:45 +0100 *** empty log message ***
Thu, 18 Dec 2003 08:20:36 +0100 *** empty log message ***
Wed, 29 Oct 2003 01:17:06 +0100 *** empty log message ***
Fri, 26 Sep 2003 10:34:57 +0200 misc tidying
Sun, 14 Sep 2003 17:53:27 +0200 Added new theorems
Tue, 15 Jul 2003 08:25:20 +0200 Some new thm (ex_map_conv?)
Fri, 11 Jul 2003 14:12:02 +0200 added fold_red, o2l, postfix, some thms
Wed, 28 May 2003 10:47:54 +0200 new theorem
Wed, 14 May 2003 10:22:09 +0200 *** empty log message ***
Wed, 16 Apr 2003 22:14:08 +0200 Added take/dropWhile thms
Tue, 25 Mar 2003 09:58:51 +0100 Re-structured some proofs in order to get rid of rule_format attribute.
Fri, 14 Mar 2003 12:03:23 +0100 more about list_all2
Fri, 29 Nov 2002 09:48:28 +0100 added a few lemmas