Nominal/NewParser.thy
2010-08-28 Christian Urban added fs-instance proofs
2010-08-28 Christian Urban added proofs for fsupp properties
2010-08-28 Christian Urban proved supports lemmas
2010-08-26 Christian Urban "isabelle make test" makes all major examples....they work up to supp theorems (excluding)
2010-08-26 Christian Urban corrected bug with fv-function generation (that was the problem with recursive binders)
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 can now deal with type variables in nominal datatype definitions
2010-08-22 Christian Urban updated to new Isabelle
2010-08-22 Christian Urban updated to new Isabelle
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-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 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 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-08 Christian Urban proved rsp-helper lemmas of size functions
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 fixed order of fold_union to make alpha and fv agree
2010-07-22 Christian Urban updated to new Isabelle; made FSet more "quiet"
2010-07-16 Christian Urban more on the paper
2010-07-07 Christian Urban more on the paper
2010-06-28 Christian Urban more quotient-definitions
2010-06-28 Christian Urban slight cleaning
2010-06-27 Christian Urban fixed according to changes in quotient
2010-06-24 Christian Urban added definition of the quotient types
2010-06-23 Christian Urban deleted compose-lemmas in Abs (not needed anymore)
2010-06-23 Christian Urban deleted equivp_hack
2010-06-22 Christian Urban proved eqvip theorems for alphas
2010-06-22 Christian Urban cleaned up the FSet (noise was introduced by error)
2010-06-22 Christian Urban prove that alpha implies alpha_bn (needed for rsp proofs)
2010-06-11 Christian Urban also symmetry
2010-06-10 Christian Urban premerge
2010-06-09 Christian Urban transitivity proofs done
2010-06-07 Christian Urban work on transitivity proof
2010-06-03 Christian Urban fixed problem with eqvt proofs
2010-06-02 Christian Urban fixed problem with bn_info
2010-06-01 Christian Urban equivariance done
2010-06-01 Christian Urban smaller code for raw-eqvt proofs
2010-05-31 Christian Urban all raw definitions are defined using function
2010-05-27 Christian Urban intermediate state
2010-05-26 Christian Urban merged
2010-05-26 Christian Urban added FSet to the correct paper
2010-05-24 Christian Urban added slides
2010-05-24 Christian Urban tuned
2010-05-24 Christian Urban tuned
2010-05-24 Christian Urban alpha works now
2010-05-23 Christian Urban started to work on alpha
2010-05-22 Christian Urban properly exported bn_descr
2010-05-21 Christian Urban hving a working fv-definition without the export
2010-05-21 Christian Urban tuned
2010-05-20 Christian Urban new fv/fv_bn function (supp breaks now); exported raw perms and raw funs into separate ML-files
2010-05-21 Cezary Kaliszyk Renamings
2010-05-17 Christian Urban minor tuning
2010-05-17 Christian Urban slight tuning
2010-05-17 Christian Urban somewhat simplified the main parsing function; failed to move a Note-statement to define_raw_perms
2010-05-16 Christian Urban moved the exporting part into the parser (this is still a hack); re-added CoreHaskell again to the examples - there seems to be a problem with the variable name pat
2010-05-13 Christian Urban made out of STEPS a configuration value so that it can be set individually in each file
2010-05-13 Christian Urban added term4 back to the examples
2010-05-12 Christian Urban merged
2010-05-12 Christian Urban moved the data-transformation into the parser
2010-05-12 Cezary Kaliszyk Move alpha_eqvt to unused.
2010-05-12 Cezary Kaliszyk Use equivariance instead of alpha_eqvt
2010-05-12 Christian Urban ingnored parameters in equivariance; added a proper interface to be called from ML
2010-05-12 Christian Urban properly exported defined bn-functions
2010-05-11 Cezary Kaliszyk Include raw permutation definitions in eqvt
2010-05-10 Cezary Kaliszyk Parser changes for compound relations
2010-05-06 Cezary Kaliszyk mem => member
2010-05-04 Christian Urban increased step counter so that all steps go through
2010-05-04 Christian Urban fixed my error with define_raw_fv
2010-05-04 Christian Urban tuned and added some comments to the code; added also an exception for early exit of the nominal2_cmd function
2010-05-04 Christian Urban roll back of the last commit (there was a difference)
2010-05-04 Christian Urban to my best knowledge the number of datatypes is equal to the length of the dt_descr; so we can save one argument in define_raw_perm
2010-05-03 Cezary Kaliszyk Comment
2010-05-03 Cezary Kaliszyk Register only non-looping rules in eq_iff
2010-05-03 Cezary Kaliszyk NewParser
2010-05-03 Cezary Kaliszyk Introduce eq_iff_simp to match the one from Parser.
2010-05-03 Cezary Kaliszyk Cheat support equations in new parser
2010-05-03 Cezary Kaliszyk Add explicit cheats in NewParser and comment out the examples for outside use.
2010-05-03 Cezary Kaliszyk Fix Datatype_Aux calls in NewParser.
2010-05-02 Christian Urban tried to add some comments in the huge(!) nominal2_cmd function
2010-05-02 Christian Urban attempted to remove dependency on (old) Fv and (old) Parser; lifting still uses Fv.thy; the examples do not work at the moment (with equivp proofs failing)
2010-05-01 Christian Urban merged
2010-05-01 Christian Urban tuned
2010-04-30 Cezary Kaliszyk NewParser with Parser functionality, but some cheats included since the order of datayupes is wrong.
2010-04-30 Cezary Kaliszyk Merged nominal_datatype into NewParser until eqvts
2010-04-30 Cezary Kaliszyk more parser/new parser synchronization.
2010-04-30 Cezary Kaliszyk Change signature of fv and alpha generation.
2010-04-29 Cezary Kaliszyk New Alpha.
2010-04-29 Cezary Kaliszyk Fixing the definitions in the Parser.
2010-04-29 Cezary Kaliszyk Include support of unknown datatypes in new fv
2010-04-28 Christian Urban simpliied and moved the remaining lemmas about the atom-function to Nominal2_Base
2010-04-28 Christian Urban use sort at_base instead of at
2010-04-27 Christian Urban added some further problemetic tests
2010-04-27 Christian Urban some tuning
2010-04-27 Cezary Kaliszyk Rewrote FV code and included the function package.
2010-04-25 Christian Urban added definition of raw-permutations to the new-parser
2010-04-25 Christian Urban tuned
2010-04-24 Christian Urban slight tuning
2010-04-24 Christian Urban added a comment about a function where I am not sure who wrote it.
2010-04-24 Christian Urban merged
less more (0) tip