2010-01-16 |
Christian Urban |
liftin and lifing_tac can now lift several "and"-separated goals at once; the raw-theorems have to be given in the order of goals
|
file |
diff |
annotate
|
2010-01-14 |
Cezary Kaliszyk |
Remove SOLVED from quotient_tac. Move atomize_eqv to 'Unused'.
|
file |
diff |
annotate
|
2010-01-14 |
Cezary Kaliszyk |
Finished organising an efficient datastructure for qconst_info.
|
file |
diff |
annotate
|
2010-01-12 |
Christian Urban |
absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM"
|
file |
diff |
annotate
|
2010-01-11 |
Christian Urban |
tuned previous commit further
|
file |
diff |
annotate
|
2010-01-10 |
Christian Urban |
the chk-functions in quotient_term also simplify the result according to the id_simps; had to remove id_def from this theorem list though; this caused in FSet3 that relied on this rule; the problem is marked with "ID PROBLEM"
|
file |
diff |
annotate
|
2010-01-08 |
Cezary Kaliszyk |
Modifictaions for new_relation.
|
file |
diff |
annotate
|
2009-12-24 |
Christian Urban |
tuned
|
file |
diff |
annotate
|
2009-12-23 |
Christian Urban |
renamed QUOT_TYPE to Quot_Type
|
file |
diff |
annotate
|
2009-12-22 |
Christian Urban |
moved get_fun into quotient_term; this simplifies the overall including structure of the package
|
file |
diff |
annotate
|
2009-12-22 |
Christian Urban |
tuned comments; renamed QUOT_TRUE to Quot_True; atomize_eqv seems to not be neccessary (has it been added to Isabelle)...it is now comented out and everything still works
|
file |
diff |
annotate
|
2009-12-21 |
Christian Urban |
get_fun needed change to cope with "('a fset) fset" types...this needs composition (op o); now id_simps contains also id_o and o_id, and map_id is also added in QuotList.thy; regularize and cleaning needed to be hacked (indicated by "HACK")...THIS NEEDS ATTENTION!!!; except two lemmas in IntEx, all examples go through; added considerable material to FSet3; tuned FIXME-TODO
|
file |
diff |
annotate
|
2009-12-17 |
Christian Urban |
minor cleaning
|
file |
diff |
annotate
|
2009-12-17 |
Christian Urban |
moved the QuotMain code into two ML-files
|
file |
diff |
annotate
|
2009-12-15 |
Cezary Kaliszyk |
lambda_prs & solve_quotient_assum cleaned.
|
file |
diff |
annotate
|
2009-12-15 |
Christian Urban |
some commenting
|
file |
diff |
annotate
|
2009-12-14 |
Cezary Kaliszyk |
Fixed previous commit.
|
file |
diff |
annotate
|
2009-12-14 |
Cezary Kaliszyk |
Moved DETERM inside Repeat & added SOLVE around quotient_tac.
|
file |
diff |
annotate
|
2009-12-14 |
Cezary Kaliszyk |
reply to question in code
|
file |
diff |
annotate
|
2009-12-14 |
Cezary Kaliszyk |
Reply in code.
|
file |
diff |
annotate
|
2009-12-13 |
Christian Urban |
a few code annotations
|
file |
diff |
annotate
|
2009-12-13 |
Christian Urban |
another pass on apply_rsp
|
file |
diff |
annotate
|
2009-12-13 |
Christian Urban |
managed to simplify apply_rsp
|
file |
diff |
annotate
|
2009-12-12 |
Christian Urban |
tried to simplify apply_rsp_tac; failed at the moment; added some questions
|
file |
diff |
annotate
|
2009-12-12 |
Christian Urban |
some trivial changes
|
file |
diff |
annotate
|
2009-12-12 |
Christian Urban |
trivial cleaning of make_inst
|
file |
diff |
annotate
|
2009-12-12 |
Christian Urban |
tried to improve test; but fails
|
file |
diff |
annotate
|
2009-12-12 |
Christian Urban |
merged
|
file |
diff |
annotate
|
2009-12-12 |
Christian Urban |
annotated some questions to the code; some simple changes
|
file |
diff |
annotate
|
2009-12-12 |
Cezary Kaliszyk |
Answering the question in code.
|
file |
diff |
annotate
|
2009-12-12 |
Christian Urban |
tuned code
|
file |
diff |
annotate
|
2009-12-12 |
Christian Urban |
renamed quotient.ML to quotient_typ.ML
|
file |
diff |
annotate
|
2009-12-11 |
Cezary Kaliszyk |
Merge + Added LarryInt & Fset3 to tests.
|
file |
diff |
annotate
|
2009-12-11 |
Cezary Kaliszyk |
Renaming
|
file |
diff |
annotate
|
2009-12-11 |
Christian Urban |
deleted struct_match by Pattern.match (fixes a problem in LarryInt)
|
file |
diff |
annotate
|
2009-12-11 |
Christian Urban |
added Int example from Larry
|
file |
diff |
annotate
|
2009-12-11 |
Christian Urban |
changed error message
|
file |
diff |
annotate
|
2009-12-11 |
Christian Urban |
reformulated the lemma lifting_procedure as ML value; gave better warning message for injection case
|
file |
diff |
annotate
|
2009-12-10 |
Christian Urban |
added maps-printout and tuned some comments
|
file |
diff |
annotate
|
2009-12-10 |
Cezary Kaliszyk |
Regularized the hard lemma.
|
file |
diff |
annotate
|
2009-12-10 |
Cezary Kaliszyk |
Found the problem with ttt3.
|
file |
diff |
annotate
|
2009-12-10 |
Cezary Kaliszyk |
minor
|
file |
diff |
annotate
|
2009-12-10 |
Cezary Kaliszyk |
Moved Unused part of locale to Unused QuotMain.
|
file |
diff |
annotate
|
2009-12-10 |
Christian Urban |
more tuning
|
file |
diff |
annotate
|
2009-12-10 |
Christian Urban |
tuned
|
file |
diff |
annotate
|
2009-12-10 |
Christian Urban |
simplified the instantiation of QUOT_TRUE in procedure_tac
|
file |
diff |
annotate
|
2009-12-10 |
Christian Urban |
completed previous commit
|
file |
diff |
annotate
|
2009-12-10 |
Christian Urban |
deleted DT/NDT diagnostic code
|
file |
diff |
annotate
|
2009-12-09 |
Cezary Kaliszyk |
Code cleaning.
|
file |
diff |
annotate
|
2009-12-09 |
Christian Urban |
tuned
|
file |
diff |
annotate
|
2009-12-09 |
Cezary Kaliszyk |
merge
|
file |
diff |
annotate
|
2009-12-09 |
Cezary Kaliszyk |
Different syntax for definitions that allows overloading and retrieving of definitions by matching whole constants.
|
file |
diff |
annotate
|
2009-12-09 |
Christian Urban |
deleted make_inst3
|
file |
diff |
annotate
|
2009-12-09 |
Christian Urban |
tuned
|
file |
diff |
annotate
|
2009-12-09 |
Christian Urban |
tuned
|
file |
diff |
annotate
|
2009-12-09 |
Christian Urban |
moved function and tuned comment
|
file |
diff |
annotate
|
2009-12-09 |
Christian Urban |
improved fun_map_conv
|
file |
diff |
annotate
|
2009-12-09 |
Cezary Kaliszyk |
Arbitrary number of fun_map_tacs.
|
file |
diff |
annotate
|
2009-12-09 |
Cezary Kaliszyk |
Temporarily repeated fun_map_tac 4 times. Cleaning for all examples work.
|
file |
diff |
annotate
|
2009-12-08 |
Christian Urban |
tuned code
|
file |
diff |
annotate
|