2009-11-30 |
Cezary Kaliszyk |
clean_tac rewrites the definitions the other way
|
file |
diff |
annotate
|
2009-11-30 |
Cezary Kaliszyk |
More code cleaning
|
file |
diff |
annotate
|
2009-11-30 |
Cezary Kaliszyk |
Code cleaning.
|
file |
diff |
annotate
|
2009-11-29 |
Christian Urban |
tried to improve the inj_repabs_trm function but left the new part commented out
|
file |
diff |
annotate
|
2009-11-29 |
Cezary Kaliszyk |
Removed unnecessary HOL_ss which proved one of the subgoals.
|
file |
diff |
annotate
|
2009-11-29 |
Cezary Kaliszyk |
Added 'TRY' to refl in clean_tac to get as far as possible. Removed unnecessary [quot_rsp] in FSet. Added necessary [quot_rsp] and one lifted thm in LamEx.
|
file |
diff |
annotate
|
2009-11-29 |
Christian Urban |
introduced a global list of respectfulness lemmas; the attribute is [quot_rsp]
|
file |
diff |
annotate
|
2009-11-28 |
Christian Urban |
improved pattern matching inside the inj_repabs_tacs
|
file |
diff |
annotate
|
2009-11-28 |
Christian Urban |
removed old inj_repabs_tac; kept only the one with (selective) debugging information
|
file |
diff |
annotate
|
2009-11-28 |
Christian Urban |
renamed r_mk_comb_tac to inj_repabs_tac
|
file |
diff |
annotate
|
2009-11-28 |
Christian Urban |
renamed LAMBDA_RES_TAC and WEAK_LAMBDA_RES_TAC to lower case names
|
file |
diff |
annotate
|
2009-11-28 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2009-11-28 |
Christian Urban |
more simplification
|
file |
diff |
annotate
|
2009-11-28 |
Cezary Kaliszyk |
Merged and tested that all works.
|
file |
diff |
annotate
|
2009-11-28 |
Cezary Kaliszyk |
Finished and tested the new regularize
|
file |
diff |
annotate
|
2009-11-28 |
Christian Urban |
fixed examples in IntEx and FSet
|
file |
diff |
annotate
|
2009-11-28 |
Christian Urban |
annotated a proof with all steps and simplified LAMBDA_RES_TAC
|
file |
diff |
annotate
|
2009-11-27 |
Christian Urban |
replaced FIRST' (map rtac list) with resolve_tac list
|
file |
diff |
annotate
|
2009-11-27 |
Cezary Kaliszyk |
Simplifying arguments; got rid of trans2_thm.
|
file |
diff |
annotate
|
2009-11-27 |
Cezary Kaliszyk |
Removing arguments of tactics: absrep, rel_refl, reps_same are computed.
|
file |
diff |
annotate
|
2009-11-27 |
Cezary Kaliszyk |
Minor cleaning
|
file |
diff |
annotate
|
2009-11-26 |
Cezary Kaliszyk |
Merge Again
|
file |
diff |
annotate
|
2009-11-26 |
Cezary Kaliszyk |
Merged
|
file |
diff |
annotate
|
2009-11-26 |
Christian Urban |
tuned comments
|
file |
diff |
annotate
|
2009-11-26 |
Christian Urban |
some diagnostic code for r_mk_comb
|
file |
diff |
annotate
|
2009-11-26 |
Christian Urban |
introduced a new property for Ball and ===> on the left
|
file |
diff |
annotate
|
2009-11-26 |
Christian Urban |
changed left-res
|
file |
diff |
annotate
|
2009-11-26 |
Cezary Kaliszyk |
Fixed FSet after merge.
|
file |
diff |
annotate
|
2009-11-26 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2009-11-26 |
Christian Urban |
test with monos
|
file |
diff |
annotate
|
2009-11-25 |
Cezary Kaliszyk |
applic_prs
|
file |
diff |
annotate
|
2009-11-25 |
Christian Urban |
reordered the code
|
file |
diff |
annotate
|
2009-11-25 |
Cezary Kaliszyk |
Moved exception handling to QuotMain and cleaned FSet.
|
file |
diff |
annotate
|
2009-11-25 |
Cezary Kaliszyk |
Finished manual lifting of list_induct_part :)
|
file |
diff |
annotate
|
2009-11-25 |
Cezary Kaliszyk |
Removed unused things from QuotMain.
|
file |
diff |
annotate
|
2009-11-25 |
Cezary Kaliszyk |
lambda_prs and cleaning the existing examples.
|
file |
diff |
annotate
|
2009-11-25 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2009-11-25 |
Christian Urban |
fixed the problem with generalising variables; at the moment it is quite a hack
|
file |
diff |
annotate
|
2009-11-24 |
Cezary Kaliszyk |
Ho-matching failures...
|
file |
diff |
annotate
|
2009-11-24 |
Cezary Kaliszyk |
Conversion
|
file |
diff |
annotate
|
2009-11-24 |
Cezary Kaliszyk |
The non-working procedure_tac.
|
file |
diff |
annotate
|
2009-11-24 |
Cezary Kaliszyk |
Fixes to the tactic after quotient_tac changed.
|
file |
diff |
annotate
|
2009-11-24 |
Cezary Kaliszyk |
Another theorem for which the new regularize differs from old one, so the goal is not proved. But it seems, that the new one is better.
|
file |
diff |
annotate
|
2009-11-23 |
Christian Urban |
fixed the error by a temporary fix (the data of the eqivalence relation should be only its name)
|
file |
diff |
annotate
|
2009-11-23 |
Cezary Kaliszyk |
Another not-typechecking regularized term.
|
file |
diff |
annotate
|
2009-11-23 |
Cezary Kaliszyk |
domain_type in regularizing equality
|
file |
diff |
annotate
|
2009-11-23 |
Cezary Kaliszyk |
More theorems lifted in the goal-directed way.
|
file |
diff |
annotate
|
2009-11-23 |
Cezary Kaliszyk |
Move atomize_goal to QuotMain
|
file |
diff |
annotate
|
2009-11-23 |
Cezary Kaliszyk |
Removed second implementation of Regularize/Inject from FSet.
|
file |
diff |
annotate
|
2009-11-23 |
Cezary Kaliszyk |
New repabs behaves the same way as old one.
|
file |
diff |
annotate
|
2009-11-23 |
Christian Urban |
code review with Cezary
|
file |
diff |
annotate
|
2009-11-23 |
Cezary Kaliszyk |
The other branch does not seem to work...
|
file |
diff |
annotate
|
2009-11-23 |
Cezary Kaliszyk |
Fixes for recent changes.
|
file |
diff |
annotate
|
2009-11-13 |
Cezary Kaliszyk |
Still don't know how to do the proof automatically.
|
file |
diff |
annotate
|
2009-11-12 |
Cezary Kaliszyk |
merged
|
file |
diff |
annotate
|
2009-11-11 |
Cezary Kaliszyk |
Lifting towards goal and manually finished the proof.
|
file |
diff |
annotate
|
2009-11-11 |
Cezary Kaliszyk |
Removed 'Toplevel.program' for polyml 5.3
|
file |
diff |
annotate
|
2009-11-10 |
Cezary Kaliszyk |
Atomizing a "goal" theorems.
|
file |
diff |
annotate
|
2009-11-09 |
Cezary Kaliszyk |
Fixes for the other get_fun implementation.
|
file |
diff |
annotate
|
2009-11-06 |
Cezary Kaliszyk |
Minor changes
|
file |
diff |
annotate
|