2009-12-04 Cezary Kaliszyk Cleaning & Renaming coming from QuotList
2009-12-04 Cezary Kaliszyk Cleaning in Quotients
2009-12-04 Cezary Kaliszyk Even more name changes and cleaning
2009-12-04 Cezary Kaliszyk More code cleaning and name changes
2009-12-04 Cezary Kaliszyk merge
2009-12-04 Cezary Kaliszyk merged
2009-12-04 Christian Urban smaller theory footprint
2009-12-04 Christian Urban merged
2009-12-04 Christian Urban merge
2009-12-04 Christian Urban smaller theory footprint
2009-12-04 Cezary Kaliszyk More name changes
2009-12-04 Cezary Kaliszyk Naming changes
2009-12-04 Cezary Kaliszyk code cleaning and renaming
2009-12-04 Cezary Kaliszyk merge
2009-12-04 Cezary Kaliszyk Removed previous inj_repabs_tac
2009-12-04 Christian Urban some tuning
2009-12-04 Cezary Kaliszyk merge
2009-12-04 Cezary Kaliszyk rep_abs_rsp_tac to replace the last use of instantiate_tac with matching and unification.
2009-12-04 Christian Urban merged
2009-12-04 Christian Urban merged
2009-12-04 Cezary Kaliszyk Change equiv_trans2 to EQUALS_RSP, since we can prove it for any quotient type, not only for eqv relations.
2009-12-04 Cezary Kaliszyk compose_tac instead of rtac to avoid unification; some code cleaning.
2009-12-04 Cezary Kaliszyk Got to about 5 seconds for the longest proof. APPLY_RSP_TAC' solves the quotient internally without instantiation resulting in a faster proof.
2009-12-04 Cezary Kaliszyk Using APPLY_RSP1; again a little bit faster.
2009-12-04 Cezary Kaliszyk Fixes after big merge.
2009-12-04 Cezary Kaliszyk The big merge; probably non-functional.
2009-12-04 Cezary Kaliszyk Testing the new tactic everywhere
2009-12-04 Cezary Kaliszyk First version of the deterministic rep-abs-inj-tac.
2009-12-04 Cezary Kaliszyk Changing = to \<equiv> in case if we want to use simp.
2009-12-04 Cezary Kaliszyk Even better: Completely got rid of the simps in both quotient_tac and inj_repabs_tac
2009-12-04 Cezary Kaliszyk merge
2009-12-04 Cezary Kaliszyk Made your version work again with LIST_REL_EQ.
2009-12-03 Christian Urban the error occurs in APPLY_RSP_TAC where the wrong quotient (for LIST_REL) is applied
2009-12-03 Christian Urban removed quot argument...not all examples work anymore
2009-12-03 Christian Urban merged
2009-12-03 Christian Urban merged
2009-12-03 Christian Urban first version of internalised quotient theorems; added FIXME-TODO
2009-12-03 Christian Urban further dead code
2009-12-03 Cezary Kaliszyk Reintroduced varifyT; we still need it for permutation definition.
2009-12-03 Cezary Kaliszyk Updated the examples
2009-12-03 Cezary Kaliszyk Fixed previous mistake
2009-12-03 Cezary Kaliszyk defs used automatically by clean_tac
2009-12-03 Cezary Kaliszyk Added qoutient_consts dest for getting all the constant definitions in the cleaning step.
2009-12-03 Cezary Kaliszyk Added the definition to quotient constant data.
2009-12-03 Cezary Kaliszyk removing unused code
2009-12-03 Christian Urban merged
2009-12-03 Christian Urban deleted some dead code
2009-12-03 Cezary Kaliszyk Included all_prs and ex_prs in the lambda_prs conversion.
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 Lifting to 2 different types :)
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 Trying a conversion based approach.
2009-12-02 Cezary Kaliszyk A bit of progress; but the object-logic vs meta-logic distinction is troublesome.
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-30 Cezary Kaliszyk Added another induction to LFex
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 added a new version of QuotMain to experiment with qids
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
(0) -300 -100 -96 +96 +100 +300 +1000 tip