src/HOL/List.thy
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
Tue, 19 May 2009 13:52:12 +0200 nipkow new lemma
Fri, 15 May 2009 10:01:57 +0200 nipkow new lemma
Thu, 14 May 2009 15:09:47 +0200 haftmann preprocessing must consider eq
Sat, 09 May 2009 07:25:22 +0200 nipkow lemmas by Andreas Lochbihler
Fri, 08 May 2009 08:06:43 +0200 nipkow more lemmas
Wed, 06 May 2009 19:09:31 +0200 haftmann proper structures for list and string code generation stuff
Wed, 06 May 2009 16:01:06 +0200 haftmann refined HOL string theories and corresponding ML fragments
Wed, 29 Apr 2009 21:10:46 +0200 nipkow added listsum lemmas
Fri, 24 Apr 2009 17:45:15 +0200 haftmann funpow and relpow with shared "^^" syntax
Mon, 20 Apr 2009 09:32:07 +0200 haftmann power operation on functions with syntax o^; power operation on relations with syntax ^^
Fri, 17 Apr 2009 15:57:26 +0200 haftmann separated funpow, relpow from power on monoids
Wed, 04 Mar 2009 11:05:29 +0100 blanchet Merge.
Wed, 04 Mar 2009 10:45:52 +0100 blanchet Merge.
Mon, 02 Mar 2009 16:53:55 +0100 nipkow name changes
Thu, 26 Feb 2009 08:44:12 -0800 huffman revert some Suc 0 lemmas back to their original forms; added some simp rules for (1::nat)
Mon, 23 Feb 2009 16:25:52 -0800 huffman make proofs work whether or not One_nat_def is a simp rule; replace 1 with Suc 0 in the rhs of some simp rules
Fri, 20 Feb 2009 10:14:32 +0100 haftmann defensive implementation of pretty serialisation of lists and characters
Mon, 16 Feb 2009 10:13:30 +0100 blanchet Added nitpick attribute, and fixed typo.
Tue, 10 Feb 2009 17:53:51 -0800 huffman const_name antiquotations
Sat, 07 Feb 2009 09:57:07 +0100 haftmann code theorems for nth, list_update
Sat, 07 Feb 2009 08:37:43 +0100 haftmann code theorems for nth, list_update
Fri, 06 Feb 2009 15:15:27 +0100 haftmann authentic syntax for List.nth
Tue, 03 Feb 2009 16:39:52 +0100 haftmann dropped global Nil/Append interpretation
Mon, 26 Jan 2009 08:23:41 +0100 haftmann sorted_take, sorted_drop
Fri, 16 Jan 2009 14:58:11 +0100 haftmann migrated class package to new locale implementation
Wed, 31 Dec 2008 20:31:36 +0100 wenzelm eliminated OldTerm.add_term_free_names;
Wed, 31 Dec 2008 18:53:16 +0100 wenzelm moved old add_type_XXX, add_term_XXX etc. to structure OldTerm;
Thu, 11 Dec 2008 18:30:26 +0100 ballarin Conversion of HOL-Main and ZF to new locales.
Thu, 04 Dec 2008 14:43:33 +0100 haftmann cleaned up binding module and related code
Mon, 17 Nov 2008 17:00:55 +0100 haftmann tuned unfold_locales invocation
Fri, 14 Nov 2008 08:50:07 +0100 haftmann added length_unique operation for code generation
Wed, 29 Oct 2008 11:33:40 +0100 haftmann explicit check for pattern discipline before code translation
Wed, 22 Oct 2008 14:15:45 +0200 haftmann code identifier namings are no longer imperative
Mon, 20 Oct 2008 23:52:59 +0200 nipkow added lemmas
Fri, 10 Oct 2008 06:45:53 +0200 haftmann `code func` now just `code`
Thu, 09 Oct 2008 08:47:27 +0200 haftmann established canonical argument order in SML code generators
Tue, 07 Oct 2008 16:07:20 +0200 haftmann dropped superfluous if
Fri, 26 Sep 2008 09:10:02 +0200 haftmann removed obsolete name convention "func"
Thu, 25 Sep 2008 09:28:03 +0200 haftmann discontinued special treatment of op = vs. eq_class.eq
Wed, 17 Sep 2008 21:27:08 +0200 wenzelm back to dynamic the_context(), because static @{theory} is invalidated if ML environment changes within the same code block;
Tue, 16 Sep 2008 16:13:09 +0200 haftmann a sophisticated char/nibble conversion combinator
Tue, 16 Sep 2008 09:21:27 +0200 haftmann explicit size of characters
Tue, 02 Sep 2008 20:38:17 +0200 haftmann distributed literal code generation out of central infrastructure
Mon, 01 Sep 2008 22:10:42 +0200 nipkow It appears that the code generator (Stefan's) needs some laws that appear superfluous: {..n} = set ...
Mon, 01 Sep 2008 19:16:40 +0200 nipkow cleaned up code generation for {.._} and {..<_}
Mon, 01 Sep 2008 10:18:37 +0200 haftmann restructured code generation of literals
Thu, 28 Aug 2008 22:09:20 +0200 haftmann restructured and split code serializer module
Fri, 01 Aug 2008 12:57:50 +0200 nipkow made setsum executable on int.
Tue, 29 Jul 2008 13:16:54 +0200 nipkow added removeAll
Sat, 28 Jun 2008 21:21:13 +0200 wenzelm @{lemma}: 'by' keyword;
Thu, 26 Jun 2008 10:07:01 +0200 haftmann established Plain theory and image
Tue, 10 Jun 2008 15:30:56 +0200 haftmann removed some dubious code lemmas
Fri, 23 May 2008 16:41:39 +0200 berghofe Replaced Pretty.str and Pretty.string_of by specific functions (from Codegen) that
Mon, 12 May 2008 22:11:06 +0200 krauss Measure functions can now be declared via special rules, allowing for a
Wed, 07 May 2008 10:56:37 +0200 berghofe - Explicitely applied predicate1I in a few proofs, because it is no longer
Fri, 02 May 2008 18:01:02 +0200 nipkow Added documentation
Fri, 25 Apr 2008 16:28:06 +0200 krauss * New attribute "termination_simp": Simp rules for termination proofs
Tue, 22 Apr 2008 08:33:20 +0200 haftmann dropped some metis calls
Wed, 09 Apr 2008 05:30:14 +0200 huffman move lemmas from Word/BinBoolList.thy to List.thy
Sat, 29 Mar 2008 19:14:00 +0100 wenzelm replaced 'ML_setup' by 'ML';
Thu, 27 Mar 2008 19:04:36 +0100 haftmann restructuring; explicit case names for rule list_induct2
Mon, 17 Mar 2008 18:37:00 +0100 wenzelm removed duplicate lemmas;
Tue, 26 Feb 2008 20:38:13 +0100 haftmann char and nibble are finite
Tue, 26 Feb 2008 11:18:43 +0100 bulwahn Added useful general lemmas from the work with the HeapMonad
Fri, 15 Feb 2008 17:36:21 +0100 nipkow more lemmas
Fri, 25 Jan 2008 14:54:44 +0100 haftmann dropped superfluous code theorems
Thu, 10 Jan 2008 19:09:21 +0100 berghofe New interface for test data generators.
Mon, 10 Dec 2007 11:24:03 +0100 haftmann swtiched ATP_Linkup and PreList in theory hierarchy
Fri, 07 Dec 2007 15:07:59 +0100 haftmann instantiation target rather than legacy instance
Thu, 06 Dec 2007 17:05:44 +0100 haftmann temporary code generator work arounds
Thu, 06 Dec 2007 16:36:19 +0100 haftmann authentic primrec
Thu, 29 Nov 2007 17:08:26 +0100 haftmann instance command as rudimentary class target
Mon, 05 Nov 2007 22:49:28 +0100 kleing rev_nth
Mon, 05 Nov 2007 18:18:39 +0100 nipkow added lemmas
Mon, 05 Nov 2007 08:31:12 +0100 nipkow added lemmas
Sun, 28 Oct 2007 13:18:00 +0100 wenzelm append/member: more light-weight way to declare authentic syntax;
Sat, 27 Oct 2007 15:53:23 +0200 krauss use "fun" for definition of "member" -> authentic syntax
Tue, 23 Oct 2007 23:27:23 +0200 nipkow went back to >0
Tue, 23 Oct 2007 13:10:19 +0200 paulson random tidying of proofs
Sun, 21 Oct 2007 14:53:44 +0200 nipkow Eliminated most of the neq0_conv occurrences. As a result, many
Sun, 21 Oct 2007 14:21:45 +0200 wenzelm avoid very slow metis invocation;
Sat, 20 Oct 2007 12:09:33 +0200 chaieb fixed proofs
Thu, 18 Oct 2007 16:09:36 +0200 haftmann tuned
Wed, 17 Oct 2007 18:09:38 +0200 nipkow added sorted_list_of_set
Tue, 16 Oct 2007 23:12:45 +0200 haftmann global class syntax
Mon, 08 Oct 2007 16:28:29 +0200 berghofe list_codegen and char_codegen now call invoke_tycodegen to ensure
Mon, 01 Oct 2007 19:21:32 +0200 haftmann added some lemmas
Sat, 29 Sep 2007 08:58:51 +0200 haftmann proper syntax during class specification
Tue, 25 Sep 2007 12:59:24 +0200 ballarin Simplified proof due to improved integration of order_tac and simp.
Tue, 25 Sep 2007 10:27:43 +0200 nipkow hide successor
Mon, 24 Sep 2007 22:00:18 +0200 nipkow fixed haftmann bug
Thu, 20 Sep 2007 16:37:29 +0200 haftmann fixed wrong syntax treatment in class target
Wed, 19 Sep 2007 17:16:40 +0200 nipkow tuned
Wed, 19 Sep 2007 13:59:13 +0200 paulson metis too slow
Wed, 19 Sep 2007 13:14:00 +0200 nipkow Generalized [_.._] from nat to linear orders
Tue, 18 Sep 2007 18:52:17 +0200 ballarin Simplified proofs due to transitivity reasoner setup.
Tue, 18 Sep 2007 17:53:37 +0200 paulson metis now available in PreList
less more (0) -120 tip