Mercurial
Mercurial
>
hg
>
nominal2
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
help
less
more
|
(0)
-1000
-120
+120
+1000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
added the final unfolded result
2010-03-16, by Christian Urban
merge and proof of support for non-recursive case
2010-03-16, by Christian Urban
Added Term5 non-recursive. The bug is there only for the recursive case.
2010-03-16, by Cezary Kaliszyk
Alpha is wrong.
2010-03-16, by Cezary Kaliszyk
alpha_bn doesn't need the permutation in non-recursive case.
2010-03-16, by Cezary Kaliszyk
alpha5_transp and equivp
2010-03-16, by Cezary Kaliszyk
alpha5_symp proved.
2010-03-16, by Cezary Kaliszyk
FV_bn generated for recursive functions as well, and used in main fv for bindings.
2010-03-16, by Cezary Kaliszyk
The proof in 'Test' gets simpler.
2010-03-16, by Cezary Kaliszyk
Removed pi o bn = bn' assumption in alpha
2010-03-16, by Cezary Kaliszyk
merged (confirmed to work with Isabelle from 6th March)
2010-03-15, by Christian Urban
another synchronisation
2010-03-15, by Christian Urban
proof for support when bn-function is present, but fb_function is empty
2010-03-15, by Christian Urban
fv_eqvt_cheat no longer needed.
2010-03-15, by Cezary Kaliszyk
derive "inducts" from "induct" instead of lifting again is much faster.
2010-03-15, by Cezary Kaliszyk
build_eqvts works with recursive case if proper induction rule is used.
2010-03-15, by Cezary Kaliszyk
cheat_alpha_eqvt no longer needed; the proofs work.
2010-03-15, by Cezary Kaliszyk
LF works with new alpha...?
2010-03-15, by Cezary Kaliszyk
explicit flag "cheat_equivp"
2010-03-15, by Cezary Kaliszyk
Prove alpha_gen_compose_eqvt
2010-03-15, by Cezary Kaliszyk
Use eqvt.
2010-03-15, by Cezary Kaliszyk
added preliminary test version....but Test works now
2010-03-15, by Christian Urban
added an eqvt-proof for bi
2010-03-15, by Christian Urban
synchronised with main hg-repository; used add_typedef_global in nominal_atoms
2010-03-15, by Christian Urban
localised the typedef in Attic (requires new Isabelle)
2010-03-14, by Christian Urban
started supp-fv proofs (is going to work)
2010-03-13, by Christian Urban
Even with pattern simplified to a single clause, the supp equation doesn't seem true.
2010-03-12, by Cezary Kaliszyk
Still don't know how to prove supp=fv for simplest Let...
2010-03-12, by Cezary Kaliszyk
Do not fail if the finite support proof fails.
2010-03-11, by Cezary Kaliszyk
generalised the supp for atoms to all concrete atoms (not just names)
2010-03-11, by Christian Urban
support of atoms at the end of Abs.thy
2010-03-11, by Christian Urban
Trying to prove atom_image_fresh_swap
2010-03-11, by Cezary Kaliszyk
Finite_support proof no longer needed in LF.
2010-03-11, by Cezary Kaliszyk
Show that the new types are in finite support typeclass.
2010-03-11, by Cezary Kaliszyk
mk_supports_eq and supports_tac.
2010-03-11, by Cezary Kaliszyk
merge
2010-03-11, by Cezary Kaliszyk
Fixes for term1 for new alpha. Still not able to show support equations.
2010-03-11, by Cezary Kaliszyk
merged
2010-03-11, by Christian Urban
finally the proof that new and old alpha agree
2010-03-11, by Christian Urban
Remove "_raw" from lifted theorems.
2010-03-11, by Cezary Kaliszyk
looking at trm5_equivp
2010-03-11, by Cezary Kaliszyk
The cheats described explicitely.
2010-03-11, by Cezary Kaliszyk
The alpha5_eqvt tactic works if I manage to build the goal.
2010-03-11, by Cezary Kaliszyk
With the 4 cheats, all examples fully lift.
2010-03-11, by Cezary Kaliszyk
Lift alpha_bn_constants.
2010-03-11, by Cezary Kaliszyk
Lifting constants.
2010-03-11, by Cezary Kaliszyk
Proper error message.
2010-03-11, by Cezary Kaliszyk
Lifting constants works for all examples.
2010-03-11, by Cezary Kaliszyk
Remove tracing from fv/alpha.
2010-03-11, by Cezary Kaliszyk
Equivp working only on the standard alpha-equivalences.
2010-03-11, by Cezary Kaliszyk
explicit cheat_fv_eqvt
2010-03-11, by Cezary Kaliszyk
extract build_eqvts_tac.
2010-03-11, by Cezary Kaliszyk
build_eqvts no longer requires permutations.
2010-03-11, by Cezary Kaliszyk
Add explicit alpha_eqvt_cheat.
2010-03-11, by Cezary Kaliszyk
Export tactic out of alpha_eqvt.
2010-03-11, by Cezary Kaliszyk
merge
2010-03-10, by Cezary Kaliszyk
More tries about the proofs in trm5
2010-03-10, by Cezary Kaliszyk
merged
2010-03-10, by Christian Urban
almost done with showing the equivalence between old and new alpha-equivalence (one subgoal remaining)
2010-03-10, by Christian Urban
alpha_equivp for trm5
2010-03-10, by Cezary Kaliszyk
Undoing mistakenly committed parser experiments.
2010-03-10, by Cezary Kaliszyk
alpha_eqvt for recursive term1.
2010-03-10, by Cezary Kaliszyk
Looking at alpha_eqvt for term5, not much progress.
2010-03-10, by Cezary Kaliszyk
Reordered examples in Test.
2010-03-10, by Cezary Kaliszyk
Allows multiple bindings with same lhs.
2010-03-10, by Cezary Kaliszyk
Linked parser to fv and alpha.
2010-03-10, by Cezary Kaliszyk
merge
2010-03-10, by Cezary Kaliszyk
A minor fix for shallow binders. LF works again.
2010-03-10, by Cezary Kaliszyk
merged
2010-03-10, by Christian Urban
parser produces ordered bn-fun information
2010-03-10, by Christian Urban
Testing equalities in trm5, all seems good.
2010-03-10, by Cezary Kaliszyk
Fv&Alpha seem to work.
2010-03-10, by Cezary Kaliszyk
include alpha in the definitions.
2010-03-10, by Cezary Kaliszyk
Filled the algorithm for alpha_bn_arg
2010-03-10, by Cezary Kaliszyk
rhs of alpha_bn, and template for the arguments.
2010-03-10, by Cezary Kaliszyk
alpha_bn_constr template
2010-03-10, by Cezary Kaliszyk
exported template for alpha_bn
2010-03-10, by Cezary Kaliszyk
merge
2010-03-10, by Cezary Kaliszyk
Use alpha_bns in normal alpha defs.
2010-03-10, by Cezary Kaliszyk
alpha_bn_frees
2010-03-10, by Cezary Kaliszyk
merged
2010-03-09, by Christian Urban
added bn-information, but it is not yet ordered according to the dts
2010-03-09, by Christian Urban
Separate lists for separate constructors, to match bn_eqs.
2010-03-09, by Cezary Kaliszyk
All examples should work.
2010-03-09, by Cezary Kaliszyk
Fix to get old alpha.
2010-03-09, by Cezary Kaliszyk
Separate primrecs in Fv.
2010-03-09, by Cezary Kaliszyk
A version of Fv that takes into account recursive and non-recursive bindings.
2010-03-09, by Cezary Kaliszyk
Trying to prove that old alpha is the same as new recursive one. Lets still to do.
2010-03-09, by Cezary Kaliszyk
fv_bi and alpha_bi
2010-03-09, by Cezary Kaliszyk
merged
2010-03-09, by Christian Urban
added first test about new compat
2010-03-09, by Christian Urban
fv_compat
2010-03-09, by Cezary Kaliszyk
added another compat example
2010-03-09, by Christian Urban
added a test-file for compatibility
2010-03-08, by Christian Urban
added compat definitions to some examples
2010-03-08, by Christian Urban
Proper recognition of atoms and atom sets.
2010-03-08, by Cezary Kaliszyk
deleted comments about "weird"
2010-03-08, by Christian Urban
merged
2010-03-08, by Christian Urban
updated to new Isabelle
2010-03-08, by Christian Urban
Term5 written as nominal_datatype is the recursive let.
2010-03-08, by Cezary Kaliszyk
With restricted_nominal=1, exp7 and exp8 work. Not sure about proving bn_rsp there.
2010-03-08, by Cezary Kaliszyk
More fine-grained nominal restriction for debugging.
2010-03-08, by Cezary Kaliszyk
Fix permutation addition.
2010-03-08, by Cezary Kaliszyk
Update the comments
2010-03-08, by Cezary Kaliszyk
Gather bindings with same binder, and generate only one permutation for them.
2010-03-08, by Cezary Kaliszyk
Undo effects of simp.
2010-03-08, by Cezary Kaliszyk
merged
2010-03-07, by Christian Urban
updated to renamings in Isabelle
2010-03-07, by Christian Urban
merged
2010-03-04, by Christian Urban
merged
2010-03-04, by Christian Urban
more proofs in Abs and work on Core Haskell
2010-03-04, by Christian Urban
added a lemma that permutations can be represented as sums of swapping
2010-03-03, by Christian Urban
Still unable to show supp=fv for let with one existential.
2010-03-05, by Cezary Kaliszyk
Ported LF to the parser interface.
2010-03-05, by Cezary Kaliszyk
merge
2010-03-05, by Cezary Kaliszyk
Lift fv and bn eqvts; no need to lift alpha_eqvt.
2010-03-05, by Cezary Kaliszyk
Not much progress about the single existential let case.
2010-03-05, by Cezary Kaliszyk
Fixed LF for one quantifier over 2 premises.
2010-03-05, by Cezary Kaliszyk
Trying to fix the proofs for the single existential... So far failed.
2010-03-05, by Cezary Kaliszyk
Lift distinct.
2010-03-04, by Cezary Kaliszyk
less
more
|
(0)
-1000
-120
+120
+1000
tip