| Thu, 30 Jun 2011 11:05:25 +0100 | Christian Urban | clarified a sentence | changeset |
files | 
| Thu, 30 Jun 2011 02:19:59 +0100 | Christian Urban | more code refactoring | changeset |
files | 
| Wed, 29 Jun 2011 23:08:44 +0100 | Christian Urban | combined distributed data for alpha in alpha_result (partially done) | changeset |
files | 
| Wed, 29 Jun 2011 19:21:26 +0100 | Christian Urban | moved Classical and Let temporarily into a section where "sorry" is allowed; this makes all test go through | changeset |
files | 
| Wed, 29 Jun 2011 17:01:09 +0100 | Christian Urban | added a warning if a theorem is already declared as equivariant | changeset |
files | 
| Wed, 29 Jun 2011 16:44:54 +0100 | Christian Urban | merged | changeset |
files | 
| Wed, 29 Jun 2011 13:04:24 +0900 | Cezary Kaliszyk | Prove bn injectivity and experiment more with Let | changeset |
files | 
| Wed, 29 Jun 2011 00:48:50 +0100 | Christian Urban | some experiments | changeset |
files | 
| Tue, 28 Jun 2011 14:45:30 +0900 | Cezary Kaliszyk | trying new fcb in let/subst | changeset |
files | 
| Tue, 28 Jun 2011 14:30:30 +0900 | Cezary Kaliszyk | Leftover only inj and eqvt | changeset |
files | 
| Tue, 28 Jun 2011 14:18:26 +0900 | Cezary Kaliszyk | eapply fcb ok | changeset |
files | 
| Tue, 28 Jun 2011 14:01:15 +0900 | Cezary Kaliszyk | Removed Inl and Inr | changeset |
files | 
| Tue, 28 Jun 2011 14:49:48 +0100 | Christian Urban | relaxed type in fcb | changeset |
files | 
| Tue, 28 Jun 2011 14:34:07 +0100 | Christian Urban | fcb with explicit bn function | changeset |
files | 
| Tue, 28 Jun 2011 14:01:52 +0100 | Christian Urban | added let-rec example | changeset |
files | 
| Tue, 28 Jun 2011 12:36:34 +0900 | Cezary Kaliszyk | Experiments with res | changeset |
files | 
| Tue, 28 Jun 2011 00:48:57 +0100 | Christian Urban | proved the fcb also for sets (no restriction yet) | changeset |
files | 
| 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 | changeset |
files | 
| Mon, 27 Jun 2011 22:51:42 +0100 | Christian Urban | streamlined the fcb-proof and made fcb1 a special case of fcb | changeset |
files | 
| Mon, 27 Jun 2011 19:22:10 +0100 | Christian Urban | completed proof in Classical; the fcb lemma works for any list of atoms (despite what was written earlier) | changeset |
files | 
| Mon, 27 Jun 2011 19:15:18 +0100 | Christian Urban | fcb for multible (list) binders; at the moment all of them have to have the same sort (at-class); this should also work for set binders, but not yet for restriction. | changeset |
files | 
| Mon, 27 Jun 2011 19:13:55 +0100 | Christian Urban | renamed ds to dset (disagreement set) | changeset |
files | 
| Mon, 27 Jun 2011 12:15:21 +0100 | Christian Urban | added small lemma about disagreement set | changeset |
files | 
| Mon, 27 Jun 2011 08:42:02 +0900 | Cezary Kaliszyk | merge | changeset |
files | 
| Mon, 27 Jun 2011 08:38:54 +0900 | Cezary Kaliszyk | New-style fcb for multiple binders. | changeset |
files | 
| Mon, 27 Jun 2011 04:01:55 +0900 | Cezary Kaliszyk | equality of lst_binder and a few helper lemmas | changeset |
files | 
| Sun, 26 Jun 2011 21:42:07 +0100 | Christian Urban | only one of the fcb precondistions are needed (probably the same with the perm-conditions) | changeset |
files | 
| 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 | changeset |
files | 
| Sat, 25 Jun 2011 22:51:43 +0100 | Christian Urban | did all cases, except the multiple binder case | changeset |
files | 
| Sat, 25 Jun 2011 21:28:24 +0100 | Christian Urban | an alternative FCB for Abs_lst1; seems simpler but not as simple as I thought; not sure whether it generalises to multiple binders. | changeset |
files | 
| Fri, 24 Jun 2011 09:42:44 +0100 | Christian Urban | except for the interated binder case, finished definition in Calssical.thy | changeset |
files | 
| Fri, 24 Jun 2011 11:18:18 +0900 | Cezary Kaliszyk | Make examples work with non-precompiled image | changeset |
files | 
| Fri, 24 Jun 2011 11:15:22 +0900 | Cezary Kaliszyk | Remove Lambda_add.thy | changeset |
files | 
| Fri, 24 Jun 2011 11:14:58 +0900 | Cezary Kaliszyk | The examples in Lambda_add can be defined by nominal_function directly | changeset |
files | 
| Fri, 24 Jun 2011 11:03:53 +0900 | Cezary Kaliszyk | Theory name changes for JEdit | changeset |
files | 
| Fri, 24 Jun 2011 10:54:31 +0900 | Cezary Kaliszyk | More usual names for substitution properties | changeset |
files | 
| Fri, 24 Jun 2011 10:30:06 +0900 | Cezary Kaliszyk | Second Fixed Point Theorem | changeset |
files | 
| Fri, 24 Jun 2011 10:12:47 +0900 | Cezary Kaliszyk | Speed-up the completeness proof. | changeset |
files | 
| 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 | changeset |
files | 
| Thu, 23 Jun 2011 13:09:17 +0100 | Christian Urban | added file | changeset |
files | 
| Thu, 23 Jun 2011 12:28:25 +0100 | Christian Urban | expanded the example | changeset |
files | 
| 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 | changeset |
files | 
| Wed, 22 Jun 2011 14:14:54 +0100 | Christian Urban | tuned | changeset |
files | 
| Wed, 22 Jun 2011 13:40:25 +0100 | Christian Urban | deleted some dead code | changeset |
files | 
| Wed, 22 Jun 2011 12:18:22 +0100 | Christian Urban | some rudimentary infrastructure for storing data about nominal datatypes | changeset |
files | 
| Wed, 22 Jun 2011 17:57:15 +0900 | Cezary Kaliszyk | constants with the same names | changeset |
files | 
| Wed, 22 Jun 2011 04:49:56 +0900 | Cezary Kaliszyk | Quotients/TODO addtion | changeset |
files | 
| Tue, 21 Jun 2011 23:59:36 +0900 | Cezary Kaliszyk | Minor | changeset |
files | 
| Tue, 21 Jun 2011 10:39:25 +0900 | Cezary Kaliszyk | merge | changeset |
files | 
| Tue, 21 Jun 2011 10:37:43 +0900 | Cezary Kaliszyk | spelling | changeset |
files | 
| Mon, 20 Jun 2011 20:09:51 +0900 | Cezary Kaliszyk | merge | changeset |
files | 
| Mon, 20 Jun 2011 20:08:16 +0900 | Cezary Kaliszyk | Abs_set_fcb | changeset |
files | 
| Mon, 20 Jun 2011 20:09:30 +0900 | Cezary Kaliszyk | function for let-rec | changeset |
files | 
| Mon, 20 Jun 2011 10:16:12 +0900 | Cezary Kaliszyk | TODO/minor | changeset |
files | 
| Mon, 20 Jun 2011 09:59:18 +0900 | Cezary Kaliszyk | Move lst_fcb to Nominal2_Abs | changeset |
files | 
| Mon, 20 Jun 2011 09:38:57 +0900 | Cezary Kaliszyk | More minor TODOs | changeset |
files | 
| Mon, 20 Jun 2011 09:36:16 +0900 | Cezary Kaliszyk | Update TODO | changeset |
files | 
| Mon, 20 Jun 2011 09:29:42 +0900 | Cezary Kaliszyk | Let/minor | changeset |
files | 
| Mon, 20 Jun 2011 08:50:13 +0900 | Cezary Kaliszyk | Update Quotient/TODO and remove some attic code | changeset |
files | 
| Sun, 19 Jun 2011 13:14:37 +0900 | Cezary Kaliszyk | merge | changeset |
files | 
| Sun, 19 Jun 2011 13:10:15 +0900 | Cezary Kaliszyk | little on cps2 | changeset |
files | 
| Thu, 16 Jun 2011 20:07:03 +0100 | Christian Urban | got rid of the boolean flag in the raw_equivariance function | changeset |
files | 
| Thu, 16 Jun 2011 23:11:50 +0900 | Cezary Kaliszyk | Fix | changeset |
files | 
| Thu, 16 Jun 2011 22:00:52 +0900 | Cezary Kaliszyk | merge | changeset |
files | 
| Thu, 16 Jun 2011 21:23:38 +0900 | Cezary Kaliszyk | CPS3 can be defined with eqvt_rhs. | changeset |
files | 
| Thu, 16 Jun 2011 13:32:36 +0100 | Christian Urban | moved for the moment CPS translations into the example directory | changeset |
files | 
| Thu, 16 Jun 2011 13:14:53 +0100 | Christian Urban | merged | changeset |
files | 
| Thu, 16 Jun 2011 13:14:16 +0100 | Christian Urban | added eqvt_at and invariant for boths sides of the equations | changeset |
files | 
| Thu, 16 Jun 2011 20:56:30 +0900 | Cezary Kaliszyk | Added the CPS translation experiments. CPS1 comes with all the proofs, CPS2,3 just have the function and need eqvt_rhs to finish the obligations. | changeset |
files | 
| Thu, 16 Jun 2011 12:12:25 +0100 | Christian Urban | added a test that every function must be of pt-sort | changeset |
files | 
| Thu, 16 Jun 2011 11:03:01 +0100 | Christian Urban | all tests work again | changeset |
files | 
| 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 | changeset |
files | 
| Wed, 15 Jun 2011 12:52:48 +0100 | Christian Urban | added an abstract | changeset |
files | 
| Wed, 15 Jun 2011 12:32:40 +0100 | Christian Urban | added a stub for function paper; "isabelle make fnpaper" | changeset |
files | 
| Wed, 15 Jun 2011 11:06:48 +0900 | Cezary Kaliszyk | merge | changeset |
files | 
| Wed, 15 Jun 2011 11:06:31 +0900 | Cezary Kaliszyk | one TODO and one Problem? | changeset |
files | 
| Wed, 15 Jun 2011 09:51:26 +0900 | Cezary Kaliszyk | merge | changeset |
files | 
| Wed, 15 Jun 2011 09:50:53 +0900 | Cezary Kaliszyk | Some TODOs | changeset |
files | 
| Wed, 15 Jun 2011 09:31:59 +0900 | Cezary Kaliszyk | merge | changeset |
files | 
| Wed, 15 Jun 2011 09:25:36 +0900 | Cezary Kaliszyk | TypeSchemes work with 'default'. | changeset |
files | 
| Tue, 14 Jun 2011 19:11:44 +0100 | Christian Urban | tuned some proofs | changeset |
files | 
| Tue, 14 Jun 2011 14:07:07 +0100 | Christian Urban | fixed the problem when giving a complex default-term; the fundef lemmas in Nominal_Base were not general enough | changeset |
files | 
| Tue, 14 Jun 2011 11:43:06 +0100 | Christian Urban | tuned | changeset |
files | 
| Fri, 10 Jun 2011 15:52:17 +0900 | Cezary Kaliszyk | Move working examples before non-working ones | changeset |
files | 
| Fri, 10 Jun 2011 15:45:49 +0900 | Cezary Kaliszyk | Optimized proofs and removed some garbage. | changeset |
files | 
| Fri, 10 Jun 2011 15:31:14 +0900 | Cezary Kaliszyk | merge | changeset |
files | 
| Fri, 10 Jun 2011 15:30:09 +0900 | Cezary Kaliszyk | Slightly modify fcb for list1 and put in common place. | changeset |
files | 
| Fri, 10 Jun 2011 09:00:24 +0900 | Cezary Kaliszyk | Experiments with Let | changeset |
files | 
| Thu, 09 Jun 2011 15:34:51 +0900 | Cezary Kaliszyk | Eval can be defined with additional freshness | changeset |
files | 
| Thu, 09 Jun 2011 15:03:58 +0900 | Cezary Kaliszyk | Minor simplification | changeset |
files | 
| Thu, 09 Jun 2011 11:10:41 +0900 | Cezary Kaliszyk | abs_res_fcb will be enough to finish the multiple-recursive proof, if we have a working 'default'. | changeset |
files | 
| Thu, 09 Jun 2011 09:44:51 +0900 | Cezary Kaliszyk | More experiments with 'default' | changeset |
files | 
| Wed, 08 Jun 2011 21:44:03 +0900 | Cezary Kaliszyk | Finished the proof with the invariant | changeset |
files | 
| Wed, 08 Jun 2011 21:32:35 +0900 | Cezary Kaliszyk | Issue with 'default' | changeset |
files | 
| Wed, 08 Jun 2011 12:30:56 +0100 | Christian Urban | merged | changeset |
files | 
| Wed, 08 Jun 2011 12:30:46 +0100 | Christian Urban | merged | changeset |
files | 
| Wed, 08 Jun 2011 08:44:01 +0100 | Christian Urban | using the option "default" the function package allows one to give an explicit default value | changeset |
files | 
| Wed, 08 Jun 2011 17:52:06 +0900 | Cezary Kaliszyk | Simpler proof of TypeSchemes/substs | changeset |
files | 
| Wed, 08 Jun 2011 17:25:54 +0900 | Cezary Kaliszyk | Simplify fcb_res | changeset |
files | 
| Wed, 08 Jun 2011 09:56:39 +0900 | Cezary Kaliszyk | FCB for res binding and simplified proof of subst for type schemes | changeset |
files | 
| Wed, 08 Jun 2011 07:06:20 +0900 | Cezary Kaliszyk | Simplify ln-trans proof | changeset |
files | 
| Wed, 08 Jun 2011 07:02:52 +0900 | Cezary Kaliszyk | cbvs can be easily defined without an invariant | changeset |
files | 
| Tue, 07 Jun 2011 20:58:00 +0100 | Christian Urban | defined the "count-bound-variables-occurences" function which has an accumulator like trans | changeset |
files | 
| Tue, 07 Jun 2011 17:45:38 +0100 | Christian Urban | merged | changeset |
files | 
| Tue, 07 Jun 2011 23:42:12 +0900 | Cezary Kaliszyk | remove garbage (proofs that assumes the invariant outside function) | changeset |
files | 
| Tue, 07 Jun 2011 23:38:39 +0900 | Cezary Kaliszyk | Proof of trans with invariant | changeset |
files | 
| Tue, 07 Jun 2011 23:22:58 +0900 | Cezary Kaliszyk | Testing invariant in Lambda_F_T | changeset |
files | 
| 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 | changeset |
files | 
| 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 | changeset |
files | 
| Mon, 06 Jun 2011 13:11:04 +0100 | Christian Urban | slightly stronger property in fundef_ex_prop | changeset |
files | 
| Sun, 05 Jun 2011 21:14:23 +0100 | Christian Urban | added an option for an invariant (at the moment only a stub) | changeset |
files | 
| Sun, 05 Jun 2011 16:58:18 +0100 | Christian Urban | added a more general lemma fro fundef_ex1 | changeset |
files |