Mercurial
Mercurial
>
hg
>
nominal2
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
help
less
more
|
(0)
-1000
-120
+120
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 another example which seems difficult to define
2011-07-05, by Christian Urban
added a tactic "all_trivials" which simplifies all trivial constructor cases and leaves the others untouched.
2011-07-05, by Christian Urban
merged
2011-07-05, by Christian Urban
all FCB lemmas
2011-07-05, by Christian Urban
exported various FCB-lemmas to a separate file
2011-07-05, by Christian Urban
Express trans_db with Option.map and Option.bind. Possibly mbind is a copy of bind?
2011-07-05, by Cezary Kaliszyk
Define a version of aux only for same binders. Completeness is fine.
2011-07-05, by Cezary Kaliszyk
Move If / Let with 'True' to the end of Lambda
2011-07-05, by Cezary Kaliszyk
merged
2011-07-04, by Christian Urban
tuned
2011-07-04, by Christian Urban
added an example that recurses over two arguments; the interesting proof-obligation is not yet done
2011-07-04, by Christian Urban
Let with a different invariant; not true.
2011-07-04, by Cezary Kaliszyk
Add non-working Lambda_F_T using FCB2
2011-07-03, by Cezary Kaliszyk
Added non-working CPS3 using FCB2
2011-07-03, by Cezary Kaliszyk
Change CPS1 to FCB2
2011-07-03, by Cezary Kaliszyk
Did the proofs of height and subst for Let with list-like binders. Having apply_assns allows proving things by alpha_bn
2011-07-02, by Cezary Kaliszyk
side-by-side tests of lets with single assignment; deep-binder case works if the recursion is avoided using an auxiliary function
2011-07-02, by Christian Urban
Exhaust Issue
2011-07-01, by Cezary Kaliszyk
clarified a sentence
2011-06-30, by Christian Urban
more code refactoring
2011-06-30, by Christian Urban
combined distributed data for alpha in alpha_result (partially done)
2011-06-29, by Christian Urban
moved Classical and Let temporarily into a section where "sorry" is allowed; this makes all test go through
2011-06-29, by Christian Urban
added a warning if a theorem is already declared as equivariant
2011-06-29, by Christian Urban
merged
2011-06-29, by Christian Urban
Prove bn injectivity and experiment more with Let
2011-06-29, by Cezary Kaliszyk
some experiments
2011-06-29, by Christian Urban
trying new fcb in let/subst
2011-06-28, by Cezary Kaliszyk
Leftover only inj and eqvt
2011-06-28, by Cezary Kaliszyk
eapply fcb ok
2011-06-28, by Cezary Kaliszyk
Removed Inl and Inr
2011-06-28, by Cezary Kaliszyk
relaxed type in fcb
2011-06-28, by Christian Urban
fcb with explicit bn function
2011-06-28, by Christian Urban
added let-rec example
2011-06-28, by Christian Urban
Experiments with res
2011-06-28, by Cezary Kaliszyk
proved the fcb also for sets (no restriction yet)
2011-06-28, by Christian Urban
copied all work to Lambda.thy; had to derive a special version of fcb1 for concrete atom
2011-06-28, by Christian Urban
streamlined the fcb-proof and made fcb1 a special case of fcb
2011-06-27, by Christian Urban
completed proof in Classical; the fcb lemma works for any list of atoms (despite what was written earlier)
2011-06-27, by Christian Urban
fcb for multible (list) binders; at the moment all of them have to have the same sort (at-class); this should also work for set binders, but not yet for restriction.
2011-06-27, by Christian Urban
renamed ds to dset (disagreement set)
2011-06-27, by Christian Urban
added small lemma about disagreement set
2011-06-27, by Christian Urban
merge
2011-06-27, by Cezary Kaliszyk
New-style fcb for multiple binders.
2011-06-27, by Cezary Kaliszyk
equality of lst_binder and a few helper lemmas
2011-06-27, by Cezary Kaliszyk
only one of the fcb precondistions are needed (probably the same with the perm-conditions)
2011-06-26, by Christian Urban
another change to the fcb2; this is needed in order to get all proofs through in Lambda.thy
2011-06-26, by Christian Urban
did all cases, except the multiple binder case
2011-06-25, by Christian Urban
an alternative FCB for Abs_lst1; seems simpler but not as simple as I thought; not sure whether it generalises to multiple binders.
2011-06-25, by Christian Urban
except for the interated binder case, finished definition in Calssical.thy
2011-06-24, by Christian Urban
Make examples work with non-precompiled image
2011-06-24, by Cezary Kaliszyk
Remove Lambda_add.thy
2011-06-24, by Cezary Kaliszyk
The examples in Lambda_add can be defined by nominal_function directly
2011-06-24, by Cezary Kaliszyk
Theory name changes for JEdit
2011-06-24, by Cezary Kaliszyk
More usual names for substitution properties
2011-06-24, by Cezary Kaliszyk
Second Fixed Point Theorem
2011-06-24, by Cezary Kaliszyk
Speed-up the completeness proof.
2011-06-24, by Cezary Kaliszyk
the simplifier can simplify "sort (atom a)" if a is a concrete atom type declared with atom_decl
2011-06-23, by Christian Urban
added file
2011-06-23, by Christian Urban
expanded the example
2011-06-23, by Christian Urban
fixed nasty bug with type variables in nominal_datatypes; this included to be careful with the output of the inductive and function package
2011-06-23, by Christian Urban
tuned
2011-06-22, by Christian Urban
deleted some dead code
2011-06-22, by Christian Urban
some rudimentary infrastructure for storing data about nominal datatypes
2011-06-22, by Christian Urban
constants with the same names
2011-06-22, by Cezary Kaliszyk
Quotients/TODO addtion
2011-06-22, by Cezary Kaliszyk
Minor
2011-06-21, by Cezary Kaliszyk
merge
2011-06-21, by Cezary Kaliszyk
spelling
2011-06-21, by Cezary Kaliszyk
merge
2011-06-20, by Cezary Kaliszyk
Abs_set_fcb
2011-06-20, by Cezary Kaliszyk
function for let-rec
2011-06-20, by Cezary Kaliszyk
TODO/minor
2011-06-20, by Cezary Kaliszyk
Move lst_fcb to Nominal2_Abs
2011-06-20, by Cezary Kaliszyk
More minor TODOs
2011-06-20, by Cezary Kaliszyk
Update TODO
2011-06-20, by Cezary Kaliszyk
Let/minor
2011-06-20, by Cezary Kaliszyk
Update Quotient/TODO and remove some attic code
2011-06-20, by Cezary Kaliszyk
merge
2011-06-19, by Cezary Kaliszyk
little on cps2
2011-06-19, by Cezary Kaliszyk
got rid of the boolean flag in the raw_equivariance function
2011-06-16, by Christian Urban
Fix
2011-06-16, by Cezary Kaliszyk
merge
2011-06-16, by Cezary Kaliszyk
CPS3 can be defined with eqvt_rhs.
2011-06-16, by Cezary Kaliszyk
moved for the moment CPS translations into the example directory
2011-06-16, by Christian Urban
merged
2011-06-16, by Christian Urban
added eqvt_at and invariant for boths sides of the equations
2011-06-16, by Christian Urban
Added the CPS translation experiments. CPS1 comes with all the proofs, CPS2,3 just have the function and need eqvt_rhs to finish the obligations.
2011-06-16, by Cezary Kaliszyk
added a test that every function must be of pt-sort
2011-06-16, by Christian Urban
all tests work again
2011-06-16, by Christian Urban
added size-lemmas to simplifier; as a result termination can be proved by the standard lexicographic_order method
2011-06-15, by Christian Urban
added an abstract
2011-06-15, by Christian Urban
added a stub for function paper; "isabelle make fnpaper"
2011-06-15, by Christian Urban
merge
2011-06-15, by Cezary Kaliszyk
one TODO and one Problem?
2011-06-15, by Cezary Kaliszyk
merge
2011-06-15, by Cezary Kaliszyk
Some TODOs
2011-06-15, by Cezary Kaliszyk
merge
2011-06-15, by Cezary Kaliszyk
TypeSchemes work with 'default'.
2011-06-15, by Cezary Kaliszyk
tuned some proofs
2011-06-14, by Christian Urban
fixed the problem when giving a complex default-term; the fundef lemmas in Nominal_Base were not general enough
2011-06-14, by Christian Urban
tuned
2011-06-14, by Christian Urban
Move working examples before non-working ones
2011-06-10, by Cezary Kaliszyk
Optimized proofs and removed some garbage.
2011-06-10, by Cezary Kaliszyk
merge
2011-06-10, by Cezary Kaliszyk
Slightly modify fcb for list1 and put in common place.
2011-06-10, by Cezary Kaliszyk
Experiments with Let
2011-06-10, by Cezary Kaliszyk
Eval can be defined with additional freshness
2011-06-09, by Cezary Kaliszyk
Minor simplification
2011-06-09, by Cezary Kaliszyk
abs_res_fcb will be enough to finish the multiple-recursive proof, if we have a working 'default'.
2011-06-09, by Cezary Kaliszyk
More experiments with 'default'
2011-06-09, by Cezary Kaliszyk
Finished the proof with the invariant
2011-06-08, by Cezary Kaliszyk
Issue with 'default'
2011-06-08, by Cezary Kaliszyk
merged
2011-06-08, by Christian Urban
merged
2011-06-08, by Christian Urban
using the option "default" the function package allows one to give an explicit default value
2011-06-08, by Christian Urban
Simpler proof of TypeSchemes/substs
2011-06-08, by Cezary Kaliszyk
Simplify fcb_res
2011-06-08, by Cezary Kaliszyk
FCB for res binding and simplified proof of subst for type schemes
2011-06-08, by Cezary Kaliszyk
Simplify ln-trans proof
2011-06-08, by Cezary Kaliszyk
cbvs can be easily defined without an invariant
2011-06-08, by Cezary Kaliszyk
less
more
|
(0)
-1000
-120
+120
tip