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.
(0) -1000 -120 +120 +1000 tip