Nominal/Nominal2.thy
Mon, 19 May 2014 12:45:26 +0100 Christian Urban changed nominal_primrec into the more appropriate nominal_function
Mon, 19 May 2014 11:19:48 +0100 Christian Urban changes from upstream
Fri, 16 May 2014 08:38:23 +0100 Christian Urban updated changes from upstream (AFP)
Mon, 24 Mar 2014 15:31:17 +0000 Christian Urban updated to massive changes in Isabelle
Thu, 13 Mar 2014 09:21:31 +0000 Christian Urban updated to Isabelle changes
Mon, 13 Jan 2014 15:42:10 +0000 Christian Urban fixed bug with support and freshness lemmas not being simplified properly
Sat, 11 Jan 2014 23:17:23 +0000 Christian Urban updated with current AFP version
Sun, 15 Dec 2013 15:14:40 +1100 Christian Urban updated to changes in Isabelle
Fri, 19 Apr 2013 00:10:52 +0100 Christian Urban updated to simplifier changes
Wed, 27 Mar 2013 16:08:30 +0100 webertj Various changes to support Nominal2 commands in local contexts.
Thu, 04 Oct 2012 12:44:43 +0100 Christian Urban removed "use" - replaced by "ML_file"
Mon, 18 Jun 2012 14:50:02 +0100 Christian Urban used ML-antiquotation command_spec for new commands
Thu, 31 May 2012 12:01:01 +0100 Christian Urban added to the simplifier nominal_datatype.fresh lemmas
Fri, 20 Apr 2012 18:58:03 +0200 Cezary Kaliszyk Find remaining rsp theorems and provide them with the quotient definitions
Fri, 20 Apr 2012 15:58:13 +0200 Cezary Kaliszyk Declare rsp for permute, permute_bn, alpha_bn together with their definitions instead of TrueI
Fri, 20 Apr 2012 15:28:35 +0200 Cezary Kaliszyk Pass proper rsp theorems for constructors and for size
Tue, 10 Apr 2012 15:22:16 +0100 Christian Urban updated to latest changes (10 April) to quotient package (lift_raw_const only takes dummy theorem TrueI....in the future this will not work anymore)
Tue, 20 Mar 2012 11:26:10 +0000 Christian Urban updated to new Isabelle (20 March)
Sat, 17 Mar 2012 05:13:59 +0000 Christian Urban updated to new Isabelle (declared keywords)
Thu, 22 Dec 2011 13:10:30 +0000 Christian Urban the default sort for type-variables in nominal specifications is fs; it is automatically addded
Sun, 18 Dec 2011 00:42:32 +0000 Christian Urban partially localised the parsing process using functions fron Datatype
Sat, 17 Dec 2011 16:36:51 +0000 Christian Urban Started Nominal2-Isabelle2011-1 branch and backported changeset 32abaea424bd Nominal2-Isabelle2011-1
Thu, 15 Dec 2011 16:20:42 +0000 Christian Urban updated to lates changes in the datatype package
Wed, 14 Dec 2011 01:32:42 +0000 Christian Urban generated the correct thm-list for showing that qfv are equal to support
Tue, 13 Dec 2011 09:39:56 +0000 Christian Urban updated to Isabelle 13 Dec
Tue, 06 Dec 2011 23:42:19 +0000 Christian Urban updated to Isabelle 6 Dec (thanks to Odrej Kuncar)
Thu, 03 Nov 2011 13:19:23 +0000 Christian Urban updated to Isabelle 3 Nov; it includes a hack to work around a bug in the localised version of the quotient package
Mon, 18 Jul 2011 17:40:13 +0100 Christian Urban added a flag (eqvt) to termination proofs arising fron nominal_primrecs
Wed, 13 Jul 2011 09:47:58 +0100 Christian Urban slight tuning
Mon, 11 Jul 2011 14:02:13 +0200 Christian Urban combinators for local theories and lists
Fri, 08 Jul 2011 05:04:23 +0200 Christian Urban some code refactoring
Thu, 07 Jul 2011 16:16:42 +0200 Christian Urban code refactoring; introduced a record for raw_dt_info
Tue, 05 Jul 2011 18:42:34 +0200 Christian Urban changed bind to binds in specifications; bind will cause trouble with Monad_Syntax
Tue, 05 Jul 2011 04:18:45 +0200 Christian Urban exported various FCB-lemmas to a separate file
Thu, 30 Jun 2011 02:19:59 +0100 Christian Urban more code refactoring
Wed, 29 Jun 2011 23:08:44 +0100 Christian Urban combined distributed data for alpha in alpha_result (partially done)
Wed, 29 Jun 2011 00:48:50 +0100 Christian Urban some experiments
Thu, 23 Jun 2011 11:30:39 +0100 Christian Urban fixed nasty bug with type variables in nominal_datatypes; this included to be careful with the output of the inductive and function package
Wed, 22 Jun 2011 14:14:54 +0100 Christian Urban tuned
Wed, 22 Jun 2011 13:40:25 +0100 Christian Urban deleted some dead code
Wed, 22 Jun 2011 12:18:22 +0100 Christian Urban some rudimentary infrastructure for storing data about nominal datatypes
Thu, 16 Jun 2011 20:07:03 +0100 Christian Urban got rid of the boolean flag in the raw_equivariance function
Wed, 15 Jun 2011 22:36:59 +0100 Christian Urban added size-lemmas to simplifier; as a result termination can be proved by the standard lexicographic_order method
Tue, 07 Jun 2011 10:40:06 +0100 Christian Urban cleaned ups a bit the examples with the invariant framework; exported nominal_function_config datatype into separate structure and file
Tue, 07 Jun 2011 08:52:59 +0100 Christian Urban fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Sun, 05 Jun 2011 21:14:23 +0100 Christian Urban added an option for an invariant (at the moment only a stub)
Wed, 25 May 2011 21:38:50 +0200 Christian Urban added eq_iff and distinct lemmas of nominal datatypes to the simplifier
Tue, 10 May 2011 07:47:06 +0100 Christian Urban updated to new Isabelle (> 9 May)
Tue, 19 Apr 2011 13:03:08 +0100 Christian Urban updated to snapshot Isabelle 19 April
Mon, 18 Apr 2011 15:56:07 +0100 Christian Urban added permute_pure back into the nominal_inductive procedure; updated to Isabelle 17 April
Mon, 28 Feb 2011 15:21:10 +0000 Christian Urban split the library into a basics file; merged Nominal_Eqvt into Nominal_Base
Wed, 19 Jan 2011 17:11:10 +0100 Christian Urban added Minimal file to test things
Mon, 17 Jan 2011 14:37:18 +0100 Christian Urban exported nominal function code to external file
Fri, 07 Jan 2011 02:30:00 +0000 Christian Urban derived equivariance for the function graph and function relation
Thu, 06 Jan 2011 23:06:45 +0000 Christian Urban a modified function package where, as a test, True has been injected into the compatibility condictions
Thu, 06 Jan 2011 19:57:57 +0000 Christian Urban removed debugging code abd introduced a guarded tracing function
Thu, 06 Jan 2011 13:28:40 +0000 Christian Urban cleaned up weakening proof and added a version with finit sets
Thu, 06 Jan 2011 11:00:16 +0000 Christian Urban made sure the raw datatypes and raw functions do not get any mixfix syntax
Wed, 05 Jan 2011 17:33:43 +0000 Christian Urban exported the code into a separate file
Fri, 31 Dec 2010 15:37:04 +0000 Christian Urban changed res keyword to set+ for restrictions; comment by a referee
less more (0) -100 -60 tip