2010-03-17 |
Cezary Kaliszyk |
cheat_alpha_eqvt no longer needed. Cleaned the tracing messages.
|
file |
diff |
annotate
|
2010-03-17 |
Cezary Kaliszyk |
Lifting theorems with compound fv and compound alpha.
|
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 |
FV_bn generated for recursive functions as well, and used in main fv for bindings.
|
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 |
explicit flag "cheat_equivp"
|
file |
diff |
annotate
|
2010-03-13 |
Christian Urban |
started supp-fv proofs (is going to work)
|
file |
diff |
annotate
|
2010-03-12 |
Cezary Kaliszyk |
Still don't know how to prove supp=fv for simplest Let...
|
file |
diff |
annotate
|
2010-03-11 |
Cezary Kaliszyk |
Do not fail if the finite support proof fails.
|
file |
diff |
annotate
|
2010-03-11 |
Christian Urban |
support of atoms at the end of Abs.thy
|
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 |
Remove "_raw" from lifted theorems.
|
file |
diff |
annotate
|
2010-03-11 |
Cezary Kaliszyk |
The cheats described explicitely.
|
file |
diff |
annotate
|
2010-03-11 |
Cezary Kaliszyk |
With the 4 cheats, all examples fully lift.
|
file |
diff |
annotate
|
2010-03-11 |
Cezary Kaliszyk |
Lift alpha_bn_constants.
|
file |
diff |
annotate
|
2010-03-11 |
Cezary Kaliszyk |
Lifting constants.
|
file |
diff |
annotate
|
2010-03-11 |
Cezary Kaliszyk |
Lifting constants works for all examples.
|
file |
diff |
annotate
|
2010-03-11 |
Cezary Kaliszyk |
Equivp working only on the standard alpha-equivalences.
|
file |
diff |
annotate
|
2010-03-11 |
Cezary Kaliszyk |
explicit cheat_fv_eqvt
|
file |
diff |
annotate
|
2010-03-11 |
Cezary Kaliszyk |
extract build_eqvts_tac.
|
file |
diff |
annotate
|
2010-03-11 |
Cezary Kaliszyk |
build_eqvts no longer requires permutations.
|
file |
diff |
annotate
|
2010-03-11 |
Cezary Kaliszyk |
Add explicit alpha_eqvt_cheat.
|
file |
diff |
annotate
|
2010-03-11 |
Cezary Kaliszyk |
Export tactic out of alpha_eqvt.
|
file |
diff |
annotate
|
2010-03-10 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2010-03-10 |
Christian Urban |
almost done with showing the equivalence between old and new alpha-equivalence (one subgoal remaining)
|
file |
diff |
annotate
|
2010-03-10 |
Cezary Kaliszyk |
Undoing mistakenly committed parser experiments.
|
file |
diff |
annotate
|
2010-03-10 |
Cezary Kaliszyk |
alpha_eqvt for recursive term1.
|
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 |
A version of Fv that takes into account recursive and non-recursive bindings.
|
file |
diff |
annotate
|
2010-03-08 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2010-03-08 |
Christian Urban |
updated to new Isabelle
|
file |
diff |
annotate
|
2010-03-08 |
Cezary Kaliszyk |
More fine-grained nominal restriction for debugging.
|
file |
diff |
annotate
|
2010-03-05 |
Cezary Kaliszyk |
Lift fv and bn eqvts; no need to lift alpha_eqvt.
|
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 |
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-03 |
Cezary Kaliszyk |
Fix eqvt for multiple quantifiers.
|
file |
diff |
annotate
|
2010-03-03 |
Cezary Kaliszyk |
weird eqvt
|
file |
diff |
annotate
|
2010-03-02 |
Cezary Kaliszyk |
Comment out the part that does not work with 2 quantifiers.
|
file |
diff |
annotate
|
2010-03-02 |
Cezary Kaliszyk |
Porting from Lift to Parser; until defining the Quotient type.
|
file |
diff |
annotate
|
2010-03-02 |
Cezary Kaliszyk |
Working bv_eqvt
|
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-02 |
Christian Urban |
rawified the bind specs (ready to be used now)
|
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 |
further code-refactoring in the parser
|
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 |
a few simplifications
|
file |
diff |
annotate
|
2010-02-25 |
Christian Urban |
added IsaMakefile...but so far included only a test for the parser
|
file |
diff |
annotate
| base
|