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