2010-03-17 |
Christian Urban |
added partial proof of supp for type schemes
|
file |
diff |
annotate
|
2010-03-17 |
Cezary Kaliszyk |
Fix in alpha; support of the recursive Let works :)
|
file |
diff |
annotate
|
2010-03-17 |
Cezary Kaliszyk |
The recursive supp just has one equation too much.
|
file |
diff |
annotate
|
2010-03-17 |
Christian Urban |
commented out examples that should not work; but for example type-scheme example should work
|
file |
diff |
annotate
|
2010-03-17 |
Christian Urban |
added another supp-proof for the non-recursive case
|
file |
diff |
annotate
|
2010-03-16 |
Christian Urban |
added the final unfolded result
|
file |
diff |
annotate
|
2010-03-16 |
Christian Urban |
merge and proof of support for non-recursive case
|
file |
diff |
annotate
|
2010-03-16 |
Cezary Kaliszyk |
alpha_bn doesn't need the permutation in non-recursive case.
|
file |
diff |
annotate
|
2010-03-16 |
Cezary Kaliszyk |
FV_bn generated for recursive functions as well, and used in main fv for bindings.
|
file |
diff |
annotate
|
2010-03-16 |
Cezary Kaliszyk |
The proof in 'Test' gets simpler.
|
file |
diff |
annotate
|
2010-03-15 |
Christian Urban |
merged (confirmed to work with Isabelle from 6th March)
|
file |
diff |
annotate
|
2010-03-15 |
Christian Urban |
proof for support when bn-function is present, but fb_function is empty
|
file |
diff |
annotate
|
2010-03-15 |
Cezary Kaliszyk |
fv_eqvt_cheat no longer needed.
|
file |
diff |
annotate
|
2010-03-15 |
Cezary Kaliszyk |
derive "inducts" from "induct" instead of lifting again is much faster.
|
file |
diff |
annotate
|
2010-03-15 |
Cezary Kaliszyk |
cheat_alpha_eqvt no longer needed; the proofs work.
|
file |
diff |
annotate
|
2010-03-15 |
Cezary Kaliszyk |
Use eqvt.
|
file |
diff |
annotate
|
2010-03-15 |
Christian Urban |
added an eqvt-proof for bi
|
file |
diff |
annotate
|
2010-03-13 |
Christian Urban |
started supp-fv proofs (is going to work)
|
file |
diff |
annotate
|
2010-03-11 |
Cezary Kaliszyk |
Show that the new types are in finite support typeclass.
|
file |
diff |
annotate
|
2010-03-11 |
Cezary Kaliszyk |
With the 4 cheats, all examples fully lift.
|
file |
diff |
annotate
|
2010-03-11 |
Cezary Kaliszyk |
Lifting constants.
|
file |
diff |
annotate
|
2010-03-10 |
Cezary Kaliszyk |
Reordered examples in Test.
|
file |
diff |
annotate
|
2010-03-10 |
Cezary Kaliszyk |
Linked parser to fv and alpha.
|
file |
diff |
annotate
|
2010-03-10 |
Christian Urban |
parser produces ordered bn-fun information
|
file |
diff |
annotate
|
2010-03-09 |
Christian Urban |
added bn-information, but it is not yet ordered according to the dts
|
file |
diff |
annotate
|
2010-03-09 |
Cezary Kaliszyk |
All examples should work.
|
file |
diff |
annotate
|
2010-03-08 |
Christian Urban |
added a test-file for compatibility
|
file |
diff |
annotate
|
2010-03-08 |
Christian Urban |
added compat definitions to some examples
|
file |
diff |
annotate
|
2010-03-08 |
Christian Urban |
deleted comments about "weird"
|
file |
diff |
annotate
|
2010-03-08 |
Cezary Kaliszyk |
With restricted_nominal=1, exp7 and exp8 work. Not sure about proving bn_rsp there.
|
file |
diff |
annotate
|
2010-03-07 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2010-03-04 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2010-03-04 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2010-03-04 |
Christian Urban |
more proofs in Abs and work on Core Haskell
|
file |
diff |
annotate
|
2010-03-04 |
Cezary Kaliszyk |
Lift distinct.
|
file |
diff |
annotate
|
2010-03-04 |
Cezary Kaliszyk |
Added lifting of pseudo-injectivity, commented out the code again and enabled the weird examples.
|
file |
diff |
annotate
|
2010-03-04 |
Cezary Kaliszyk |
Lift BV,FV,Permutations and injection :).
|
file |
diff |
annotate
|
2010-03-04 |
Cezary Kaliszyk |
A version that just leaves the supp/\supp goal. Obviously not true.
|
file |
diff |
annotate
|
2010-03-04 |
Cezary Kaliszyk |
Prove symp and transp of weird without the supp /\ supp = {} assumption.
|
file |
diff |
annotate
|
2010-03-03 |
Cezary Kaliszyk |
merge
|
file |
diff |
annotate
|
2010-03-03 |
Cezary Kaliszyk |
Experiments with proving weird transp
|
file |
diff |
annotate
|
2010-03-03 |
Christian Urban |
fixed mess in Test.thy
|
file |
diff |
annotate
|
2010-03-03 |
Cezary Kaliszyk |
Fix eqvt for multiple quantifiers.
|
file |
diff |
annotate
|
2010-03-03 |
Christian Urban |
only tuned
|
file |
diff |
annotate
|
2010-03-03 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2010-03-03 |
Christian Urban |
added ACM style file for ICFP
|
file |
diff |
annotate
|
2010-03-03 |
Cezary Kaliszyk |
weird eqvt
|
file |
diff |
annotate
|
2010-03-02 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2010-03-02 |
Christian Urban |
preliinary test about alpha-weirdo
|
file |
diff |
annotate
|
2010-03-02 |
Christian Urban |
Another problem with permutations in alpha and possibly also in fv
|
file |
diff |
annotate
|
2010-03-02 |
Christian Urban |
potential problem with the phd-example, where two permutations are generated, but only one is used
|
file |
diff |
annotate
|
2010-03-02 |
Cezary Kaliszyk |
merge
|
file |
diff |
annotate
|
2010-03-02 |
Cezary Kaliszyk |
Porting from Lift to Parser; until defining the Quotient type.
|
file |
diff |
annotate
|
2010-03-02 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2010-03-02 |
Christian Urban |
added some more examples from Peter Sewell's bestiary
|
file |
diff |
annotate
|
2010-03-02 |
Cezary Kaliszyk |
Working bv_eqvt
|
file |
diff |
annotate
|
2010-03-02 |
Cezary Kaliszyk |
Change type schemes to name set.
|
file |
diff |
annotate
|
2010-03-02 |
Cezary Kaliszyk |
Length fix for nested recursions.
|
file |
diff |
annotate
|
2010-03-02 |
Christian Urban |
most tests work - the ones that do not I commented out
|
file |
diff |
annotate
|
2010-03-02 |
Cezary Kaliszyk |
merge
|
file |
diff |
annotate
|
2010-03-02 |
Cezary Kaliszyk |
Add a check of fv_functions.
|
file |
diff |
annotate
|
2010-03-02 |
Christian Urban |
some tuning
|
file |
diff |
annotate
|
2010-03-02 |
Cezary Kaliszyk |
Link calls to Raw permutations, FV definition and alpha_definition into the parser.
|
file |
diff |
annotate
|
2010-03-01 |
Christian Urban |
modified for new binding format - hope it is the intended one
|
file |
diff |
annotate
|
2010-03-01 |
Christian Urban |
slight simplification of the raw-decl generation
|
file |
diff |
annotate
|
2010-03-01 |
Christian Urban |
added example from my phd
|
file |
diff |
annotate
|
2010-02-27 |
Christian Urban |
streamlined parser
|
file |
diff |
annotate
|
2010-02-26 |
Christian Urban |
generated the "binding list" from the input; at the moment it is only printed out as tracing; does not yet include the "bind itself binders"
|
file |
diff |
annotate
|
2010-02-25 |
Christian Urban |
added ott-example about Leroy96
|
file |
diff |
annotate
|
2010-02-25 |
Christian Urban |
first attempt to make sense out of the core-haskell definition
|
file |
diff |
annotate
|
2010-02-25 |
Christian Urban |
added IsaMakefile...but so far included only a test for the parser
|
file |
diff |
annotate
|
2010-02-25 |
Christian Urban |
moved Nominal to "toplevel"
|
file |
diff |
annotate
| base
|