2010-09-17 Christian Urban updated to Isabelle Sept 13
2010-09-12 Christian Urban tuned code
2010-09-10 Christian Urban tuned (to conform with indentation policy of Markus)
2010-09-10 Christian Urban supp-proofs work except for CoreHaskell and Modules (induct is probably not finding the correct instance)
2010-09-04 Christian Urban generated inducts rule by Project_Rule.projections
2010-09-04 Christian Urban added the definition supp_rel (support w.r.t. a relation)
2010-09-04 Christian Urban merged
2010-09-03 Christian Urban got rid of Nominal2_Supp (is now in Nomina2_Base)
2010-09-03 Christian Urban moved everything out of Nominal_Supp
2010-09-03 Christian Urban renamed alpha_gen -> alpha_set and Abs -> Abs_set etc
2010-09-03 Christian Urban moved a proof to Abs
2010-09-03 Christian Urban got rid of Nominal_Atoms (folded into Nominal2_Base)
2010-09-03 Christian Urban cleaned a bit various thy-files in Nominal-General
2010-09-03 Christian Urban adapted paper to changes
2010-09-03 Christian Urban made the fv-definition aggree more with alpha (needed in the support proofs)
2010-09-03 Christian Urban removed lemma finite_set (already in simpset)
2010-09-03 Christian Urban added supp_set lemma
2010-09-02 Christian Urban some experiments with support
2010-09-01 Christian Urban added eqvt-attribute for permute_abs lemmas
2010-08-31 Christian Urban slides of my talk
2010-08-30 Cezary Kaliszyk merge
2010-08-30 Cezary Kaliszyk update qpaper to new isabelle
2010-08-30 Cezary Kaliszyk No need to unfold mem_def with rsp/prs (requires new isabelle).
2010-08-30 Cezary Kaliszyk Anonymize, change Quotient to Quot and fix indentation
2010-08-29 Christian Urban renamed NewParser to Nominal2
2010-08-29 Christian Urban tuned
2010-08-29 Christian Urban updated todos
2010-08-28 Christian Urban added fs-instance proofs
2010-08-28 Christian Urban added proofs for fsupp properties
2010-08-28 Christian Urban fiexed problem with constructors that have no arguments
2010-08-28 Christian Urban proved supports lemmas
2010-08-28 Christian Urban slight cleaning
2010-08-28 Christian Urban updated to new Isabelle
2010-08-27 Christian Urban cut out most of the lifting section and cleaned up everything
2010-08-27 Christian Urban made all typographic changes
2010-08-27 Christian Urban first pass on section 1
2010-08-27 Christian Urban make copies of the "old" files
2010-08-27 Cezary Kaliszyk Ball Bex can be lifted after unfolding.
2010-08-26 Christian Urban "isabelle make test" makes all major examples....they work up to supp theorems (excluding)
2010-08-26 Christian Urban merged
2010-08-26 Christian Urban corrected bug with fv-function generation (that was the problem with recursive binders)
2010-08-26 Cezary Kaliszyk minor
2010-08-25 Christian Urban cleaned up (almost completely) the examples
2010-08-25 Christian Urban cleaning of unused files and code
2010-08-25 Christian Urban automatic lifting
2010-08-25 Christian Urban everything now lifts as expected
2010-08-25 Christian Urban now every lemma lifts (even with type variables)
2010-08-25 Christian Urban can now deal with type variables in nominal datatype definitions
2010-08-22 Christian Urban updated to new Isabelle
2010-08-22 Christian Urban merged
2010-08-22 Christian Urban updated to new Isabelle
2010-08-21 Christian Urban not needed anymore
2010-08-21 Christian Urban moved lifting code from Lift.thy to nominal_dt_quot.ML
2010-08-21 Christian Urban nominal_datatypes with type variables do not work
2010-08-21 Christian Urban changed parser so that the binding mode is indicated as "bind (list)", "bind (set)" or "bind (res)"; if only "bind" is given, then bind (list) is assumed as default
2010-08-20 Cezary Kaliszyk Clarifications to FIXMEs.
2010-08-20 Cezary Kaliszyk Finished adding remarks from the reviewers.
2010-08-20 Cezary Kaliszyk few remaining remarks as fixme's.
2010-08-19 Christian Urban used @{const_name} hopefully everywhere
2010-08-19 Cezary Kaliszyk Intuition behind REL
2010-08-19 Cezary Kaliszyk add missing mathpartir
2010-08-19 Cezary Kaliszyk Add 2 FIXMEs
2010-08-19 Cezary Kaliszyk The type does determine respectfulness, the constant without an instantiated type does not.
2010-08-19 Cezary Kaliszyk Add the SAC stylesheet and updated root file.
2010-08-19 Cezary Kaliszyk TODO
2010-08-19 Cezary Kaliszyk further comments from the referees
2010-08-19 Cezary Kaliszyk fixes for referees
2010-08-17 Christian Urban put everything in a "timeit"
2010-08-17 Christian Urban improved runtime slightly, by constructing an explicit size measure for the function definitions
2010-08-17 Christian Urban more tuning of the code
2010-08-17 Christian Urban deleted unused code
2010-08-17 Christian Urban improved code
2010-08-16 Christian Urban can also lift the various eqvt lemmas for bn, fv, fv_bn and size
2010-08-16 Christian Urban also able to lift the bn_defs
2010-08-16 Christian Urban added rsp-lemmas for alpha_bns
2010-08-16 Christian Urban cezary made the eq_iff lemmas to lift (still needs some infrastructure in quotient)
2010-08-16 Christian Urban pinpointed the problem
2010-08-16 Christian Urban modified the code for class instantiations (with help from Florian)
2010-08-15 Christian Urban defined qperms and qsizes
2010-08-15 Christian Urban simplified code
2010-08-14 Christian Urban improved code
2010-08-14 Christian Urban more experiments with lifting
2010-08-12 Christian Urban updated to Isabelle 12th Aug
2010-08-11 Christian Urban rsp for constructors
2010-08-11 Christian Urban updated to Isabelle 11 Aug
2010-08-11 Christian Urban added a function that transforms the helper-rsp lemmas into real rsp lemmas
2010-08-08 Christian Urban proved rsp-helper lemmas of size functions
2010-07-31 Christian Urban tuning
2010-07-31 Christian Urban further simplification with alpha_prove
2010-07-31 Christian Urban introduced a general alpha_prove method
2010-07-29 Christian Urban equivariance for size
2010-07-29 Christian Urban helper lemmas for rsp-lemmas
2010-07-27 Christian Urban tests
2010-07-27 Christian Urban cleaned up a bit Abs.thy
2010-07-27 Christian Urban fixed order of fold_union to make alpha and fv agree
2010-07-26 Christian Urban small cleaning
2010-07-25 Christian Urban added paper by james; some minor cleaning
2010-07-23 Christian Urban samll changes
2010-07-23 Christian Urban made compatible
2010-07-23 Christian Urban added
2010-07-22 Christian Urban updated to new Isabelle; made FSet more "quiet"
2010-07-20 Christian Urban merged
2010-07-19 Christian Urban minor
2010-07-19 Christian Urban minor polishing
2010-07-19 Christian Urban quote for a new paper
2010-07-19 Christian Urban corrected lambda-preservation theorem
2010-07-19 Christian Urban minor
2010-07-18 Christian Urban minor things on the paper
2010-07-18 Christian Urban merged
2010-07-18 Christian Urban minor things
2010-07-18 Christian Urban some test with quotient
2010-07-17 Christian Urban some minor changes
(0) -1000 -112 +112 tip