src/HOL/List.thy
Fri, 12 May 2006 11:19:41 +0200 nipkow added lemma in_measure
Tue, 09 May 2006 14:18:40 +0200 haftmann introduced characters for code generator; some improved code lemmas for some list functions
Sun, 07 May 2006 00:22:05 +0200 wenzelm removed 'concl is' patterns;
Thu, 27 Apr 2006 17:40:17 +0200 nipkow added zip/take/drop lemmas
Sun, 09 Apr 2006 19:41:30 +0200 nipkow Added function "splice"
Sat, 08 Apr 2006 22:51:06 +0200 wenzelm refined 'abbreviation';
Tue, 21 Mar 2006 12:18:10 +0100 wenzelm abbreviation upto, length;
Sat, 25 Feb 2006 15:19:47 +0100 haftmann improved codegen bootstrap
Mon, 23 Jan 2006 14:07:52 +0100 haftmann removed problematic keyword 'atom'
Thu, 19 Jan 2006 21:22:08 +0100 wenzelm setup: theory -> theory;
Wed, 18 Jan 2006 11:55:50 +0100 haftmann substantial improvement in serialization handling
Tue, 17 Jan 2006 16:36:57 +0100 haftmann substantial improvements in code generator
Mon, 09 Jan 2006 13:27:44 +0100 paulson theorems need names
Thu, 22 Dec 2005 13:00:53 +0100 nipkow new lemmas
Wed, 21 Dec 2005 15:18:17 +0100 haftmann slight clean ups
Wed, 21 Dec 2005 12:02:57 +0100 paulson removed or modified some instances of [iff]
Fri, 16 Dec 2005 16:59:32 +0100 nipkow new lemmas
Fri, 02 Dec 2005 16:43:42 +0100 krauss Added recdef congruence rules for bounded quantifiers and commonly used
Mon, 31 Oct 2005 01:43:22 +0100 nipkow A few new lemmas
Fri, 21 Oct 2005 18:14:34 +0200 wenzelm Goal.prove;
Wed, 19 Oct 2005 06:46:45 +0200 nipkow added 2 lemmas
Mon, 17 Oct 2005 23:10:15 +0200 wenzelm Simplifier.inherit_context instead of Simplifier.inherit_bounds;
Tue, 11 Oct 2005 17:30:00 +0200 nipkow added hd lemma
Wed, 05 Oct 2005 14:01:32 +0200 nipkow added last in set lemma
Tue, 04 Oct 2005 23:39:42 +0200 nipkow new hd/rev/last lemmas
Thu, 29 Sep 2005 17:02:57 +0200 paulson simprules need names
Sat, 24 Sep 2005 21:13:15 +0200 nipkow a few new filter lemmas
Thu, 22 Sep 2005 23:56:15 +0200 nipkow renamed rules to iprover
Tue, 20 Sep 2005 13:17:55 +0200 nipkow added a number of lemmas
Wed, 17 Aug 2005 11:44:02 +0200 nipkow small mods to code lemmas
Tue, 16 Aug 2005 19:25:32 +0200 nipkow added quite a few functions for code generation
Tue, 02 Aug 2005 13:13:18 +0200 nipkow Added filter lemma
Mon, 01 Aug 2005 19:20:26 +0200 wenzelm simprocs: Simplifier.inherit_bounds;
Mon, 01 Aug 2005 11:24:19 +0200 nipkow added map_filter lemmas
Tue, 12 Jul 2005 11:51:31 +0200 berghofe Auxiliary functions to be used in generated code are now defined using "attach".
Fri, 01 Jul 2005 13:54:57 +0200 berghofe Adapted to new interface of code generator.
Wed, 15 Jun 2005 11:54:13 +0200 nipkow added lemmas
Thu, 28 Apr 2005 12:04:34 +0200 kleing more on rev
Thu, 28 Apr 2005 09:21:35 +0200 kleing more about list_update
Mon, 11 Apr 2005 12:14:23 +0200 nipkow tuned Map, renamed lex stuff in List.
Tue, 05 Apr 2005 13:05:38 +0200 paulson lexicographic order by Norbert Voelker
Thu, 03 Mar 2005 12:43:01 +0100 skalberg Move towards standard functions.
Sun, 13 Feb 2005 17:15:14 +0100 skalberg Deleted Library.option type.
Wed, 02 Feb 2005 18:19:43 +0100 berghofe Replaced application of subst by simplesubst in proof of rev_induct
Fri, 14 Jan 2005 12:00:27 +0100 nipkow made diff_less a simp rule
Tue, 04 Jan 2005 04:06:29 +0100 kleing added list_all_rev
Wed, 22 Dec 2004 11:36:33 +0100 nipkow [ .. (] -> [ ..< ]
Thu, 09 Dec 2004 18:30:59 +0100 nipkow First step in reorganizing Finite_Set
Mon, 22 Nov 2004 13:52:27 +0100 paulson indentation
Mon, 22 Nov 2004 11:53:56 +0100 nipkow added lemmas
Sun, 21 Nov 2004 18:39:25 +0100 nipkow Added more lemmas
Sun, 21 Nov 2004 15:44:20 +0100 nipkow added lemmas
Sun, 21 Nov 2004 12:52:03 +0100 nipkow Restructured List and added "rotate"
Sat, 13 Nov 2004 07:47:34 +0100 nipkow More lemmas
Tue, 19 Oct 2004 18:18:45 +0200 paulson converted some induct_tac to induct
Fri, 15 Oct 2004 18:16:03 +0200 nipkow added and renamed
Thu, 14 Oct 2004 12:18:52 +0200 nipkow Added a few lemmas
Mon, 11 Oct 2004 07:42:22 +0200 nipkow Proofs needed to be updated because induction now preserves name of
Fri, 03 Sep 2004 10:26:39 +0200 paulson listrel operator for lifting relations to lists
Wed, 01 Sep 2004 15:03:41 +0200 paulson new functions for sets of lists
Wed, 18 Aug 2004 11:09:40 +0200 nipkow import -> imports
Mon, 16 Aug 2004 14:22:27 +0200 nipkow New theory header syntax.
Thu, 05 Aug 2004 10:50:58 +0200 paulson some structured proofs
Wed, 04 Aug 2004 19:10:45 +0200 nipkow Added a number of new thms and the new function remove1
Thu, 22 Jul 2004 10:33:26 +0200 paulson new material courtesy of Norbert Voelker
Mon, 19 Jul 2004 18:19:42 +0200 berghofe - Moved code generator setup for lists from Main.thy to List.thy
Thu, 15 Jul 2004 13:11:34 +0200 nipkow Moved to new m<..<n syntax for set intervals.
Mon, 21 Jun 2004 10:25:57 +0200 kleing Merged in license change from Isabelle2004
Mon, 24 May 2004 18:35:34 +0200 nipkow added drop_take:thm
Fri, 21 May 2004 21:16:51 +0200 wenzelm removed duplicate thms;
Fri, 16 Apr 2004 15:46:50 +0200 mehta lemma drop_Suc_conv_tl added.
Fri, 16 Apr 2004 13:51:04 +0200 wenzelm tuned document;
Wed, 14 Apr 2004 14:13:05 +0200 kleing use more symbols in HTML output
Mon, 12 Apr 2004 19:54:32 +0200 oheimb removed o2l and fold_rel; moved postfix to Library/List_Prefix.thy
Tue, 30 Mar 2004 08:45:39 +0200 nipkow Added append_eq_append_conv2
Fri, 20 Feb 2004 01:32:59 +0100 nipkow moved lemmas from MicroJava/Comp/AuxLemmas.thy to List.thy
Thu, 19 Feb 2004 10:40:28 +0100 paulson new theorem
Mon, 16 Feb 2004 03:25:52 +0100 kleing lemmas about card (set xs)
Wed, 07 Jan 2004 07:52:12 +0100 kleing map_idI
Mon, 05 Jan 2004 23:10:32 +0100 nipkow *** empty log message ***
Mon, 05 Jan 2004 22:43:03 +0100 nipkow *** empty log message ***
Wed, 24 Dec 2003 08:54:30 +0100 kleing list_all2_nthD no good as [intro?]
Tue, 23 Dec 2003 23:40:16 +0100 kleing list_all2_mono should not be [trans]
Tue, 23 Dec 2003 06:35:41 +0100 kleing added some [intro?] and [trans] for list_all2 lemmas
Fri, 19 Dec 2003 04:28:45 +0100 nipkow *** empty log message ***
Thu, 18 Dec 2003 08:20:36 +0100 nipkow *** empty log message ***
Wed, 29 Oct 2003 01:17:06 +0100 nipkow *** empty log message ***
Fri, 26 Sep 2003 10:34:57 +0200 paulson misc tidying
Sun, 14 Sep 2003 17:53:27 +0200 nipkow Added new theorems
Tue, 15 Jul 2003 08:25:20 +0200 nipkow Some new thm (ex_map_conv?)
Fri, 11 Jul 2003 14:12:02 +0200 oheimb added fold_red, o2l, postfix, some thms
Wed, 28 May 2003 10:47:54 +0200 paulson new theorem
Wed, 14 May 2003 10:22:09 +0200 nipkow *** empty log message ***
Wed, 16 Apr 2003 22:14:08 +0200 nipkow Added take/dropWhile thms
Tue, 25 Mar 2003 09:58:51 +0100 berghofe Re-structured some proofs in order to get rid of rule_format attribute.
Fri, 14 Mar 2003 12:03:23 +0100 kleing more about list_all2
Fri, 29 Nov 2002 09:48:28 +0100 nipkow added a few lemmas
Mon, 30 Sep 2002 16:14:02 +0200 berghofe Adapted to new simplifier.
Thu, 26 Sep 2002 10:51:29 +0200 paulson Converted Fun to Isar style.
Wed, 21 Aug 2002 15:53:30 +0200 paulson Frederic Blanqui's new "guard" examples
Thu, 08 Aug 2002 23:46:09 +0200 wenzelm use Tactic.prove instead of prove_goalw_cterm in internal proofs!
Tue, 06 Aug 2002 11:22:05 +0200 wenzelm sane interface for simprocs;
Tue, 16 Jul 2002 18:26:36 +0200 wenzelm moved stuff from Main.thy;
Thu, 30 May 2002 10:12:52 +0200 nipkow Modifications due to enhanced linear arithmetic.
Mon, 13 May 2002 15:45:21 +0200 nipkow *** empty log message ***
Mon, 13 May 2002 15:39:56 +0200 nipkow *** empty log message ***
Mon, 13 May 2002 15:27:28 +0200 nipkow *** empty log message ***
Mon, 13 May 2002 11:05:27 +0200 wenzelm tuned document;
Wed, 08 May 2002 13:01:40 +0200 nipkow new thm distinct_conv_nth
Wed, 08 May 2002 12:15:30 +0200 wenzelm oops;
Tue, 07 May 2002 19:54:29 +0200 wenzelm converted;
Thu, 14 Feb 2002 11:50:52 +0100 nipkow nodups -> distinct
Fri, 09 Nov 2001 00:09:47 +0100 wenzelm eliminated old "symbols" syntax, use "xsymbols" instead;
Tue, 09 Jan 2001 15:22:13 +0100 nipkow `` -> and ``` -> ``
Sun, 16 Jul 2000 20:49:56 +0200 wenzelm avoid 'split';
Fri, 14 Jul 2000 16:28:49 +0200 oheimb tuned syntax
Fri, 14 Jul 2000 14:47:15 +0200 paulson moved sublist from UNITY/AllocBase to List
Fri, 26 May 2000 18:04:17 +0200 paulson named the primrec clauses of upt
Thu, 25 May 2000 15:14:20 +0200 paulson better indentation; declared function "null"
Mon, 15 May 2000 17:30:19 +0200 berghofe Removed unnecessary primrec equations of hd and last involving arbitrary.
less more (0) -120 tip