Mon, 11 Jul 2011 12:23:24 +0100 Christian Urban some more experiments with let and bns
Fri, 08 Jul 2011 05:04:23 +0200 Christian Urban some code refactoring
Thu, 07 Jul 2011 16:17:03 +0200 Christian Urban merged
Thu, 07 Jul 2011 16:16:42 +0200 Christian Urban code refactoring; introduced a record for raw_dt_info
Wed, 06 Jul 2011 23:11:30 +0200 Christian Urban more on NBE
Wed, 06 Jul 2011 15:59:11 +0200 Christian Urban more on the NBE function
Wed, 06 Jul 2011 01:04:09 +0200 Christian Urban a little further with NBE
Wed, 06 Jul 2011 07:42:12 +0900 Cezary Kaliszyk Setup eqvt_at for first goal
Wed, 06 Jul 2011 00:34:42 +0200 Christian Urban attempt for NBE
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 18:01:54 +0200 Christian Urban side commment for future use
Tue, 05 Jul 2011 16:22:18 +0200 Christian Urban made the tests go through again
Tue, 05 Jul 2011 15:01:10 +0200 Christian Urban added another example which seems difficult to define
Tue, 05 Jul 2011 15:00:41 +0200 Christian Urban added a tactic "all_trivials" which simplifies all trivial constructor cases and leaves the others untouched.
Tue, 05 Jul 2011 04:23:33 +0200 Christian Urban merged
Tue, 05 Jul 2011 04:19:02 +0200 Christian Urban all FCB lemmas
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:56:19 +0200 Christian Urban merged
Mon, 04 Jul 2011 23:55:46 +0200 Christian Urban tuned
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
Mon, 04 Jul 2011 14:47:21 +0900 Cezary Kaliszyk Let with a different invariant; not true.
Sun, 03 Jul 2011 21:04:46 +0900 Cezary Kaliszyk Add non-working Lambda_F_T using FCB2
Sun, 03 Jul 2011 21:04:06 +0900 Cezary Kaliszyk Added non-working CPS3 using FCB2
Sun, 03 Jul 2011 21:01:07 +0900 Cezary Kaliszyk Change CPS1 to FCB2
Sat, 02 Jul 2011 12:40:59 +0900 Cezary Kaliszyk Did the proofs of height and subst for Let with list-like binders. Having apply_assns allows proving things by alpha_bn
Sat, 02 Jul 2011 00:27:47 +0100 Christian Urban side-by-side tests of lets with single assignment; deep-binder case works if the recursion is avoided using an auxiliary function
Fri, 01 Jul 2011 17:46:15 +0900 Cezary Kaliszyk Exhaust Issue
Thu, 30 Jun 2011 11:05:25 +0100 Christian Urban clarified a sentence
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 19:21:26 +0100 Christian Urban moved Classical and Let temporarily into a section where "sorry" is allowed; this makes all test go through
Wed, 29 Jun 2011 17:01:09 +0100 Christian Urban added a warning if a theorem is already declared as equivariant
Wed, 29 Jun 2011 16:44:54 +0100 Christian Urban merged
Wed, 29 Jun 2011 13:04:24 +0900 Cezary Kaliszyk Prove bn injectivity and experiment more with Let
Wed, 29 Jun 2011 00:48:50 +0100 Christian Urban some experiments
Tue, 28 Jun 2011 14:45:30 +0900 Cezary Kaliszyk trying new fcb in let/subst
Tue, 28 Jun 2011 14:30:30 +0900 Cezary Kaliszyk Leftover only inj and eqvt
Tue, 28 Jun 2011 14:18:26 +0900 Cezary Kaliszyk eapply fcb ok
Tue, 28 Jun 2011 14:01:15 +0900 Cezary Kaliszyk Removed Inl and Inr
Tue, 28 Jun 2011 14:49:48 +0100 Christian Urban relaxed type in fcb
Tue, 28 Jun 2011 14:34:07 +0100 Christian Urban fcb with explicit bn function
Tue, 28 Jun 2011 14:01:52 +0100 Christian Urban added let-rec example
Tue, 28 Jun 2011 12:36:34 +0900 Cezary Kaliszyk Experiments with res
Tue, 28 Jun 2011 00:48:57 +0100 Christian Urban proved the fcb also for sets (no restriction yet)
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
Mon, 27 Jun 2011 22:51:42 +0100 Christian Urban streamlined the fcb-proof and made fcb1 a special case of fcb
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)
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.
Mon, 27 Jun 2011 19:13:55 +0100 Christian Urban renamed ds to dset (disagreement set)
Mon, 27 Jun 2011 12:15:21 +0100 Christian Urban added small lemma about disagreement set
Mon, 27 Jun 2011 08:42:02 +0900 Cezary Kaliszyk merge
Mon, 27 Jun 2011 08:38:54 +0900 Cezary Kaliszyk New-style fcb for multiple binders.
Mon, 27 Jun 2011 04:01:55 +0900 Cezary Kaliszyk equality of lst_binder and a few helper lemmas
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)
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
Sat, 25 Jun 2011 22:51:43 +0100 Christian Urban did all cases, except the multiple binder case
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.
Fri, 24 Jun 2011 09:42:44 +0100 Christian Urban except for the interated binder case, finished definition in Calssical.thy
Fri, 24 Jun 2011 11:18:18 +0900 Cezary Kaliszyk Make examples work with non-precompiled image
Fri, 24 Jun 2011 11:15:22 +0900 Cezary Kaliszyk Remove Lambda_add.thy
Fri, 24 Jun 2011 11:14:58 +0900 Cezary Kaliszyk The examples in Lambda_add can be defined by nominal_function directly
Fri, 24 Jun 2011 11:03:53 +0900 Cezary Kaliszyk Theory name changes for JEdit
Fri, 24 Jun 2011 10:54:31 +0900 Cezary Kaliszyk More usual names for substitution properties
Fri, 24 Jun 2011 10:30:06 +0900 Cezary Kaliszyk Second Fixed Point Theorem
Fri, 24 Jun 2011 10:12:47 +0900 Cezary Kaliszyk Speed-up the completeness proof.
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
Thu, 23 Jun 2011 13:09:17 +0100 Christian Urban added file
Thu, 23 Jun 2011 12:28:25 +0100 Christian Urban expanded the example
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
Wed, 22 Jun 2011 17:57:15 +0900 Cezary Kaliszyk constants with the same names
Wed, 22 Jun 2011 04:49:56 +0900 Cezary Kaliszyk Quotients/TODO addtion
Tue, 21 Jun 2011 23:59:36 +0900 Cezary Kaliszyk Minor
Tue, 21 Jun 2011 10:39:25 +0900 Cezary Kaliszyk merge
Tue, 21 Jun 2011 10:37:43 +0900 Cezary Kaliszyk spelling
Mon, 20 Jun 2011 20:09:51 +0900 Cezary Kaliszyk merge
Mon, 20 Jun 2011 20:08:16 +0900 Cezary Kaliszyk Abs_set_fcb
Mon, 20 Jun 2011 20:09:30 +0900 Cezary Kaliszyk function for let-rec
Mon, 20 Jun 2011 10:16:12 +0900 Cezary Kaliszyk TODO/minor
Mon, 20 Jun 2011 09:59:18 +0900 Cezary Kaliszyk Move lst_fcb to Nominal2_Abs
Mon, 20 Jun 2011 09:38:57 +0900 Cezary Kaliszyk More minor TODOs
Mon, 20 Jun 2011 09:36:16 +0900 Cezary Kaliszyk Update TODO
Mon, 20 Jun 2011 09:29:42 +0900 Cezary Kaliszyk Let/minor
Mon, 20 Jun 2011 08:50:13 +0900 Cezary Kaliszyk Update Quotient/TODO and remove some attic code
Sun, 19 Jun 2011 13:14:37 +0900 Cezary Kaliszyk merge
Sun, 19 Jun 2011 13:10:15 +0900 Cezary Kaliszyk little on cps2
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 23:11:50 +0900 Cezary Kaliszyk Fix
Thu, 16 Jun 2011 22:00:52 +0900 Cezary Kaliszyk merge
Thu, 16 Jun 2011 21:23:38 +0900 Cezary Kaliszyk CPS3 can be defined with eqvt_rhs.
Thu, 16 Jun 2011 13:32:36 +0100 Christian Urban moved for the moment CPS translations into the example directory
Thu, 16 Jun 2011 13:14:53 +0100 Christian Urban merged
Thu, 16 Jun 2011 13:14:16 +0100 Christian Urban added eqvt_at and invariant for boths sides of the equations
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.
Thu, 16 Jun 2011 12:12:25 +0100 Christian Urban added a test that every function must be of pt-sort
Thu, 16 Jun 2011 11:03:01 +0100 Christian Urban all tests work again
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 12:52:48 +0100 Christian Urban added an abstract
Wed, 15 Jun 2011 12:32:40 +0100 Christian Urban added a stub for function paper; "isabelle make fnpaper"
Wed, 15 Jun 2011 11:06:48 +0900 Cezary Kaliszyk merge
Wed, 15 Jun 2011 11:06:31 +0900 Cezary Kaliszyk one TODO and one Problem?
Wed, 15 Jun 2011 09:51:26 +0900 Cezary Kaliszyk merge
Wed, 15 Jun 2011 09:50:53 +0900 Cezary Kaliszyk Some TODOs
Wed, 15 Jun 2011 09:31:59 +0900 Cezary Kaliszyk merge
Wed, 15 Jun 2011 09:25:36 +0900 Cezary Kaliszyk TypeSchemes work with 'default'.
Tue, 14 Jun 2011 19:11:44 +0100 Christian Urban tuned some proofs
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
Tue, 14 Jun 2011 11:43:06 +0100 Christian Urban tuned
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:31:14 +0900 Cezary Kaliszyk merge
Fri, 10 Jun 2011 15:30:09 +0900 Cezary Kaliszyk Slightly modify fcb for list1 and put in common place.
Fri, 10 Jun 2011 09:00:24 +0900 Cezary Kaliszyk Experiments with Let
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
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'.
Thu, 09 Jun 2011 09:44:51 +0900 Cezary Kaliszyk More experiments with 'default'
Wed, 08 Jun 2011 21:44:03 +0900 Cezary Kaliszyk Finished the proof with the invariant
Wed, 08 Jun 2011 21:32:35 +0900 Cezary Kaliszyk Issue with 'default'
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 08:44:01 +0100 Christian Urban using the option "default" the function package allows one to give an explicit default value
Wed, 08 Jun 2011 17:52:06 +0900 Cezary Kaliszyk Simpler proof of TypeSchemes/substs
Wed, 08 Jun 2011 17:25:54 +0900 Cezary Kaliszyk Simplify fcb_res
Wed, 08 Jun 2011 09:56:39 +0900 Cezary Kaliszyk FCB for res binding and simplified proof of subst for type schemes
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 23:22:58 +0900 Cezary Kaliszyk Testing invariant in Lambda_F_T
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
Mon, 06 Jun 2011 13:11:04 +0100 Christian Urban slightly stronger property in fundef_ex_prop
Sun, 05 Jun 2011 21:14:23 +0100 Christian Urban added an option for an invariant (at the moment only a stub)
Sun, 05 Jun 2011 16:58:18 +0100 Christian Urban added a more general lemma fro fundef_ex1
Sat, 04 Jun 2011 14:50:57 +0900 Cezary Kaliszyk Trying the induction on the graph
Sat, 04 Jun 2011 09:07:50 +0900 Cezary Kaliszyk Finish and test the locale approach
Fri, 03 Jun 2011 22:31:44 +0900 Cezary Kaliszyk FiniteSupp precondition in the function is enough to get rid of completeness obligationss
Fri, 03 Jun 2011 12:46:23 +0100 Christian Urban recursion combinator inside a locale
Fri, 03 Jun 2011 18:33:11 +0900 Cezary Kaliszyk merge
Fri, 03 Jun 2011 18:32:22 +0900 Cezary Kaliszyk F for lambda used to define translation to locally nameless
Thu, 02 Jun 2011 16:15:18 +0100 Christian Urban typo
Thu, 02 Jun 2011 15:35:33 +0100 Christian Urban removed dead code
Thu, 02 Jun 2011 22:24:33 +0900 Cezary Kaliszyk finished the missing obligations
Thu, 02 Jun 2011 12:14:03 +0100 Christian Urban merged
Thu, 02 Jun 2011 12:09:31 +0100 Christian Urban a test with a recursion combinator defined on top of nominal_primrec
Thu, 02 Jun 2011 16:41:09 +0900 Cezary Kaliszyk Use FCB to simplify proof
Thu, 02 Jun 2011 10:11:50 +0900 Cezary Kaliszyk merge
Thu, 02 Jun 2011 10:09:23 +0900 Cezary Kaliszyk Remove SMT
Wed, 01 Jun 2011 22:55:14 +0100 Christian Urban hopefully final fix for ho-functions
Wed, 01 Jun 2011 21:03:30 +0100 Christian Urban first test to fix the problem with free variables
Wed, 01 Jun 2011 16:13:42 +0900 Cezary Kaliszyk proved subst for All constructor in type schemes.
Wed, 01 Jun 2011 13:41:30 +0900 Cezary Kaliszyk DB translation using index; easier to reason about.
Wed, 01 Jun 2011 13:35:37 +0900 Cezary Kaliszyk Problem: free variables in the goal
Wed, 01 Jun 2011 11:01:39 +0900 Cezary Kaliszyk fixed previous commit
Wed, 01 Jun 2011 10:59:07 +0900 Cezary Kaliszyk equivariance of db_trans
Tue, 31 May 2011 12:22:28 +0100 Christian Urban fixed the problem with cps-like functions
Tue, 31 May 2011 14:12:31 +0900 Cezary Kaliszyk DeBruijn translation in a simplifier friendly way
Tue, 31 May 2011 13:25:35 +0900 Cezary Kaliszyk map_term can be defined when equivariance is assumed
Tue, 31 May 2011 13:21:00 +0900 Cezary Kaliszyk map_term is not a function the way it is defined
Tue, 31 May 2011 12:59:10 +0900 Cezary Kaliszyk Defined translation from nominal to de-Bruijn; with a freshness condition for the lambda case.
Tue, 31 May 2011 12:54:21 +0900 Cezary Kaliszyk Simple eqvt proofs with perm_simps for clarity
Tue, 31 May 2011 00:36:16 +0100 Christian Urban tuned last commit
Tue, 31 May 2011 00:17:22 +0100 Christian Urban functions involving if and case do not throw exceptions anymore; but eqvt_at assumption has now a precondition
Thu, 26 May 2011 06:36:29 +0200 Christian Urban updated to new Isabelle
Wed, 25 May 2011 21:38:50 +0200 Christian Urban added eq_iff and distinct lemmas of nominal datatypes to the simplifier
Tue, 24 May 2011 19:39:38 +0200 Christian Urban more on slides
Sun, 22 May 2011 10:20:18 +0200 Christian Urban added slides for copenhagen
Sat, 14 May 2011 10:16:16 +0100 Christian Urban added a problem with inductive_cases (reported by Randy)
Fri, 13 May 2011 14:50:17 +0100 Christian Urban misc
Tue, 10 May 2011 17:10:22 +0100 Christian Urban made the subtyping work again
Tue, 10 May 2011 07:47:06 +0100 Christian Urban updated to new Isabelle (> 9 May)
Mon, 09 May 2011 04:49:58 +0100 Christian Urban merged
Tue, 03 May 2011 15:39:30 +0100 Christian Urban added two mutual recursive inductive definitions
Tue, 03 May 2011 13:25:02 +0100 Christian Urban deleted two functions from the API
Tue, 03 May 2011 13:09:08 +0100 Christian Urban proved that lfp is equivariant (that simplifies equivariance proofs of inductively defined predicates)
Mon, 09 May 2011 04:46:43 +0100 Christian Urban more on pearl-paper
Wed, 04 May 2011 15:27:04 +0800 Christian Urban more on pearl-paper
Mon, 02 May 2011 13:01:02 +0800 Christian Urban updated Quotient paper so that it compiles again
Thu, 28 Apr 2011 11:51:01 +0800 Christian Urban merged
Thu, 28 Apr 2011 11:44:36 +0800 Christian Urban added slides for beijing
Fri, 22 Apr 2011 00:18:25 +0800 Christian Urban more to the pearl paper
Tue, 19 Apr 2011 13:03:08 +0100 Christian Urban updated to snapshot Isabelle 19 April
Mon, 18 Apr 2011 15:57:45 +0100 Christian Urban merged
Mon, 18 Apr 2011 15:56:07 +0100 Christian Urban added permute_pure back into the nominal_inductive procedure; updated to Isabelle 17 April
Fri, 15 Apr 2011 15:20:56 +0900 Cezary Kaliszyk New way of forward elimination of Abs1_eq and simplifications of the function obligation proofs.
Wed, 13 Apr 2011 13:44:25 +0100 Christian Urban merged
Wed, 13 Apr 2011 13:41:52 +0100 Christian Urban introduced framework for finetuning eqvt-rules; this solves problem with permute_pure called in nominal_inductive
Tue, 12 Apr 2011 15:46:35 +0800 Christian Urban shanghai slides
Mon, 11 Apr 2011 02:25:25 +0100 Christian Urban pictures for slides
Mon, 11 Apr 2011 02:04:11 +0100 Christian Urban Shanghai slides
Sun, 10 Apr 2011 14:13:55 +0800 Christian Urban more paper
Sun, 10 Apr 2011 07:41:52 +0800 Christian Urban eqvt of supp and fresh is proved using equivariance infrastructure
Sun, 10 Apr 2011 04:07:15 +0800 Christian Urban more paper
Sat, 09 Apr 2011 13:44:49 +0800 Christian Urban more on the paper
Sat, 09 Apr 2011 00:29:40 +0100 Christian Urban tuned paper
Sat, 09 Apr 2011 00:28:53 +0100 Christian Urban tuned paper
Sat, 09 Apr 2011 02:10:49 +0800 Christian Urban typo
Fri, 08 Apr 2011 14:23:28 +0800 Christian Urban more on paper
Fri, 08 Apr 2011 03:47:50 +0800 Christian Urban eqvt_lambda without eta-expansion
Wed, 06 Apr 2011 13:47:08 +0100 Christian Urban changed default preprocessor that does not catch variables only occuring on the right
Thu, 31 Mar 2011 15:25:35 +0200 Christian Urban final version of slides
Wed, 30 Mar 2011 22:27:26 +0200 Christian Urban more on the slides
Wed, 30 Mar 2011 08:11:36 +0200 Christian Urban tuned IsaMakefile
Tue, 29 Mar 2011 23:52:14 +0200 Christian Urban rearranged directories and updated to new Isabelle
Wed, 16 Mar 2011 21:14:43 +0100 Christian Urban precise path to LaTeXsugar
Wed, 16 Mar 2011 21:07:50 +0100 Christian Urban a lit bit more on the pearl-jv paper
Wed, 16 Mar 2011 20:42:14 +0100 Christian Urban ported changes from function package....needs Isabelle 16 March or above
Tue, 15 Mar 2011 00:40:39 +0100 Christian Urban more on the pearl paper
Mon, 14 Mar 2011 16:35:59 +0100 Christian Urban equivariance for All and Ex can be proved in terms of their definition
Fri, 11 Mar 2011 08:51:39 +0000 Christian Urban more on the paper
Tue, 08 Mar 2011 09:07:49 +0000 Christian Urban merged
Tue, 08 Mar 2011 09:07:27 +0000 Christian Urban more on the pearl paper
Wed, 02 Mar 2011 16:07:56 +0900 Cezary Kaliszyk distinct names at toplevel
Wed, 02 Mar 2011 12:49:01 +0900 Cezary Kaliszyk merge
Wed, 02 Mar 2011 12:48:00 +0900 Cezary Kaliszyk Pairing function
Wed, 02 Mar 2011 00:06:28 +0000 Christian Urban updated pearl papers
Tue, 01 Mar 2011 00:14:02 +0000 Christian Urban a bit more tuning
Mon, 28 Feb 2011 16:47:13 +0000 Christian Urban included old test cases for perm_simp into ROOT.ML file
Mon, 28 Feb 2011 15:21:10 +0000 Christian Urban split the library into a basics file; merged Nominal_Eqvt into Nominal_Base
Fri, 25 Feb 2011 21:23:30 +0000 Christian Urban some slight polishing
Thu, 24 Feb 2011 18:50:02 +0000 Christian Urban merged
Thu, 24 Feb 2011 16:26:11 +0000 Christian Urban added a lemma about fresh_star and Abs
Wed, 23 Feb 2011 11:11:02 +0900 Cezary Kaliszyk Reduce the definition of trans to FCB; test that FCB can be proved with simp rules.
Sat, 19 Feb 2011 09:31:22 +0900 Cezary Kaliszyk typeschemes/subst
Thu, 17 Feb 2011 17:02:25 +0900 Cezary Kaliszyk further experiments with typeschemes subst
Thu, 17 Feb 2011 12:01:08 +0900 Cezary Kaliszyk Finished the proof of a function that invents fresh variable names.
Wed, 16 Feb 2011 14:44:33 +0000 Christian Urban added eqvt for length
Wed, 16 Feb 2011 14:03:26 +0000 Christian Urban added eqvt lemmas for filter and distinct
Mon, 07 Feb 2011 16:00:24 +0000 Christian Urban added eqvt for cartesian products
Mon, 07 Feb 2011 15:59:37 +0000 Christian Urban cleaned up the experiments so that the tests go through
Sat, 05 Feb 2011 07:39:00 +0900 Cezary Kaliszyk merge
(0) -1000 -240 +240 tip