Nominal/Parser.thy
Fri, 14 May 2010 18:12:07 +0100 Christian Urban started a new file for the parser to make some experiments
Mon, 03 May 2010 11:43:27 +0200 Cezary Kaliszyk remove tracing
Mon, 03 May 2010 11:35:38 +0200 Cezary Kaliszyk Fix Parser
Mon, 03 May 2010 00:01:12 +0100 Christian Urban moved old parser and old fv back into their original places; isabelle make works again
Fri, 30 Apr 2010 15:45:39 +0200 Cezary Kaliszyk NewParser with Parser functionality, but some cheats included since the order of datayupes is wrong.
Fri, 30 Apr 2010 14:48:13 +0200 Cezary Kaliszyk Merged nominal_datatype into NewParser until eqvts
Fri, 30 Apr 2010 13:57:59 +0200 Cezary Kaliszyk more parser/new parser synchronization.
Fri, 30 Apr 2010 10:48:48 +0200 Cezary Kaliszyk Simplify old parser for integration
Sun, 25 Apr 2010 08:18:06 +0200 Christian Urban tuned and made to compile
Sat, 24 Apr 2010 09:49:23 +0200 Christian Urban merged
Wed, 21 Apr 2010 10:09:07 +0200 Christian Urban merged
Tue, 20 Apr 2010 18:24:50 +0200 Christian Urban renamed Ex1.thy to SingleLet.thy
Tue, 20 Apr 2010 10:23:39 +0200 Cezary Kaliszyk Fix of comment
Mon, 19 Apr 2010 10:00:52 +0200 Cezary Kaliszyk merge
Mon, 19 Apr 2010 09:59:32 +0200 Cezary Kaliszyk Locations of files in Parser
Wed, 14 Apr 2010 10:39:03 +0200 Cezary Kaliszyk Initial cleaning/reorganization in Fv.
Sun, 11 Apr 2010 18:11:23 +0200 Christian Urban tuned
Sun, 04 Apr 2010 21:39:28 +0200 Christian Urban separated general nominal theory into separate folder
Thu, 01 Apr 2010 08:48:33 +0200 Cezary Kaliszyk Let with multiple bindings.
Sat, 27 Mar 2010 16:20:39 +0100 Cezary Kaliszyk Lets finally abstract lists.
Sat, 27 Mar 2010 14:55:07 +0100 Cezary Kaliszyk Automatically lift theorems and constants only using the new quotient types. Requires new Isabelle.
Sat, 27 Mar 2010 13:50:59 +0100 Cezary Kaliszyk Get lifted types information from the quotient package.
Sat, 27 Mar 2010 12:01:28 +0100 Cezary Kaliszyk Parsing of list-bn functions into components.
Sat, 27 Mar 2010 08:42:07 +0100 Cezary Kaliszyk New compose lemmas. Reverted alpha_gen sym/trans changes. Equivp for alpha_res should work now.
Sat, 27 Mar 2010 08:11:11 +0100 Cezary Kaliszyk Fv/Alpha now takes into account Alpha_Type given from the parser.
Fri, 26 Mar 2010 17:22:02 +0100 Cezary Kaliszyk Describe 'nominal_datatype2'.
Fri, 26 Mar 2010 16:20:39 +0100 Cezary Kaliszyk Removed remaining cheats + some cleaning.
Fri, 26 Mar 2010 10:07:26 +0100 Cezary Kaliszyk Removed another cheat and cleaned the code a bit.
Thu, 25 Mar 2010 20:12:57 +0100 Cezary Kaliszyk Proper bn_rsp, for bn functions calling each other.
Thu, 25 Mar 2010 17:30:46 +0100 Cezary Kaliszyk Gathering things to prove by induction together; removed cheat_bn_eqvt.
Wed, 24 Mar 2010 10:49:50 +0100 Cezary Kaliszyk Export all the cheats needed for Core Haskell.
Tue, 23 Mar 2010 16:28:29 +0100 Cezary Kaliszyk Parsing bn functions that call other bn functions and transmitting this information to fv/alpha.
Tue, 23 Mar 2010 08:33:48 +0100 Cezary Kaliszyk Move examples which create more permutations out
Mon, 22 Mar 2010 18:29:29 +0100 Cezary Kaliszyk equivp_cheat can be removed for all one-permutation examples.
Mon, 22 Mar 2010 17:21:27 +0100 Cezary Kaliszyk Got rid of alpha_bn_rsp_cheat.
Mon, 22 Mar 2010 14:07:07 +0100 Cezary Kaliszyk fv_rsp proved automatically.
Sat, 20 Mar 2010 09:27:28 +0100 Cezary Kaliszyk Use 'alpha_bn_refl' to get rid of one of the sorrys.
Sat, 20 Mar 2010 08:04:59 +0100 Cezary Kaliszyk Prove reflp for all relations.
Fri, 19 Mar 2010 18:42:57 +0100 Cezary Kaliszyk Automatically derive support for datatypes with at-most one binding per constructor.
Fri, 19 Mar 2010 14:54:30 +0100 Cezary Kaliszyk Use fs typeclass in showing finite support + some cheat cleaning.
Fri, 19 Mar 2010 10:24:16 +0100 Cezary Kaliszyk Remove atom_decl from the parser.
Thu, 18 Mar 2010 23:19:55 +0100 Cezary Kaliszyk Reached strong_induction in fset-based TySch. Will not work until isabelle changes are pushed.
Thu, 18 Mar 2010 15:13:20 +0100 Cezary Kaliszyk Rename "_property" to ".property"
Thu, 18 Mar 2010 14:05:49 +0100 Cezary Kaliszyk case names also for _induct
Thu, 18 Mar 2010 12:32:03 +0100 Cezary Kaliszyk Case_Names for _inducts. Does not work for _induct yet.
Thu, 18 Mar 2010 12:09:59 +0100 Cezary Kaliszyk Added fv,bn,distinct,perm to the simplifier.
Thu, 18 Mar 2010 08:03:42 +0100 Cezary Kaliszyk Move most of the exporting out of the parser.
Thu, 18 Mar 2010 07:43:44 +0100 Cezary Kaliszyk Prove pseudo-inject (eq-iff) on the exported level and rename appropriately.
Thu, 18 Mar 2010 07:35:44 +0100 Cezary Kaliszyk Prove eqvts on exported terms.
Thu, 18 Mar 2010 07:26:36 +0100 Cezary Kaliszyk Clean 'Lift', start working only on exported things in Parser.
Wed, 17 Mar 2010 17:11:23 +0100 Christian Urban merged
Wed, 17 Mar 2010 15:13:31 +0100 Christian Urban made paper to compile
Wed, 17 Mar 2010 12:18:35 +0100 Cezary Kaliszyk cheat_alpha_eqvt no longer needed. Cleaned the tracing messages.
Wed, 17 Mar 2010 08:39:46 +0100 Cezary Kaliszyk Lifting theorems with compound fv and compound alpha.
Tue, 16 Mar 2010 20:07:13 +0100 Cezary Kaliszyk Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
Tue, 16 Mar 2010 15:27:47 +0100 Cezary Kaliszyk FV_bn generated for recursive functions as well, and used in main fv for bindings.
Mon, 15 Mar 2010 17:42:17 +0100 Cezary Kaliszyk fv_eqvt_cheat no longer needed.
Mon, 15 Mar 2010 14:32:05 +0100 Cezary Kaliszyk derive "inducts" from "induct" instead of lifting again is much faster.
Mon, 15 Mar 2010 11:50:12 +0100 Cezary Kaliszyk cheat_alpha_eqvt no longer needed; the proofs work.
Mon, 15 Mar 2010 10:07:15 +0100 Cezary Kaliszyk explicit flag "cheat_equivp"
Sat, 13 Mar 2010 13:49:15 +0100 Christian Urban started supp-fv proofs (is going to work)
Fri, 12 Mar 2010 12:42:35 +0100 Cezary Kaliszyk Still don't know how to prove supp=fv for simplest Let...
Thu, 11 Mar 2010 20:49:31 +0100 Cezary Kaliszyk Do not fail if the finite support proof fails.
Thu, 11 Mar 2010 19:41:11 +0100 Christian Urban support of atoms at the end of Abs.thy
Thu, 11 Mar 2010 17:47:29 +0100 Cezary Kaliszyk Show that the new types are in finite support typeclass.
Thu, 11 Mar 2010 15:11:57 +0100 Cezary Kaliszyk Remove "_raw" from lifted theorems.
Thu, 11 Mar 2010 14:05:36 +0100 Cezary Kaliszyk The cheats described explicitely.
Thu, 11 Mar 2010 13:34:45 +0100 Cezary Kaliszyk With the 4 cheats, all examples fully lift.
Thu, 11 Mar 2010 12:30:53 +0100 Cezary Kaliszyk Lift alpha_bn_constants.
Thu, 11 Mar 2010 12:26:24 +0100 Cezary Kaliszyk Lifting constants.
Thu, 11 Mar 2010 11:32:37 +0100 Cezary Kaliszyk Lifting constants works for all examples.
Thu, 11 Mar 2010 11:25:18 +0100 Cezary Kaliszyk Equivp working only on the standard alpha-equivalences.
Thu, 11 Mar 2010 11:20:50 +0100 Cezary Kaliszyk explicit cheat_fv_eqvt
Thu, 11 Mar 2010 11:15:14 +0100 Cezary Kaliszyk extract build_eqvts_tac.
Thu, 11 Mar 2010 10:39:29 +0100 Cezary Kaliszyk build_eqvts no longer requires permutations.
Thu, 11 Mar 2010 10:22:24 +0100 Cezary Kaliszyk Add explicit alpha_eqvt_cheat.
Thu, 11 Mar 2010 10:10:23 +0100 Cezary Kaliszyk Export tactic out of alpha_eqvt.
Wed, 10 Mar 2010 16:51:15 +0100 Christian Urban merged
Wed, 10 Mar 2010 16:50:42 +0100 Christian Urban almost done with showing the equivalence between old and new alpha-equivalence (one subgoal remaining)
Wed, 10 Mar 2010 15:34:13 +0100 Cezary Kaliszyk Undoing mistakenly committed parser experiments.
Wed, 10 Mar 2010 15:32:51 +0100 Cezary Kaliszyk alpha_eqvt for recursive term1.
Wed, 10 Mar 2010 13:10:00 +0100 Cezary Kaliszyk Linked parser to fv and alpha.
Wed, 10 Mar 2010 12:48:38 +0100 Christian Urban parser produces ordered bn-fun information
Tue, 09 Mar 2010 22:08:38 +0100 Christian Urban added bn-information, but it is not yet ordered according to the dts
Tue, 09 Mar 2010 16:24:39 +0100 Cezary Kaliszyk A version of Fv that takes into account recursive and non-recursive bindings.
Mon, 08 Mar 2010 15:01:26 +0100 Christian Urban merged
Mon, 08 Mar 2010 15:01:01 +0100 Christian Urban updated to new Isabelle
Mon, 08 Mar 2010 11:12:15 +0100 Cezary Kaliszyk More fine-grained nominal restriction for debugging.
Fri, 05 Mar 2010 14:55:21 +0100 Cezary Kaliszyk Lift fv and bn eqvts; no need to lift alpha_eqvt.
Thu, 04 Mar 2010 18:57:23 +0100 Cezary Kaliszyk Lift distinct.
Thu, 04 Mar 2010 15:55:53 +0100 Cezary Kaliszyk Added lifting of pseudo-injectivity, commented out the code again and enabled the weird examples.
Thu, 04 Mar 2010 15:15:44 +0100 Cezary Kaliszyk Lift BV,FV,Permutations and injection :).
Thu, 04 Mar 2010 12:00:11 +0100 Cezary Kaliszyk Comment out Weird and Phd until we have an idea how to handle multiple permutations. Transp that works for multiple existentials.
Wed, 03 Mar 2010 14:22:58 +0100 Cezary Kaliszyk Fix eqvt for multiple quantifiers.
Wed, 03 Mar 2010 11:42:15 +0100 Cezary Kaliszyk weird eqvt
Tue, 02 Mar 2010 21:43:27 +0100 Cezary Kaliszyk Comment out the part that does not work with 2 quantifiers.
Tue, 02 Mar 2010 17:48:41 +0100 Cezary Kaliszyk Porting from Lift to Parser; until defining the Quotient type.
Tue, 02 Mar 2010 15:11:41 +0100 Cezary Kaliszyk Working bv_eqvt
Tue, 02 Mar 2010 08:42:10 +0100 Cezary Kaliszyk Link calls to Raw permutations, FV definition and alpha_definition into the parser.
Tue, 02 Mar 2010 06:42:43 +0100 Christian Urban rawified the bind specs (ready to be used now)
Mon, 01 Mar 2010 19:23:08 +0100 Christian Urban modified for new binding format - hope it is the intended one
Mon, 01 Mar 2010 16:55:41 +0100 Christian Urban further code-refactoring in the parser
Mon, 01 Mar 2010 14:26:14 +0100 Christian Urban slight simplification of the raw-decl generation
Mon, 01 Mar 2010 07:46:50 +0100 Christian Urban added example from my phd
Sat, 27 Feb 2010 11:54:59 +0100 Christian Urban streamlined parser
Fri, 26 Feb 2010 18:38:25 +0100 Christian Urban generated the "binding list" from the input; at the moment it is only printed out as tracing; does not yet include the "bind itself binders"
Thu, 25 Feb 2010 11:51:34 +0100 Christian Urban a few simplifications
Thu, 25 Feb 2010 08:40:52 +0100 Christian Urban added IsaMakefile...but so far included only a test for the parser
less more (0) tip