src/HOL/Library/Efficient_Nat.thy
Mon, 23 Jul 2012 09:28:03 +0200 haftmann restrict unqualified imports from Haskell Prelude to a small set of fundamental operations
Tue, 05 Jun 2012 07:10:51 +0200 haftmann prefer sys.error over plain error in Scala to avoid deprecation warning
Sun, 25 Mar 2012 20:15:39 +0200 huffman merged fork with new numeral representation (see NEWS)
Wed, 15 Feb 2012 23:19:30 +0100 wenzelm renamed Thm.capply to Thm.apply, and Thm.cabs to Thm.lambda in conformance with similar operations in structure Term and Logic;
Thu, 29 Dec 2011 10:47:55 +0100 haftmann attribute code_abbrev superseedes code_unfold_post
Fri, 09 Dec 2011 12:21:03 +0100 bulwahn deactivating quickcheck_narrowing if Efficient_Nat theory is loaded
Wed, 19 Oct 2011 09:11:15 +0200 bulwahn removing old code generator setup for efficient natural numbers; cleaned typo
Sat, 02 Jul 2011 22:14:47 +0200 haftmann tuned typo
Thu, 09 Jun 2011 16:34:49 +0200 wenzelm discontinued Name.variant to emphasize that this is old-style / indirect;
Thu, 18 Nov 2010 17:01:16 +0100 haftmann map_pair replaces prod_fun
Wed, 29 Sep 2010 10:05:44 +0200 haftmann scala is reserved identifier
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
Wed, 01 Sep 2010 11:09:50 +0200 haftmann do not print object frame around Scala includes -- this is in the responsibility of the user
Fri, 27 Aug 2010 19:34:23 +0200 haftmann renamed class/constant eq to equal; tuned some instantiations
Thu, 26 Aug 2010 12:19:50 +0200 haftmann tuned includes
Thu, 26 Aug 2010 10:16:22 +0200 haftmann code_include Scala: qualify module nmae
Mon, 26 Jul 2010 11:10:36 +0200 haftmann corrected range check once more
Sat, 24 Jul 2010 18:08:41 +0200 haftmann another refinement chapter in the neverending numeral story
Fri, 23 Jul 2010 10:58:13 +0200 haftmann avoid unreliable Haskell Int type
Tue, 20 Jul 2010 08:54:21 +0200 haftmann avoid deprecation
Mon, 19 Jul 2010 11:55:42 +0200 haftmann dropped superfluous prefixes
Fri, 16 Jul 2010 15:28:23 +0200 haftmann corrected range chec
Tue, 08 Jun 2010 16:37:22 +0200 haftmann tuned quotes, antiquotations and whitespace
Tue, 01 Jun 2010 10:30:53 +0200 haftmann corrected implementation
Fri, 21 May 2010 11:50:34 +0200 haftmann nats in Haskell are readable
Fri, 30 Apr 2010 23:53:37 +0200 wenzelm renamed Variable.thm_context to Variable.global_thm_context to emphasize that this is not the real thing;
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;
Wed, 10 Mar 2010 15:29:22 +0100 haftmann fixed typo
Sun, 07 Mar 2010 12:19:47 +0100 wenzelm modernized structure Object_Logic;
Fri, 22 Jan 2010 13:38:28 +0100 haftmann code literals: distinguish numeral classes by different entries
Thu, 14 Jan 2010 17:54:54 +0100 haftmann dedicated conversions to and from Int
Thu, 14 Jan 2010 17:47:39 +0100 haftmann added Scala setup
Wed, 13 Jan 2010 10:18:45 +0100 haftmann function transformer preprocessor applies to both code generators
Fri, 30 Oct 2009 18:32:40 +0100 haftmann tuned code setup
Thu, 29 Oct 2009 22:16:40 +0100 haftmann adjusted to changes in theory Divides
Wed, 23 Sep 2009 14:00:12 +0200 haftmann Code_Eval(uation)
Fri, 31 Jul 2009 10:49:08 +0200 haftmann repair mess produced by resolution afterwards
Wed, 15 Jul 2009 10:11:13 +0200 haftmann additional preprocessor rule
Tue, 14 Jul 2009 16:27:32 +0200 haftmann prefer code_inline over code_unfold; use code_unfold_post where appropriate
Tue, 14 Jul 2009 10:54:04 +0200 haftmann code attributes use common underscore convention
Tue, 07 Jul 2009 17:37:00 +0200 haftmann Stefan Berghofer's code generator uses Pure equality instead of HOL equality now
Tue, 02 Jun 2009 15:53:05 +0200 haftmann OCaml builtin intergers are elusive; avoid
Sat, 30 May 2009 08:16:44 +0200 haftmann corrected bound/unbounded flag for nat numerals
Tue, 19 May 2009 16:54:55 +0200 haftmann String.literal replaces message_string, code_numeral replaces (code_)index
Tue, 19 May 2009 13:57:32 +0200 haftmann moved Code_Index, Random and Quickcheck before Main
Tue, 12 May 2009 21:17:38 +0200 haftmann adapted to changes in module Code
Mon, 11 May 2009 10:53:19 +0200 haftmann clarified matter of "proper" flag in code equations
Mon, 23 Mar 2009 08:14:24 +0100 haftmann Main is (Complex_Main) base entry point in library theories
Mon, 16 Feb 2009 19:11:16 +0100 haftmann faster preprocessor
Mon, 16 Feb 2009 13:38:09 +0100 haftmann dropped clause_suc_preproc for generic code generator
Fri, 06 Feb 2009 09:05:19 +0100 haftmann mandatory prefix for index conversion operations
Tue, 03 Feb 2009 19:37:00 +0100 haftmann changed name space policy for Haskell includes
Wed, 28 Jan 2009 13:36:11 +0100 haftmann slightly adapted towards more uniformity with div/mod on nat
Thu, 01 Jan 2009 14:23:39 +0100 wenzelm eliminated OldTerm.(add_)term_consts;
Wed, 31 Dec 2008 18:53:16 +0100 wenzelm moved old add_type_XXX, add_term_XXX etc. to structure OldTerm;
Tue, 30 Dec 2008 21:46:48 +0100 wenzelm canonical Term.add_var_names;
Thu, 04 Dec 2008 08:47:45 -0800 huffman change more lemmas to avoid using iszero
Mon, 27 Oct 2008 16:15:49 +0100 haftmann slightly tuned
less more (0) -60 tip