2010-03-18 Christian Urban added TODO
2010-03-18 Christian Urban vixed variable names
2010-03-18 Christian Urban simplified strong induction proof by using flip
2010-03-18 Cezary Kaliszyk Rename bound variables + minor cleaning.
2010-03-18 Cezary Kaliszyk Move most of the exporting out of the parser.
2010-03-18 Cezary Kaliszyk Prove pseudo-inject (eq-iff) on the exported level and rename appropriately.
2010-03-18 Cezary Kaliszyk Prove eqvts on exported terms.
2010-03-18 Cezary Kaliszyk Clean 'Lift', start working only on exported things in Parser.
2010-03-17 Christian Urban slightly more of the paper
2010-03-17 Christian Urban merged
2010-03-17 Christian Urban paper uses now a heap file - does not compile so long anymore
2010-03-17 Cezary Kaliszyk merge
2010-03-17 Cezary Kaliszyk compose_sym2 works also for term5
2010-03-17 Cezary Kaliszyk Updated Term1, including statement of strong induction.
2010-03-17 Cezary Kaliszyk Proper compose_sym2
2010-03-17 Christian Urban merged
2010-03-17 Christian Urban temporarily disabled tests in Nominal/ROOT
2010-03-17 Christian Urban made paper to compile
2010-03-17 Christian Urban added partial proof for the strong induction principle
2010-03-17 Cezary Kaliszyk Trying to find a compose lemma for 2 arguments.
2010-03-17 Cezary Kaliszyk merge
2010-03-17 Cezary Kaliszyk cheat_alpha_eqvt no longer needed. Cleaned the tracing messages.
2010-03-17 Christian Urban merged
2010-03-17 Christian Urban added proof of supp/fv for type schemes
2010-03-17 Cezary Kaliszyk Updated Type Schemes to automatic lifting. One goal is not true because of the restriction.
2010-03-17 Cezary Kaliszyk Remove Term5a, since it is now identical to Term5.
2010-03-17 Cezary Kaliszyk merge
2010-03-17 Cezary Kaliszyk Finished all proofs in Term5 and Term5n.
2010-03-17 Christian Urban added partial proof of supp for type schemes
2010-03-17 Cezary Kaliszyk Fix in alpha; support of the recursive Let works :)
2010-03-17 Cezary Kaliszyk The recursive supp just has one equation too much.
2010-03-17 Cezary Kaliszyk Fix for the change of alpha_gen.
2010-03-17 Cezary Kaliszyk merge
2010-03-17 Cezary Kaliszyk Generate compound FV and Alpha for recursive bindings.
2010-03-17 Cezary Kaliszyk Lifting theorems with compound fv and compound alpha.
2010-03-17 Christian Urban commented out examples that should not work; but for example type-scheme example should work
2010-03-17 Christian Urban added another supp-proof for the non-recursive case
2010-03-16 Cezary Kaliszyk Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
2010-03-16 Cezary Kaliszyk merge
2010-03-16 Cezary Kaliszyk The old recursive alpha works fine.
2010-03-16 Christian Urban added the final unfolded result
2010-03-16 Christian Urban merge and proof of support for non-recursive case
2010-03-16 Cezary Kaliszyk Added Term5 non-recursive. The bug is there only for the recursive case.
2010-03-16 Cezary Kaliszyk Alpha is wrong.
2010-03-16 Cezary Kaliszyk alpha_bn doesn't need the permutation in non-recursive case.
2010-03-16 Cezary Kaliszyk alpha5_transp and equivp
2010-03-16 Cezary Kaliszyk alpha5_symp proved.
2010-03-16 Cezary Kaliszyk FV_bn generated for recursive functions as well, and used in main fv for bindings.
2010-03-16 Cezary Kaliszyk The proof in 'Test' gets simpler.
2010-03-16 Cezary Kaliszyk Removed pi o bn = bn' assumption in alpha
2010-03-15 Christian Urban merged (confirmed to work with Isabelle from 6th March)
2010-03-15 Christian Urban another synchronisation
2010-03-15 Christian Urban proof for support when bn-function is present, but fb_function is empty
2010-03-15 Cezary Kaliszyk fv_eqvt_cheat no longer needed.
2010-03-15 Cezary Kaliszyk derive "inducts" from "induct" instead of lifting again is much faster.
2010-03-15 Cezary Kaliszyk build_eqvts works with recursive case if proper induction rule is used.
2010-03-15 Cezary Kaliszyk cheat_alpha_eqvt no longer needed; the proofs work.
2010-03-15 Cezary Kaliszyk LF works with new alpha...?
2010-03-15 Cezary Kaliszyk explicit flag "cheat_equivp"
2010-03-15 Cezary Kaliszyk Prove alpha_gen_compose_eqvt
2010-03-15 Cezary Kaliszyk Use eqvt.
2010-03-15 Christian Urban added preliminary test version....but Test works now
2010-03-15 Christian Urban added an eqvt-proof for bi
2010-03-15 Christian Urban synchronised with main hg-repository; used add_typedef_global in nominal_atoms
2010-03-14 Christian Urban localised the typedef in Attic (requires new Isabelle)
2010-03-13 Christian Urban started supp-fv proofs (is going to work)
2010-03-12 Cezary Kaliszyk Even with pattern simplified to a single clause, the supp equation doesn't seem true.
2010-03-12 Cezary Kaliszyk Still don't know how to prove supp=fv for simplest Let...
2010-03-11 Cezary Kaliszyk Do not fail if the finite support proof fails.
2010-03-11 Christian Urban generalised the supp for atoms to all concrete atoms (not just names)
2010-03-11 Christian Urban support of atoms at the end of Abs.thy
2010-03-11 Cezary Kaliszyk Trying to prove atom_image_fresh_swap
2010-03-11 Cezary Kaliszyk Finite_support proof no longer needed in LF.
2010-03-11 Cezary Kaliszyk Show that the new types are in finite support typeclass.
2010-03-11 Cezary Kaliszyk mk_supports_eq and supports_tac.
2010-03-11 Cezary Kaliszyk merge
2010-03-11 Cezary Kaliszyk Fixes for term1 for new alpha. Still not able to show support equations.
2010-03-11 Christian Urban merged
2010-03-11 Christian Urban finally the proof that new and old alpha agree
2010-03-11 Cezary Kaliszyk Remove "_raw" from lifted theorems.
2010-03-11 Cezary Kaliszyk looking at trm5_equivp
2010-03-11 Cezary Kaliszyk The cheats described explicitely.
2010-03-11 Cezary Kaliszyk The alpha5_eqvt tactic works if I manage to build the goal.
2010-03-11 Cezary Kaliszyk With the 4 cheats, all examples fully lift.
2010-03-11 Cezary Kaliszyk Lift alpha_bn_constants.
2010-03-11 Cezary Kaliszyk Lifting constants.
2010-03-11 Cezary Kaliszyk Proper error message.
2010-03-11 Cezary Kaliszyk Lifting constants works for all examples.
2010-03-11 Cezary Kaliszyk Remove tracing from fv/alpha.
2010-03-11 Cezary Kaliszyk Equivp working only on the standard alpha-equivalences.
2010-03-11 Cezary Kaliszyk explicit cheat_fv_eqvt
2010-03-11 Cezary Kaliszyk extract build_eqvts_tac.
2010-03-11 Cezary Kaliszyk build_eqvts no longer requires permutations.
2010-03-11 Cezary Kaliszyk Add explicit alpha_eqvt_cheat.
2010-03-11 Cezary Kaliszyk Export tactic out of alpha_eqvt.
2010-03-10 Cezary Kaliszyk merge
2010-03-10 Cezary Kaliszyk More tries about the proofs in trm5
2010-03-10 Christian Urban merged
2010-03-10 Christian Urban almost done with showing the equivalence between old and new alpha-equivalence (one subgoal remaining)
2010-03-10 Cezary Kaliszyk alpha_equivp for trm5
2010-03-10 Cezary Kaliszyk Undoing mistakenly committed parser experiments.
2010-03-10 Cezary Kaliszyk alpha_eqvt for recursive term1.
2010-03-10 Cezary Kaliszyk Looking at alpha_eqvt for term5, not much progress.
2010-03-10 Cezary Kaliszyk Reordered examples in Test.
2010-03-10 Cezary Kaliszyk Allows multiple bindings with same lhs.
2010-03-10 Cezary Kaliszyk Linked parser to fv and alpha.
2010-03-10 Cezary Kaliszyk merge
2010-03-10 Cezary Kaliszyk A minor fix for shallow binders. LF works again.
2010-03-10 Christian Urban merged
2010-03-10 Christian Urban parser produces ordered bn-fun information
2010-03-10 Cezary Kaliszyk Testing equalities in trm5, all seems good.
2010-03-10 Cezary Kaliszyk Fv&Alpha seem to work.
2010-03-10 Cezary Kaliszyk include alpha in the definitions.
2010-03-10 Cezary Kaliszyk Filled the algorithm for alpha_bn_arg
2010-03-10 Cezary Kaliszyk rhs of alpha_bn, and template for the arguments.
2010-03-10 Cezary Kaliszyk alpha_bn_constr template
2010-03-10 Cezary Kaliszyk exported template for alpha_bn
2010-03-10 Cezary Kaliszyk merge
2010-03-10 Cezary Kaliszyk Use alpha_bns in normal alpha defs.
2010-03-10 Cezary Kaliszyk alpha_bn_frees
2010-03-09 Christian Urban merged
2010-03-09 Christian Urban added bn-information, but it is not yet ordered according to the dts
2010-03-09 Cezary Kaliszyk Separate lists for separate constructors, to match bn_eqs.
2010-03-09 Cezary Kaliszyk All examples should work.
2010-03-09 Cezary Kaliszyk Fix to get old alpha.
2010-03-09 Cezary Kaliszyk Separate primrecs in Fv.
2010-03-09 Cezary Kaliszyk A version of Fv that takes into account recursive and non-recursive bindings.
2010-03-09 Cezary Kaliszyk Trying to prove that old alpha is the same as new recursive one. Lets still to do.
2010-03-09 Cezary Kaliszyk fv_bi and alpha_bi
2010-03-09 Christian Urban merged
2010-03-09 Christian Urban added first test about new compat
2010-03-09 Cezary Kaliszyk fv_compat
2010-03-09 Christian Urban added another compat example
2010-03-08 Christian Urban added a test-file for compatibility
2010-03-08 Christian Urban added compat definitions to some examples
2010-03-08 Cezary Kaliszyk Proper recognition of atoms and atom sets.
2010-03-08 Christian Urban deleted comments about "weird"
2010-03-08 Christian Urban merged
2010-03-08 Christian Urban updated to new Isabelle
2010-03-08 Cezary Kaliszyk Term5 written as nominal_datatype is the recursive let.
2010-03-08 Cezary Kaliszyk With restricted_nominal=1, exp7 and exp8 work. Not sure about proving bn_rsp there.
2010-03-08 Cezary Kaliszyk More fine-grained nominal restriction for debugging.
2010-03-08 Cezary Kaliszyk Fix permutation addition.
2010-03-08 Cezary Kaliszyk Update the comments
2010-03-08 Cezary Kaliszyk Gather bindings with same binder, and generate only one permutation for them.
2010-03-08 Cezary Kaliszyk Undo effects of simp.
2010-03-07 Christian Urban merged
2010-03-07 Christian Urban updated to renamings in Isabelle
2010-03-04 Christian Urban merged
2010-03-04 Christian Urban merged
2010-03-04 Christian Urban more proofs in Abs and work on Core Haskell
2010-03-03 Christian Urban added a lemma that permutations can be represented as sums of swapping
2010-03-05 Cezary Kaliszyk Still unable to show supp=fv for let with one existential.
2010-03-05 Cezary Kaliszyk Ported LF to the parser interface.
2010-03-05 Cezary Kaliszyk merge
2010-03-05 Cezary Kaliszyk Lift fv and bn eqvts; no need to lift alpha_eqvt.
2010-03-05 Cezary Kaliszyk Not much progress about the single existential let case.
2010-03-05 Cezary Kaliszyk Fixed LF for one quantifier over 2 premises.
2010-03-05 Cezary Kaliszyk Trying to fix the proofs for the single existential... So far failed.
2010-03-04 Cezary Kaliszyk Lift distinct.
2010-03-04 Cezary Kaliszyk Added lifting of pseudo-injectivity, commented out the code again and enabled the weird examples.
2010-03-04 Cezary Kaliszyk Lift BV,FV,Permutations and injection :).
2010-03-04 Cezary Kaliszyk Comment out Weird and Phd until we have an idea how to handle multiple permutations. Transp that works for multiple existentials.
2010-03-04 Cezary Kaliszyk A version that just leaves the supp/\supp goal. Obviously not true.
2010-03-04 Cezary Kaliszyk Prove symp and transp of weird without the supp /\ supp = {} assumption.
2010-03-03 Cezary Kaliszyk merge
2010-03-03 Cezary Kaliszyk Experiments with proving weird transp
2010-03-03 Cezary Kaliszyk Code for solving symp goals with multiple existentials.
2010-03-03 Cezary Kaliszyk reflp for multiple quantifiers.
2010-03-03 Christian Urban fixed mess in Test.thy
2010-03-03 Cezary Kaliszyk Fix eqvt for multiple quantifiers.
2010-03-03 Christian Urban only tuned
2010-03-03 Christian Urban merged
2010-03-03 Christian Urban start of paper - does not compile yet
2010-03-03 Christian Urban added ACM style file for ICFP
2010-03-03 Cezary Kaliszyk weird eqvt
2010-03-03 Cezary Kaliszyk Add the supp intersection conditions.
2010-03-02 Cezary Kaliszyk Comment out the part that does not work with 2 quantifiers.
2010-03-02 Cezary Kaliszyk Fixes for the fv problem and alpha problem.
2010-03-02 Christian Urban merged
2010-03-02 Christian Urban preliinary test about alpha-weirdo
2010-03-02 Christian Urban Another problem with permutations in alpha and possibly also in fv
2010-03-02 Christian Urban potential problem with the phd-example, where two permutations are generated, but only one is used
2010-03-02 Cezary Kaliszyk Some tests around Term4. Not sure how to fix the generated fv function.
2010-03-02 Cezary Kaliszyk merge
2010-03-02 Cezary Kaliszyk Porting from Lift to Parser; until defining the Quotient type.
2010-03-02 Cezary Kaliszyk Add image_eqvt and atom_eqvt to eqvt bases.
2010-03-02 Cezary Kaliszyk Include the raw eqvt lemmas.
2010-03-02 Christian Urban merged
2010-03-02 Christian Urban added some more examples from Peter Sewell's bestiary
2010-03-02 Cezary Kaliszyk merge
2010-03-02 Cezary Kaliszyk Minor
(0) -1000 -192 +192 +1000 tip