src/HOL/Record.thy
Tue, 08 May 2012 14:31:03 +0200 bulwahn specialised fact in the Record theory should not be appear in proofs discovered by sledgehammer
Thu, 15 Mar 2012 22:08:53 +0100 wenzelm declare command keywords via theory header, including strict checking outside Pure;
Tue, 13 Sep 2011 17:25:19 -0700 huffman tuned proofs
Thu, 09 Jun 2011 08:32:16 +0200 bulwahn adding theory Quickcheck_Narrowing to HOL-Main image
Thu, 05 May 2011 10:47:31 +0200 bulwahn adding creation of exhaustive generators for records; simplifying dependencies in Main theory
Fri, 17 Dec 2010 17:43:54 +0100 wenzelm replaced command 'nonterminals' by slightly modernized version 'nonterminal';
Wed, 18 Aug 2010 16:59:35 +0200 haftmann removed separate quickcheck_record module
Tue, 17 Aug 2010 15:19:37 +0200 haftmann dropped make_/dest_ naming convention
Tue, 17 Aug 2010 15:13:16 +0200 haftmann eliminated typecopy interpretation
Thu, 12 Aug 2010 17:56:43 +0200 haftmann moved Record.thy from session Plain to Main; avoid variable name acc
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;
Tue, 16 Feb 2010 16:03:06 +0100 wenzelm simplified/clarified record translations;
Tue, 16 Feb 2010 14:08:39 +0100 wenzelm moved generic update_name to Pure syntax -- not specific to HOL/record;
Tue, 16 Feb 2010 13:35:42 +0100 wenzelm tuned;
Mon, 15 Feb 2010 19:16:45 +0100 wenzelm tuned document;
Mon, 21 Dec 2009 08:32:04 +0100 haftmann prefer prefix "iso" over potentially misleading "is"; tuned
Tue, 10 Nov 2009 16:11:43 +0100 haftmann substantial simplification restores code generation
Thu, 01 Oct 2009 01:03:36 +0200 wenzelm eliminated dead code, redundant bindings and parameters;
Tue, 29 Sep 2009 22:33:27 +0200 wenzelm replaced meta_iffD2 by existing Drule.equal_elim_rule2;
Tue, 29 Sep 2009 21:36:49 +0200 wenzelm tuned header;
Mon, 28 Sep 2009 14:16:01 +1000 Thomas Sewell Fix unescaped expressions breaking latex output in Record.thy
Wed, 23 Sep 2009 19:17:48 +1000 tsewell Initial response to feedback from Norbert, Makarius on record patch
Thu, 10 Sep 2009 16:38:18 +1000 Thomas Sewell Simplification of various aspects of the IsTuple component
Thu, 10 Sep 2009 15:18:43 +1000 Thomas Sewell Record patch imported and working.
Thu, 27 Aug 2009 00:40:53 +1000 tsewell Initial attempt at porting record update to repository Isabelle.
Fri, 19 Jun 2009 17:23:21 +0200 haftmann discontinued ancient tradition to suffix certain ML module names with "_package"
Wed, 19 Dec 2007 16:32:12 +0100 schirmer replaced K_record by lambda term %x. c
Thu, 26 Apr 2007 16:39:11 +0200 wenzelm added header;
Fri, 20 Apr 2007 17:58:25 +0200 haftmann reverted to classical syntax for K_record
Fri, 20 Apr 2007 11:21:42 +0200 haftmann Isar definitions are now added explicitly to code theorem table
Tue, 07 Nov 2006 18:25:48 +0100 schirmer field-update in records is generalised to take a function on the field
Fri, 21 Oct 2005 18:14:36 +0200 wenzelm avoid home-grown meta_allE;
Fri, 17 Jun 2005 16:12:49 +0200 haftmann migrated theory headers to new format
Mon, 30 May 2005 23:07:58 +0200 wenzelm tuned;
Wed, 18 Aug 2004 11:09:40 +0200 nipkow import -> imports
Mon, 16 Aug 2004 14:22:27 +0200 nipkow New theory header syntax.
Tue, 04 May 2004 11:24:02 +0200 schirmer tuned;
Mon, 03 May 2004 23:22:17 +0200 schirmer reimplementation of HOL records; only one type is created for
Sun, 29 Jun 2003 21:27:28 +0200 berghofe Added split_paired_All rule for splitting variables bound by
Wed, 24 Jul 2002 22:15:55 +0200 wenzelm simplified locale predicates;
Wed, 24 Jul 2002 00:10:52 +0200 wenzelm predicate defs via locales;
Sat, 27 Oct 2001 00:00:55 +0200 wenzelm removed "more" class;
Thu, 18 Oct 2001 21:22:40 +0200 wenzelm tuned;
Thu, 18 Oct 2001 21:01:18 +0200 wenzelm proper setup for abstract product types;
Wed, 17 Oct 2001 20:24:37 +0200 wenzelm abstract product types;
Wed, 08 Aug 2001 17:38:53 +0200 wenzelm _constify;
Tue, 07 Aug 2001 22:37:30 +0200 wenzelm fix problem with user translations by making field names appear as consts;
Mon, 11 Dec 2000 20:10:18 +0100 wenzelm added "_update_name" and parse_translation;
Wed, 25 Oct 2000 18:32:02 +0200 wenzelm more "xsymbols" syntax;
Mon, 23 Oct 2000 22:10:36 +0200 wenzelm intro_classes by default;
Wed, 27 Sep 2000 19:34:46 +0200 wenzelm more symbolic syntax (currently "input");
Tue, 29 Aug 2000 20:12:54 +0200 wenzelm \<dots> syntax;
Wed, 25 Aug 1999 20:49:02 +0200 wenzelm proper bootstrap of HOL theory and packages;
Thu, 22 Oct 1998 20:15:26 +0200 wenzelm tuned block indent;
Tue, 20 Oct 1998 16:35:37 +0200 wenzelm Datatype instead of Prod;
Tue, 28 Jul 1998 17:05:34 +0200 wenzelm removed global_names flag;
Fri, 24 Jul 1998 17:54:58 +0200 wenzelm added type and update syntax;
Fri, 12 Jun 1998 17:06:14 +0200 wenzelm changed {: :} syntax to (| |);
Wed, 29 Apr 1998 11:42:04 +0200 wenzelm Extensible records with structural subtyping in HOL. See
less more (0) tip