Nominal/Ex/Lambda.thy
Sat, 19 Mar 2016 21:06:48 +0000 Christian Urban updated to Isabelle 2016 Nominal2-Isabelle2016
Mon, 20 Jul 2015 11:21:59 +0100 Christian Urban removed junk
Thu, 09 Jul 2015 02:32:46 +0100 Christian Urban updated for Isabelle 2015
Mon, 19 May 2014 16:45:46 +0100 Christian Urban changed nominal_primrec to nominal_function and termination to nominal_termination
Mon, 19 May 2014 12:45:26 +0100 Christian Urban changed nominal_primrec into the more appropriate nominal_function
Sun, 06 Apr 2014 13:07:24 +0100 Christian Urban some small additions to examples
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
Tue, 04 Jun 2013 09:39:23 +0100 Christian Urban updated to new Isabelle
Tue, 19 Feb 2013 06:58:14 +0000 Christian Urban updated for 2013 release Nominal2-Isabelle2013
Tue, 07 Aug 2012 18:54:52 +0100 Christian Urban definition of an auxiliary graph in nominal-primrec definitions
Sun, 15 Jul 2012 13:03:47 +0100 Christian Urban added a simproc for alpha-equivalence to the simplifier
Thu, 12 Jul 2012 10:11:32 +0100 Christian Urban streamlined definition of alpha-equivalence for single binders (used flip instead of swap)
Mon, 04 Jun 2012 21:39:51 +0100 Christian Urban added permutation simplification to the simplifier; this makes the simplifier more powerful, but it potentially loops more often
Thu, 31 May 2012 12:01:01 +0100 Christian Urban added to the simplifier nominal_datatype.fresh lemmas
Wed, 23 May 2012 23:57:27 +0100 Christian Urban improved handling in the simplifier for inequalities derived from freshness assumptions
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)
Sat, 17 Mar 2012 05:13:59 +0000 Christian Urban updated to new Isabelle (declared keywords)
Wed, 21 Dec 2011 13:06:09 +0900 Cezary Kaliszyk Port CR_Takahashi from Nominal1, no more "sorry" in BetaCR.
Sat, 17 Dec 2011 17:08:47 +0000 Christian Urban cleaned examples for stable branch Nominal2-Isabelle2011-1
Thu, 15 Dec 2011 16:20:42 +0000 Christian Urban updated to lates changes in the datatype package
Tue, 08 Nov 2011 22:31:31 +0000 Cezary Kaliszyk Add equivariance for alpha_lam_raw and abs_lam.
Mon, 07 Nov 2011 13:58:18 +0000 Christian Urban all examples work again after quotient package has been "de-localised"
Fri, 19 Aug 2011 11:01:52 +0900 Cezary Kaliszyk Comment out examples with 'True' that do not work because function still does not work
Fri, 22 Jul 2011 11:37:16 +0100 Christian Urban completed the eqvt-proofs for functions; they are stored under the name function_name.eqvt and added to the eqvt-list
Tue, 19 Jul 2011 02:30:05 +0100 Christian Urban preliminary version of automatically generation the eqvt-lemmas for functions defined with nominal_primrec
Tue, 19 Jul 2011 01:40:36 +0100 Christian Urban generated the partial eqvt-theorem for functions
Mon, 18 Jul 2011 17:40:13 +0100 Christian Urban added a flag (eqvt) to termination proofs arising fron nominal_primrecs
Mon, 18 Jul 2011 10:50:21 +0100 Christian Urban moved eqvt for Option.map
Tue, 05 Jul 2011 23:47:20 +0200 Christian Urban added some relatively simple examples from paper by Norrish
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 16:22:18 +0200 Christian Urban made the tests go through again
Tue, 05 Jul 2011 04:23:33 +0200 Christian Urban merged
Tue, 05 Jul 2011 04:18:45 +0200 Christian Urban exported various FCB-lemmas to a separate file
Tue, 05 Jul 2011 10:13:34 +0900 Cezary Kaliszyk Express trans_db with Option.map and Option.bind. Possibly mbind is a copy of bind?
Tue, 05 Jul 2011 09:28:16 +0900 Cezary Kaliszyk Define a version of aux only for same binders. Completeness is fine.
Tue, 05 Jul 2011 09:26:20 +0900 Cezary Kaliszyk Move If / Let with 'True' to the end of Lambda
Mon, 04 Jul 2011 23:54:05 +0200 Christian Urban added an example that recurses over two arguments; the interesting proof-obligation is not yet done
Tue, 28 Jun 2011 00:30:30 +0100 Christian Urban copied all work to Lambda.thy; had to derive a special version of fcb1 for concrete atom
Sun, 26 Jun 2011 17:55:22 +0100 Christian Urban another change to the fcb2; this is needed in order to get all proofs through in Lambda.thy
Thu, 23 Jun 2011 22:21:43 +0100 Christian Urban the simplifier can simplify "sort (atom a)" if a is a concrete atom type declared with atom_decl
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
Thu, 16 Jun 2011 12:12:25 +0100 Christian Urban added a test that every function must be of pt-sort
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
Wed, 15 Jun 2011 09:50:53 +0900 Cezary Kaliszyk Some TODOs
Fri, 10 Jun 2011 15:52:17 +0900 Cezary Kaliszyk Move working examples before non-working ones
Fri, 10 Jun 2011 15:45:49 +0900 Cezary Kaliszyk Optimized proofs and removed some garbage.
Fri, 10 Jun 2011 15:30:09 +0900 Cezary Kaliszyk Slightly modify fcb for list1 and put in common place.
Thu, 09 Jun 2011 15:34:51 +0900 Cezary Kaliszyk Eval can be defined with additional freshness
Thu, 09 Jun 2011 15:03:58 +0900 Cezary Kaliszyk Minor simplification
Wed, 08 Jun 2011 12:30:56 +0100 Christian Urban merged
Wed, 08 Jun 2011 12:30:46 +0100 Christian Urban merged
Wed, 08 Jun 2011 07:06:20 +0900 Cezary Kaliszyk Simplify ln-trans proof
Wed, 08 Jun 2011 07:02:52 +0900 Cezary Kaliszyk cbvs can be easily defined without an invariant
Tue, 07 Jun 2011 20:58:00 +0100 Christian Urban defined the "count-bound-variables-occurences" function which has an accumulator like trans
Tue, 07 Jun 2011 17:45:38 +0100 Christian Urban merged
Tue, 07 Jun 2011 23:42:12 +0900 Cezary Kaliszyk remove garbage (proofs that assumes the invariant outside function)
Tue, 07 Jun 2011 23:38:39 +0900 Cezary Kaliszyk Proof of trans with invariant
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
less more (0) -100 -60 tip