2010-03-27 |
Cezary Kaliszyk |
Fv/Alpha now takes into account Alpha_Type given from the parser.
|
file |
diff |
annotate
|
2010-03-27 |
Cezary Kaliszyk |
Minor cleaning.
|
file |
diff |
annotate
|
2010-03-26 |
Cezary Kaliszyk |
Fixed renamings.
|
file |
diff |
annotate
|
2010-03-26 |
Cezary Kaliszyk |
Removed remaining cheats + some cleaning.
|
file |
diff |
annotate
|
2010-03-26 |
Cezary Kaliszyk |
Removed another cheat and cleaned the code a bit.
|
file |
diff |
annotate
|
2010-03-25 |
Cezary Kaliszyk |
Proper bn_rsp, for bn functions calling each other.
|
file |
diff |
annotate
|
2010-03-25 |
Cezary Kaliszyk |
Gathering things to prove by induction together; removed cheat_bn_eqvt.
|
file |
diff |
annotate
|
2010-03-24 |
Cezary Kaliszyk |
Support proof modification for Core Haskell.
|
file |
diff |
annotate
|
2010-03-24 |
Cezary Kaliszyk |
Compute Fv for non-recursive bn functions calling other bn functions
|
file |
diff |
annotate
|
2010-03-23 |
Cezary Kaliszyk |
Parsing bn functions that call other bn functions and transmitting this information to fv/alpha.
|
file |
diff |
annotate
|
2010-03-23 |
Cezary Kaliszyk |
Modification to Core Haskell to make it accepted with an empty binding function.
|
file |
diff |
annotate
|
2010-03-22 |
Cezary Kaliszyk |
equivp_cheat can be removed for all one-permutation examples.
|
file |
diff |
annotate
|
2010-03-20 |
Cezary Kaliszyk |
Build alpha-->alphabn implications
|
file |
diff |
annotate
|
2010-03-20 |
Cezary Kaliszyk |
Prove reflp for all relations.
|
file |
diff |
annotate
|
2010-03-19 |
Cezary Kaliszyk |
Automatically derive support for datatypes with at-most one binding per constructor.
|
file |
diff |
annotate
|
2010-03-19 |
Cezary Kaliszyk |
Use fs typeclass in showing finite support + some cheat cleaning.
|
file |
diff |
annotate
|
2010-03-19 |
Cezary Kaliszyk |
The nominal infrastructure for fset. 'fs' missing, but not needed so far.
|
file |
diff |
annotate
|
2010-03-18 |
Cezary Kaliszyk |
Continued description of alpha.
|
file |
diff |
annotate
|
2010-03-18 |
Cezary Kaliszyk |
First part of the description of alpha_ty.
|
file |
diff |
annotate
|
2010-03-18 |
Cezary Kaliszyk |
Description of generation of alpha_bn.
|
file |
diff |
annotate
|
2010-03-18 |
Cezary Kaliszyk |
Added fv,bn,distinct,perm to the simplifier.
|
file |
diff |
annotate
|
2010-03-18 |
Cezary Kaliszyk |
Simplified the description.
|
file |
diff |
annotate
|
2010-03-18 |
Cezary Kaliszyk |
Update the description of the generation of fv function.
|
file |
diff |
annotate
|
2010-03-18 |
Cezary Kaliszyk |
Rename bound variables + minor cleaning.
|
file |
diff |
annotate
|
2010-03-17 |
Cezary Kaliszyk |
Proper compose_sym2
|
file |
diff |
annotate
|
2010-03-17 |
Cezary Kaliszyk |
Trying to find a compose lemma for 2 arguments.
|
file |
diff |
annotate
|
2010-03-17 |
Cezary Kaliszyk |
cheat_alpha_eqvt no longer needed. Cleaned the tracing messages.
|
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 |
Generate compound FV and Alpha for recursive bindings.
|
file |
diff |
annotate
|
2010-03-16 |
Cezary Kaliszyk |
Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
|
file |
diff |
annotate
|
2010-03-16 |
Cezary Kaliszyk |
The old recursive alpha works fine.
|
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 |
Removed pi o bn = bn' assumption in alpha
|
file |
diff |
annotate
|
2010-03-11 |
Cezary Kaliszyk |
Do not fail if the finite support proof fails.
|
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 |
mk_supports_eq and supports_tac.
|
file |
diff |
annotate
|
2010-03-11 |
Cezary Kaliszyk |
Remove "_raw" from lifted theorems.
|
file |
diff |
annotate
|
2010-03-11 |
Cezary Kaliszyk |
Proper error message.
|
file |
diff |
annotate
|
2010-03-11 |
Cezary Kaliszyk |
Remove tracing from fv/alpha.
|
file |
diff |
annotate
|
2010-03-10 |
Cezary Kaliszyk |
Allows multiple bindings with same lhs.
|
file |
diff |
annotate
|
2010-03-10 |
Cezary Kaliszyk |
A minor fix for shallow binders. LF works again.
|
file |
diff |
annotate
|
2010-03-10 |
Cezary Kaliszyk |
Fv&Alpha seem to work.
|
file |
diff |
annotate
|
2010-03-10 |
Cezary Kaliszyk |
include alpha in the definitions.
|
file |
diff |
annotate
|
2010-03-10 |
Cezary Kaliszyk |
Filled the algorithm for alpha_bn_arg
|
file |
diff |
annotate
|
2010-03-10 |
Cezary Kaliszyk |
rhs of alpha_bn, and template for the arguments.
|
file |
diff |
annotate
|
2010-03-10 |
Cezary Kaliszyk |
alpha_bn_constr template
|
file |
diff |
annotate
|
2010-03-10 |
Cezary Kaliszyk |
exported template for alpha_bn
|
file |
diff |
annotate
|
2010-03-10 |
Cezary Kaliszyk |
Use alpha_bns in normal alpha defs.
|
file |
diff |
annotate
|
2010-03-10 |
Cezary Kaliszyk |
alpha_bn_frees
|
file |
diff |
annotate
|
2010-03-09 |
Cezary Kaliszyk |
Separate lists for separate constructors, to match bn_eqs.
|
file |
diff |
annotate
|
2010-03-09 |
Cezary Kaliszyk |
Fix to get old alpha.
|
file |
diff |
annotate
|
2010-03-09 |
Cezary Kaliszyk |
Separate primrecs in Fv.
|
file |
diff |
annotate
|
2010-03-09 |
Cezary Kaliszyk |
A version of Fv that takes into account recursive and non-recursive bindings.
|
file |
diff |
annotate
|
2010-03-08 |
Cezary Kaliszyk |
Proper recognition of atoms and atom sets.
|
file |
diff |
annotate
|
2010-03-08 |
Cezary Kaliszyk |
Term5 written as nominal_datatype is the recursive let.
|
file |
diff |
annotate
|
2010-03-08 |
Cezary Kaliszyk |
Fix permutation addition.
|
file |
diff |
annotate
|
2010-03-08 |
Cezary Kaliszyk |
Update the comments
|
file |
diff |
annotate
|
2010-03-08 |
Cezary Kaliszyk |
Gather bindings with same binder, and generate only one permutation for them.
|
file |
diff |
annotate
|
2010-03-04 |
Cezary Kaliszyk |
Comment out Weird and Phd until we have an idea how to handle multiple permutations. Transp that works for multiple existentials.
|
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 |
Code for solving symp goals with multiple existentials.
|
file |
diff |
annotate
|
2010-03-03 |
Cezary Kaliszyk |
reflp for multiple quantifiers.
|
file |
diff |
annotate
|
2010-03-03 |
Cezary Kaliszyk |
Add the supp intersection conditions.
|
file |
diff |
annotate
|
2010-03-02 |
Cezary Kaliszyk |
Fixes for the fv problem and alpha problem.
|
file |
diff |
annotate
|
2010-03-02 |
Cezary Kaliszyk |
Moving wrappers out of Lift.
|
file |
diff |
annotate
|
2010-03-02 |
Cezary Kaliszyk |
More fixes for new alpha, the whole lift script should now work again.
|
file |
diff |
annotate
|
2010-03-02 |
Cezary Kaliszyk |
Length fix for nested recursions.
|
file |
diff |
annotate
|
2010-03-02 |
Cezary Kaliszyk |
Fix equivp.
|
file |
diff |
annotate
|
2010-03-01 |
Cezary Kaliszyk |
The new alpha-equivalence and testing in Trm2 and Trm5.
|
file |
diff |
annotate
|
2010-02-26 |
Cezary Kaliszyk |
Permutation and FV_Alpha interface change.
|
file |
diff |
annotate
|
2010-02-25 |
Christian Urban |
moved Nominal to "toplevel"
|
file |
diff |
annotate
| base
|