IntEx.thy
2009-12-06 Christian Urban working on lambda_prs with examples; polished code of clean_tac
2009-12-05 Christian Urban merged
2009-12-05 Christian Urban added new example for Ints; regularise does not work in all instances
2009-12-05 Cezary Kaliszyk Proved foldl_rsp and ho_map_rsp
2009-12-05 Christian Urban moved all_prs and ex_prs out from the conversion into the simplifier
2009-12-05 Cezary Kaliszyk Added nil_rsp and cons_rsp to quotient_rsp; simplified IntEx.
2009-12-05 Christian Urban merged
2009-12-05 Christian Urban merged
2009-12-05 Christian Urban merged
2009-12-05 Christian Urban simpler version of clean_tac
2009-12-05 Cezary Kaliszyk Handling of respects in the fast inj_repabs_tac; includes respects with quotient assumptions.
2009-12-05 Cezary Kaliszyk Solutions to IntEx tests.
2009-12-05 Christian Urban made some slight simplifications to the examples
2009-12-05 Christian Urban added three examples to IntEx for testing ideas - regularisation and injection seem to be not quite right yet
2009-12-04 Christian Urban not yet quite functional treatment of constants
2009-12-04 Cezary Kaliszyk More code cleaning and renaming: moved rsp and prs lemmas from Int to QuotList
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 More name changes
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 Cezary Kaliszyk Updated the examples
2009-12-03 Christian Urban merged
2009-12-03 Christian Urban deleted some dead code
2009-12-02 Christian Urban deleted now obsolete argument rty everywhere
2009-12-02 Cezary Kaliszyk More experiments with higher order quotients and theorems with non-lifted constants.
2009-12-01 Cezary Kaliszyk Cleaning 'aps'.
2009-11-30 Cezary Kaliszyk Code cleaning.
2009-11-29 Christian Urban tried to improve the inj_repabs_trm function but left the new part commented out
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-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 Cezary Kaliszyk Merged and tested that all works.
2009-11-28 Cezary Kaliszyk Finished and tested the new regularize
2009-11-28 Christian Urban fixed examples in IntEx and FSet
2009-11-28 Christian Urban fixed previous commit
2009-11-28 Christian Urban annotated a proof with all steps and simplified LAMBDA_RES_TAC
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 Minor cleaning
2009-11-27 Christian Urban introduced a separate lemma for id_simps
2009-11-27 Christian Urban deleted obsolete qenv code
2009-11-27 Christian Urban renamed REGULARIZE to be regularize
2009-11-25 Cezary Kaliszyk applic_prs
2009-11-25 Cezary Kaliszyk Removed unused things from QuotMain.
2009-11-25 Cezary Kaliszyk cleaning in MyInt
2009-11-25 Christian Urban fixed the problem with generalising variables; at the moment it is quite a hack
2009-11-24 Christian Urban added a prepare_tac
2009-11-24 Cezary Kaliszyk Moved cleaning to QuotMain
2009-11-24 Cezary Kaliszyk New cleaning tactic
2009-11-24 Christian Urban explicit phases for the cleaning
2009-11-24 Christian Urban addded a tactic, which sets up the three goals of the `algorithm'
2009-11-23 Cezary Kaliszyk Finished temporary goal-directed lift_theorem wrapper.
2009-11-23 Cezary Kaliszyk Fixes for atomize
2009-11-23 Cezary Kaliszyk lift_thm with a goal.
2009-11-23 Cezary Kaliszyk Fixes for new code
2009-11-23 Cezary Kaliszyk Moved new repabs_inj code to QuotMain
2009-11-23 Cezary Kaliszyk New repabs behaves the same way as old one.
2009-11-23 Christian Urban code review with Cezary
2009-11-21 Christian Urban a little tuning of comments
2009-11-21 Christian Urban slight tuning
2009-11-21 Christian Urban some debugging code, but cannot find the place where the cprems_of exception is raised
2009-11-21 Christian Urban tried to prove the repabs_inj lemma, but failed for the moment
2009-11-21 Christian Urban my first version of repabs injection
2009-11-21 Christian Urban tunded
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-18 Christian Urban fixed the storage of qconst definitions
2009-11-12 Christian Urban looking up data in quot_info works now (needs qualified string)
2009-11-12 Christian Urban added a container for quotient constants (does not work yet though)
2009-11-11 Christian Urban updated to new Theory_Data and to new Isabelle
2009-11-11 Cezary Kaliszyk Removed 'Toplevel.program' for polyml 5.3
2009-11-05 Christian Urban removed typing information from get_fun in quotient_def; *potentially* dangerous
2009-11-05 Christian Urban merged
2009-11-04 Cezary Kaliszyk Experiments with lifting partially applied constants.
2009-11-04 Cezary Kaliszyk Experiments in Int
2009-11-04 Christian Urban fixed definition of PLUS
2009-11-04 Christian Urban simplified the quotient_def code
2009-11-03 Christian Urban simplified the quotient_def code; type of the defined constant must now be given; for-part eliminated
2009-11-02 Christian Urban slightly saner way of parsing the quotient_def
2009-11-02 Christian Urban merged
2009-11-02 Christian Urban changed Type.typ_match to Sign.typ_match
2009-11-02 Cezary Kaliszyk Fixes after optimization and preparing for a general FORALL_PRS
2009-10-30 Cezary Kaliszyk Cleaning of the interface to lift.
2009-10-28 Cezary Kaliszyk disambiguate ===> syntax
2009-10-28 Cezary Kaliszyk Cleaning the unnecessary theorems in 'IntEx'.
2009-10-28 Cezary Kaliszyk merge
2009-10-28 Cezary Kaliszyk Fixes
2009-10-28 Christian Urban updated all definitions
2009-10-28 Christian Urban added infrastructure for defining lifted constants
2009-10-27 Cezary Kaliszyk Simplfied interface to repabs_injection.
2009-10-27 Cezary Kaliszyk Fixed APPLY_RSP vs Cong in the InjRepAbs tactic.
2009-10-27 Christian Urban made quotients compatiple with Nominal; updated keyword file
2009-10-27 Christian Urban merged
2009-10-27 Cezary Kaliszyk Completely cleaned Int.
2009-10-27 Cezary Kaliszyk Further reordering in Int code.
2009-10-26 Cezary Kaliszyk Simplifying Int.
2009-10-26 Cezary Kaliszyk Merge
2009-10-26 Cezary Kaliszyk Simplifying Int and Working on map
2009-10-26 Christian Urban merged
2009-10-26 Cezary Kaliszyk Simplifying code in int
2009-10-26 Cezary Kaliszyk Symmetry of integer addition
2009-10-24 Christian Urban added "print_quotients" command to th ekeyword file
2009-10-24 Christian Urban added another example file about integers (see HOL/Int.thy)
less more (0) tip