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.
Updated Term1, including statement of strong induction.
2010-03-17, by Cezary Kaliszyk
Proper compose_sym2
2010-03-17, by Cezary Kaliszyk
merged
2010-03-17, by Christian Urban
temporarily disabled tests in Nominal/ROOT
2010-03-17, by Christian Urban
made paper to compile
2010-03-17, by Christian Urban
added partial proof for the strong induction principle
2010-03-17, by Christian Urban
Trying to find a compose lemma for 2 arguments.
2010-03-17, by Cezary Kaliszyk
merge
2010-03-17, by Cezary Kaliszyk
cheat_alpha_eqvt no longer needed. Cleaned the tracing messages.
2010-03-17, by Cezary Kaliszyk
merged
2010-03-17, by Christian Urban
added proof of supp/fv for type schemes
2010-03-17, by Christian Urban
Updated Type Schemes to automatic lifting. One goal is not true because of the restriction.
2010-03-17, by Cezary Kaliszyk
Remove Term5a, since it is now identical to Term5.
2010-03-17, by Cezary Kaliszyk
merge
2010-03-17, by Cezary Kaliszyk
Finished all proofs in Term5 and Term5n.
2010-03-17, by Cezary Kaliszyk
added partial proof of supp for type schemes
2010-03-17, by Christian Urban
Fix in alpha; support of the recursive Let works :)
2010-03-17, by Cezary Kaliszyk
The recursive supp just has one equation too much.
2010-03-17, by Cezary Kaliszyk
Fix for the change of alpha_gen.
2010-03-17, by Cezary Kaliszyk
merge
2010-03-17, by Cezary Kaliszyk
Generate compound FV and Alpha for recursive bindings.
2010-03-17, by Cezary Kaliszyk
Lifting theorems with compound fv and compound alpha.
2010-03-17, by Cezary Kaliszyk
commented out examples that should not work; but for example type-scheme example should work
2010-03-17, by Christian Urban
added another supp-proof for the non-recursive case
2010-03-17, by Christian Urban
Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
2010-03-16, by Cezary Kaliszyk
merge
2010-03-16, by Cezary Kaliszyk
The old recursive alpha works fine.
2010-03-16, by Cezary Kaliszyk
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
less
more
|
(0)
-1000
-120
+120
+1000
tip