QuotMain.thy
2009-12-03 Christian Urban further simplification
2009-12-03 Christian Urban simplified lambda_prs_conv
2009-12-02 Christian Urban deleted now obsolete argument rty everywhere
2009-12-02 Christian Urban deleted tests at the beginning of QuotMain
2009-12-02 Cezary Kaliszyk Experiments with OPTION_map
2009-12-02 Cezary Kaliszyk merge
2009-12-02 Cezary Kaliszyk More experiments with higher order quotients and theorems with non-lifted constants.
2009-12-02 Christian Urban merged
2009-12-02 Cezary Kaliszyk New APPLY_RSP which finally does automatic partial lifting :). Doesn't support same relation yet.
2009-12-02 Cezary Kaliszyk Fixed unlam for non-abstractions and updated list_induct_part proof.
2009-12-02 Cezary Kaliszyk Removed the use of 'rty' from APPLY_RSP, finally LF proofs go automatically.
2009-12-02 Cezary Kaliszyk The conversion approach works.
2009-12-02 Cezary Kaliszyk Added tactic for dealing with QUOT_TRUE and introducing QUOT_TRUE.
2009-12-01 Cezary Kaliszyk back in working state
2009-12-01 Cezary Kaliszyk clean
2009-12-01 Christian Urban fixed previous commit
2009-12-01 Christian Urban fixed problems with FOCUS
2009-12-01 Christian Urban added a make_inst test
2009-12-01 Cezary Kaliszyk Transformation of QUOT_TRUE assumption by any given function
2009-12-01 Christian Urban QUOT_TRUE joke
2009-12-01 Cezary Kaliszyk Removed last HOL_ss
2009-12-01 Cezary Kaliszyk more cleaning
2009-12-01 Cezary Kaliszyk Cleaning 'aps'.
2009-11-30 Cezary Kaliszyk merge
2009-11-30 Christian Urban cleaned inj_regabs_trm
2009-11-30 Cezary Kaliszyk merge
2009-11-30 Cezary Kaliszyk clean_tac rewrites the definitions the other way
2009-11-30 Christian Urban merged
2009-11-30 Christian Urban added facilities to get all stored quotient data (equiv thms etc)
2009-11-30 Cezary Kaliszyk More code cleaning
2009-11-30 Cezary Kaliszyk Code cleaning.
2009-11-30 Cezary Kaliszyk Commented clean-tac
2009-11-29 Christian Urban tried to improve the inj_repabs_trm function but left the new part commented out
2009-11-29 Christian Urban started functions for qid-insertion and fixed a bug in regularise
2009-11-29 Cezary Kaliszyk Removed unnecessary HOL_ss which proved one of the subgoals.
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.
2009-11-29 Christian Urban introduced a global list of respectfulness lemmas; the attribute is [quot_rsp]
2009-11-29 Christian Urban tuned
2009-11-28 Christian Urban improved pattern matching inside the inj_repabs_tacs
2009-11-28 Christian Urban selective debugging of the inj_repabs_tac (at the moment for step 3 and 4 debugging information is printed)
2009-11-28 Christian Urban removed old inj_repabs_tac; kept only the one with (selective) debugging information
2009-11-28 Christian Urban renamed r_mk_comb_tac to inj_repabs_tac
2009-11-28 Christian Urban tuning
2009-11-28 Christian Urban tuned comments
2009-11-28 Christian Urban renamed LAMBDA_RES_TAC and WEAK_LAMBDA_RES_TAC to lower case names
2009-11-28 Cezary Kaliszyk Moved fast instantiation to QuotMain
2009-11-28 Christian Urban further proper merge
2009-11-28 Christian Urban merged
2009-11-28 Christian Urban more simplification
2009-11-28 Cezary Kaliszyk Merged and tested that all works.
2009-11-28 Cezary Kaliszyk Finished and tested the new regularize
2009-11-28 Christian Urban more tuning of the repabs-tactics
2009-11-28 Christian Urban merged
2009-11-28 Christian Urban fixed previous commit
2009-11-28 Cezary Kaliszyk Cleaned all lemmas about regularisation of Ball and Bex and moved in one place. Second Ball simprox.
2009-11-28 Cezary Kaliszyk Merged comment
2009-11-28 Christian Urban some slight tuning of the apply-tactic
2009-11-28 Christian Urban annotated a proof with all steps and simplified LAMBDA_RES_TAC
2009-11-27 Christian Urban replaced FIRST' (map rtac list) with resolve_tac list
2009-11-27 Cezary Kaliszyk Simplifying arguments; got rid of trans2_thm.
2009-11-27 Cezary Kaliszyk Removing arguments of tactics: absrep, rel_refl, reps_same are computed.
2009-11-27 Cezary Kaliszyk More cleaning in QuotMain, identity handling.
2009-11-27 Christian Urban tuned
2009-11-27 Christian Urban some tuning
2009-11-27 Christian Urban simplified gen_frees_tac and properly named abstracted variables
2009-11-27 Christian Urban removed CHANGED'
2009-11-27 Christian Urban introduced a separate lemma for id_simps
2009-11-27 Christian Urban renamed inj_REPABS to inj_repabs_trm
2009-11-27 Christian Urban tuned comments and moved slightly some code
2009-11-27 Christian Urban renamed REGULARIZE to be regularize
2009-11-26 Christian Urban more tuning
2009-11-26 Christian Urban deleted get_fun_old and stuff
2009-11-26 Christian Urban recommited changes of comments
2009-11-26 Cezary Kaliszyk Merge Again
2009-11-26 Cezary Kaliszyk Merged
2009-11-26 Christian Urban tuned comments
2009-11-26 Christian Urban some diagnostic code for r_mk_comb
2009-11-26 Christian Urban merged
2009-11-26 Christian Urban test with monos
2009-11-25 Cezary Kaliszyk applic_prs
2009-11-25 Christian Urban polishing
2009-11-25 Christian Urban reordered the code
2009-11-25 Cezary Kaliszyk Moved exception handling to QuotMain and cleaned FSet.
2009-11-25 Christian Urban comments tuning and slight reordering
2009-11-25 Cezary Kaliszyk Merge
2009-11-25 Cezary Kaliszyk More moving from QuotMain to UnusedQuotMain
2009-11-25 Christian Urban deleted some obsolete diagnostic code
2009-11-25 Cezary Kaliszyk Removed unused things from QuotMain.
2009-11-25 Cezary Kaliszyk lambda_prs and cleaning the existing examples.
2009-11-25 Christian Urban fixed the problem with generalising variables; at the moment it is quite a hack
2009-11-24 Christian Urban changed unification to matching
2009-11-24 Christian Urban unification
2009-11-24 Cezary Kaliszyk Lambda & SOLVED' for new quotient_tac
2009-11-24 Christian Urban merged
2009-11-24 Christian Urban merged
2009-11-24 Christian Urban use error instead of raising our own exception
2009-11-24 Cezary Kaliszyk Fixes to the tactic after quotient_tac changed.
2009-11-24 Christian Urban merged
2009-11-24 Christian Urban added a prepare_tac
2009-11-24 Cezary Kaliszyk TRY' for clean_tac
2009-11-24 Cezary Kaliszyk Moved cleaning to QuotMain
2009-11-24 Cezary Kaliszyk New cleaning tactic
2009-11-24 Cezary Kaliszyk Separate regularize_tac
2009-11-24 Cezary Kaliszyk More fixes for inj_REPABS
2009-11-24 Christian Urban addded a tactic, which sets up the three goals of the `algorithm'
2009-11-23 Christian Urban fixed the error by a temporary fix (the data of the eqivalence relation should be only its name)
2009-11-23 Christian Urban tuned some comments
2009-11-23 Cezary Kaliszyk domain_type in regularizing equality
2009-11-23 Cezary Kaliszyk More theorems lifted in the goal-directed way.
2009-11-23 Cezary Kaliszyk Finished temporary goal-directed lift_theorem wrapper.
2009-11-23 Christian Urban merged
2009-11-23 Christian Urban a version of inj_REPABS (needs to be looked at again later)
2009-11-23 Cezary Kaliszyk Fixes for atomize
2009-11-23 Christian Urban slight change in code layout
2009-11-23 Cezary Kaliszyk Removing dead code
2009-11-23 Cezary Kaliszyk Move atomize_goal to QuotMain
2009-11-23 Cezary Kaliszyk Moved new repabs_inj code to QuotMain
2009-11-23 Christian Urban code review with Cezary
2009-11-21 Christian Urban a little tuning of comments
2009-11-21 Christian Urban my first version of repabs injection
2009-11-21 Christian Urban tuned
2009-11-21 Christian Urban tuned
2009-11-21 Christian Urban simplified get_fun so that it uses directly rty and qty, instead of qenv
2009-11-20 Christian Urban started regularize of rtrm/qtrm version; looks quite promising
2009-11-19 Christian Urban updated to new Isabelle
2009-11-13 Christian Urban added some tracing information to all phases of lifting to the function lift_thm
2009-11-12 Cezary Kaliszyk merged
2009-11-12 Christian Urban changed the quotdata to be a symtab table (needs fixing)
less more (0) -128 tip