Nominal/Nominal2.thy
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
Fri, 31 Dec 2010 13:31:39 +0000 Christian Urban added proper case names for all induct and exhaust theorems
Thu, 30 Dec 2010 10:00:09 +0000 Christian Urban removed local fix for bug in induction_schema; added setup method for strong inductions
Tue, 28 Dec 2010 19:51:25 +0000 Christian Urban automated all strong induction lemmas
Tue, 28 Dec 2010 00:20:50 +0000 Christian Urban proper application of induction_schema and strong_exhaust rules; needs local fix in induction_schema.ML
Sun, 26 Dec 2010 16:35:16 +0000 Christian Urban generated goals for strong induction theorems.
Thu, 23 Dec 2010 00:46:06 +0000 Christian Urban moved all strong_exhaust code to nominal_dt_quot; tuned examples
Thu, 23 Dec 2010 00:22:41 +0000 Christian Urban moved generic functions into nominal_library
Wed, 22 Dec 2010 23:12:51 +0000 Christian Urban slight tuning
Wed, 22 Dec 2010 22:30:43 +0000 Christian Urban slight tuning
Wed, 22 Dec 2010 21:13:32 +0000 Christian Urban added fold_right which produces the correct term for left-infix operators
Wed, 22 Dec 2010 12:17:49 +0000 Christian Urban a bit tuning
Wed, 22 Dec 2010 10:32:01 +0000 Christian Urban corrected premises of strong exhausts theorems
Wed, 22 Dec 2010 09:13:25 +0000 Christian Urban properly exported strong exhaust theorem; cleaned up some examples
Tue, 21 Dec 2010 10:28:08 +0000 Christian Urban all examples for strong exhausts work; recursive binders need to be treated differently; still unclean version with lots of diagnostic code
Fri, 17 Dec 2010 01:01:44 +0000 Christian Urban tuned
Fri, 17 Dec 2010 00:39:27 +0000 Christian Urban tuned
Thu, 16 Dec 2010 08:42:48 +0000 Christian Urban simple cases for strong inducts done; infrastructure for the difficult ones is there
Tue, 14 Dec 2010 14:23:40 +0000 Christian Urban freshness theorem in strong exhausts; (temporarily includes a cheat_tac to make all tests go through)
Sun, 12 Dec 2010 22:09:11 +0000 Christian Urban created strong_exhausts terms
Sun, 12 Dec 2010 00:10:40 +0000 Christian Urban moved setify and listify functions into the library; introduced versions that have a type argument
Wed, 08 Dec 2010 17:07:08 +0000 Christian Urban first tests about exhaust
Wed, 08 Dec 2010 13:16:25 +0000 Christian Urban moved some code into the nominal_library
Wed, 08 Dec 2010 13:05:04 +0000 Christian Urban moved definition of raw bn-functions into nominal_dt_rawfuns
less more (0) -60 tip