2009-12-09 Cezary Kaliszyk Finished one proof in IntEx2.
2009-12-09 Christian Urban slightly more on IntEx2
2009-12-09 Christian Urban proved (with a lot of pain) that times_raw is respectful
2009-12-09 Christian Urban merged
2009-12-09 Christian Urban fixed minor stupidity
2009-12-09 Cezary Kaliszyk Exception handling.
2009-12-09 Cezary Kaliszyk Code cleaning.
2009-12-09 Cezary Kaliszyk merge
2009-12-09 Cezary Kaliszyk foldr_rsp.
2009-12-09 Christian Urban tuned
2009-12-09 Cezary Kaliszyk merge
2009-12-09 Cezary Kaliszyk Different syntax for definitions that allows overloading and retrieving of definitions by matching whole constants.
2009-12-09 Christian Urban deleted make_inst3
2009-12-09 Christian Urban tuned
2009-12-09 Christian Urban tuned
2009-12-09 Christian Urban moved function and tuned comment
2009-12-09 Christian Urban improved fun_map_conv
2009-12-09 Cezary Kaliszyk Arbitrary number of fun_map_tacs.
2009-12-09 Cezary Kaliszyk Temporarily repeated fun_map_tac 4 times. Cleaning for all examples work.
2009-12-08 Christian Urban tuned code
2009-12-08 Christian Urban tuned the examples and flagged the problematic cleaning lemmas in FSet
2009-12-08 Christian Urban merged
2009-12-08 Christian Urban implemented cleaning strategy with fun_map.simps on non-bounded variables; still a few rough edges
2009-12-08 Cezary Kaliszyk merge
2009-12-08 Cezary Kaliszyk manually cleaned the hard lemma.
2009-12-08 Christian Urban merged
2009-12-08 Christian Urban decoupled QuotProd from QuotMain and also started new cleaning strategy
2009-12-08 Cezary Kaliszyk merge
2009-12-08 Cezary Kaliszyk An example which is hard to lift because of the interplay between lambda_prs and unfolding.
2009-12-08 Christian Urban proper formulation of all preservation theorems
2009-12-08 Christian Urban started to reformulate preserve lemmas
2009-12-08 Christian Urban properly set up the prs_rules
2009-12-08 Christian Urban merged
2009-12-08 Christian Urban added preserve rules to the cleaning_tac
2009-12-08 Cezary Kaliszyk merge
2009-12-08 Cezary Kaliszyk cleaning.
2009-12-08 Christian Urban merged
2009-12-08 Christian Urban chnaged syntax to "lifting theorem"
2009-12-08 Christian Urban changed names of attributes
2009-12-08 Cezary Kaliszyk merge
2009-12-08 Cezary Kaliszyk Manual regularization of a goal in FSet.
2009-12-08 Christian Urban merged
2009-12-08 Christian Urban added methods for the lifting_tac and the other tacs
2009-12-08 Cezary Kaliszyk make_inst3
2009-12-08 Cezary Kaliszyk Merge
2009-12-08 Cezary Kaliszyk trans2 replaced with equals_rsp_tac
2009-12-08 Christian Urban corrected name of FSet in ROOT.ML
2009-12-08 Cezary Kaliszyk Made fset work again to test all.
2009-12-08 Cezary Kaliszyk Finished the proof of ttt2 and found bug in regularize when trying ttt3.
2009-12-08 Cezary Kaliszyk Another lambda example theorem proved. Seems it starts working properly.
2009-12-08 Cezary Kaliszyk Removed pattern from quot_rel_rsp, since list_rel and all used introduced ones cannot be patterned
2009-12-08 Cezary Kaliszyk Proper checked map_rsp.
2009-12-08 Cezary Kaliszyk Nitpick found a counterexample for one lemma.
2009-12-08 Cezary Kaliszyk Added a 'rep_abs' in inj_repabs_trm of babs; and proved two lam examples.
2009-12-08 Cezary Kaliszyk It also regularizes.
2009-12-08 Cezary Kaliszyk inj_repabs also works.
2009-12-08 Cezary Kaliszyk merge
2009-12-08 Cezary Kaliszyk An example of working cleaning for lambda lifting. Still not sure why Babs helps.
2009-12-08 Christian Urban tuned
2009-12-08 Christian Urban the lift_tac produces a warning message if one of the three automatic proofs fails
2009-12-08 Christian Urban added a thm list for ids
2009-12-08 Christian Urban removed a fixme: map_info is now checked
2009-12-07 Christian Urban tuning of the code
2009-12-07 Christian Urban merged
2009-12-07 Christian Urban removed "global" data and lookup functions; had to move a tactic out from the inj_repabs_match tactic since apply_rsp interferes with a trans2 rule for ===>
2009-12-07 Cezary Kaliszyk 3 lambda examples in FSet. In the last one regularize_term fails.
2009-12-07 Cezary Kaliszyk Handling of errors in lambda_prs_conv.
2009-12-07 Cezary Kaliszyk babs_prs
2009-12-07 Christian Urban clarified the function examples
2009-12-07 Christian Urban first attempt to deal with Babs in regularise and cleaning (not yet working)
2009-12-07 Christian Urban isabelle make tests all examples
2009-12-07 Cezary Kaliszyk merge
2009-12-07 Cezary Kaliszyk make_inst for lambda_prs where the second quotient is not identity.
2009-12-07 Christian Urban added "end" to each example theory
2009-12-07 Cezary Kaliszyk List moved after QuotMain
2009-12-07 Christian Urban cleaning
2009-12-07 Christian Urban final move
2009-12-07 Christian Urban directory re-arrangement
2009-12-07 Cezary Kaliszyk inj_repabs_tac handles Babs now.
2009-12-07 Cezary Kaliszyk Fix of regularize for babs and proof of babs_rsp.
2009-12-07 Cezary Kaliszyk Using pair_prs; debugging the error in regularize of a lambda.
2009-12-07 Cezary Kaliszyk QuotProd with product_quotient and a 3 respects and preserves lemmas.
2009-12-07 Cezary Kaliszyk merge
2009-12-07 Cezary Kaliszyk 3 new example thms in MyInt; reveal problems with handling of lambdas; regularize fails with "Loose Bound".
2009-12-07 Christian Urban simplified the regularize simproc
2009-12-07 Christian Urban now simpler regularize_tac with added solver works
2009-12-07 Christian Urban removed usage of HOL_basic_ss by using a slighly extended version of empty_ss
2009-12-06 Christian Urban merged
2009-12-06 Christian Urban fixed examples
2009-12-06 Cezary Kaliszyk Fix IntEx2 for equiv_list
2009-12-06 Christian Urban merged
2009-12-06 Christian Urban working state again
2009-12-06 Christian Urban added a theorem list for equivalence theorems
2009-12-06 Cezary Kaliszyk Merge
2009-12-06 Cezary Kaliszyk Name changes.
2009-12-06 Cezary Kaliszyk Solved all quotient goals.
2009-12-06 Christian Urban updated Isabelle and deleted mono rules
2009-12-06 Christian Urban more tuning of the code
2009-12-06 Christian Urban puting code in separate sections
2009-12-06 Cezary Kaliszyk Handle 'find_qt_asm' exception. Now all inj_repabs_goals should be solved automatically.
2009-12-06 Cezary Kaliszyk merge
2009-12-06 Cezary Kaliszyk Simpler definition code that works with any type maps.
2009-12-06 Christian Urban working on lambda_prs with examples; polished code of clean_tac
2009-12-06 Christian Urban renamed lambda_allex_prs
2009-12-06 Christian Urban added more to IntEx2
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 Definitions folded first.
2009-12-05 Cezary Kaliszyk Used symmetric definitions. Moved quotient_rsp to QuotMain.
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 Christian Urban further cleaning
2009-12-05 Cezary Kaliszyk Merge
2009-12-05 Cezary Kaliszyk Added nil_rsp and cons_rsp to quotient_rsp; simplified IntEx.
2009-12-05 Christian Urban simplified inj_repabs_trm
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 tuned code
2009-12-04 Christian Urban merged
2009-12-04 Christian Urban not yet quite functional treatment of constants
2009-12-04 Cezary Kaliszyk Changed FOCUS to SUBGOAL in rep_abs_rsp_tac; another 20% speedup :)
2009-12-04 Cezary Kaliszyk Changing FOCUS to CSUBGOAL (part 1)
2009-12-04 Cezary Kaliszyk abs_rep as ==
2009-12-04 Cezary Kaliszyk Cleaning the Quotients file
2009-12-04 Cezary Kaliszyk Minor renames and moving
2009-12-04 Cezary Kaliszyk Cleaning/review of QuotScript.
2009-12-04 Cezary Kaliszyk More cleaning
2009-12-04 Cezary Kaliszyk more name cleaning and removing
2009-12-04 Cezary Kaliszyk More code cleaning and renaming: moved rsp and prs lemmas from Int to QuotList
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
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 Manually finished LF induction.
2009-11-28 Cezary Kaliszyk Moved fast instantiation to QuotMain
2009-11-28 Cezary Kaliszyk LFex proof a bit further.
2009-11-28 Cezary Kaliszyk merge
2009-11-28 Cezary Kaliszyk Looking at repabs proof in LF.
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 fixed examples in IntEx and FSet
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 Cezary Kaliszyk Integrated Stefan's tactic and changed substs to simps with empty context.
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 Cezary Kaliszyk Merge
2009-11-27 Cezary Kaliszyk The magical code from Stefan, will need to be integrated in the Simproc.
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 Cleaning of LFex. Lambda_prs fails to unify in 2 places.
2009-11-27 Cezary Kaliszyk Recommit
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 Cezary Kaliszyk Minor cleaning
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 deleted obsolete qenv 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 introduced a new property for Ball and ===> on the left
2009-11-26 Christian Urban fixed QuotList
2009-11-26 Christian Urban changed left-res
2009-11-26 Cezary Kaliszyk Manually regularized akind_aty_atrm.induct
2009-11-26 Cezary Kaliszyk Playing with Monos in LFex.
2009-11-26 Cezary Kaliszyk Fixed FSet after merge.
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 Cezary Kaliszyk Merge
2009-11-25 Cezary Kaliszyk Finished manual lifting of list_induct_part :)
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 All examples work again.
2009-11-25 Cezary Kaliszyk cleaning in MyInt
2009-11-25 Cezary Kaliszyk lambda_prs and cleaning the existing examples.
2009-11-25 Christian Urban merged
2009-11-25 Christian Urban fixed the problem with generalising variables; at the moment it is quite a hack
2009-11-24 Cezary Kaliszyk Ho-matching failures...
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 Cezary Kaliszyk Conversion
2009-11-24 Cezary Kaliszyk The non-working procedure_tac.
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 Christian Urban explicit phases for the cleaning
2009-11-24 Cezary Kaliszyk Separate regularize_tac
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.
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 merged
2009-11-23 Christian Urban tuned some comments
2009-11-23 Cezary Kaliszyk Another not-typechecking regularized term.
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 Cezary Kaliszyk merge
2009-11-23 Cezary Kaliszyk lift_thm with a goal.
2009-11-23 Christian Urban slight change in code layout
2009-11-23 Cezary Kaliszyk Fixes for new code
2009-11-23 Cezary Kaliszyk Removing dead code
2009-11-23 Cezary Kaliszyk Move atomize_goal to QuotMain
2009-11-23 Cezary Kaliszyk Removed second implementation of Regularize/Inject from FSet.
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-23 Cezary Kaliszyk The other branch does not seem to work...
2009-11-23 Cezary Kaliszyk Fixes for recent changes.
2009-11-22 Christian Urban updated to Isabelle 22nd November
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 tuned
2009-11-21 Christian Urban tunded
2009-11-21 Christian Urban tuned
2009-11-21 Christian Urban flagged qenv-stuff as obsolete
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-13 Cezary Kaliszyk Still don't know how to do the proof automatically.
2009-11-13 Christian Urban added some tracing information to all phases of lifting to the function lift_thm
2009-11-12 Cezary Kaliszyk merge of the merge?
2009-11-12 Cezary Kaliszyk merged
2009-11-12 Christian Urban added a FIXME commment
2009-11-12 Christian Urban looking up data in quot_info works now (needs qualified string)
2009-11-12 Christian Urban changed the quotdata to be a symtab table (needs fixing)
2009-11-12 Christian Urban added a container for quotient constants (does not work yet though)
2009-11-11 Cezary Kaliszyk Lifting towards goal and manually finished the proof.
2009-11-11 Cezary Kaliszyk merge
2009-11-11 Cezary Kaliszyk Modifications while preparing the goal-directed version.
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-10 Cezary Kaliszyk Atomizing a "goal" theorems.
2009-11-10 Cezary Kaliszyk More code cleaning and commenting
2009-11-09 Cezary Kaliszyk Minor cleaning and removing of some 'handle _'.
2009-11-09 Cezary Kaliszyk Cleaning and commenting
2009-11-09 Cezary Kaliszyk Fixes for the other get_fun implementation.
2009-11-06 Christian Urban permutation lifting works now also
2009-11-06 Christian Urban merged
2009-11-06 Christian Urban updated to new Isabelle version and added a new example file
2009-11-06 Cezary Kaliszyk Minor changes
2009-11-06 Cezary Kaliszyk merge
2009-11-06 Cezary Kaliszyk fold_rsp
2009-11-06 Christian Urban tuned the code in quotient and quotient_def
2009-11-05 Cezary Kaliszyk More functionality for lifting list.cases and list.recs.
2009-11-05 Christian Urban merged
2009-11-05 Christian Urban removed typing information from get_fun in quotient_def; *potentially* dangerous
2009-11-05 Cezary Kaliszyk Remaining fixes for polymorphic types. map_append now lifts properly with 'a list and 'b list.
2009-11-05 Christian Urban removed Simplifier.context
2009-11-05 Christian Urban replaced check_term o parse_term by read_term
2009-11-05 Christian Urban merged
2009-11-05 Cezary Kaliszyk Infrastructure for polymorphic types
2009-11-04 Cezary Kaliszyk Two new tests for get_fun. Second one fails.
2009-11-04 Cezary Kaliszyk Type instantiation in regularize
2009-11-04 Cezary Kaliszyk Description of regularize
2009-11-04 Cezary Kaliszyk Experiments with lifting partially applied constants.
2009-11-04 Christian Urban more tuning
2009-11-04 Christian Urban slightly tuned
2009-11-04 Christian Urban merged
2009-11-04 Christian Urban separated the quotient_def into a separate file
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-04 Cezary Kaliszyk Lifting 'fold1.simps(2)' and some cleaning.
2009-11-03 Cezary Kaliszyk Playing with alpha_refl.
2009-11-03 Cezary Kaliszyk Alpha.induct now lifts automatically.
2009-11-03 Cezary Kaliszyk merge
2009-11-03 Cezary Kaliszyk applic_prs
2009-11-03 Christian Urban simplified the quotient_def code; type of the defined constant must now be given; for-part eliminated
2009-11-03 Cezary Kaliszyk Automatic FORALL_PRS. 'list.induct' lifts automatically. Faster ALLEX_RSP
2009-11-03 Cezary Kaliszyk merge
2009-11-03 Cezary Kaliszyk Preparing infrastructure for general FORALL_PRS
2009-11-02 Christian Urban split quotient.ML into two files
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-11-02 Cezary Kaliszyk Optimization
2009-11-02 Cezary Kaliszyk Map does not fully work yet.
2009-11-02 Cezary Kaliszyk Fixed quotdata_lookup.
2009-11-02 Christian Urban fixed problem with maps_update
2009-11-02 Christian Urban merged
2009-11-02 Christian Urban fixed the problem with types in map
2009-10-31 Cezary Kaliszyk Automatic computation of application preservation and manually finished "alpha.induct". Slow...
2009-10-30 Cezary Kaliszyk Regularize for equalities and a better tactic. "alpha.cases" now lifts.
2009-10-30 Cezary Kaliszyk Regularization
2009-10-30 Christian Urban merged
2009-10-30 Christian Urban added some facts about fresh and support of lam
2009-10-30 Cezary Kaliszyk Finally merged the code of the versions of regularize and tested examples.
2009-10-30 Cezary Kaliszyk Lemmas about fv.
2009-10-30 Christian Urban changed the order of rfv and reformulated a3 with rfv
2009-10-30 Christian Urban merged
2009-10-30 Christian Urban not sure what changed here
2009-10-30 Christian Urban added fv-function
2009-10-30 Cezary Kaliszyk The proper real_alpha
2009-10-30 Cezary Kaliszyk Finding applications and duplicates filtered out in abstractions
2009-10-30 Cezary Kaliszyk Cleaning also in Lam
2009-10-30 Cezary Kaliszyk Cleaning of the interface to lift.
2009-10-29 Cezary Kaliszyk Tried manually lifting real_alpha
2009-10-29 Cezary Kaliszyk More tests in Lam
2009-10-29 Cezary Kaliszyk Cleaning of 'map id' and 'prod_fun id id' in lower_defs.
2009-10-29 Cezary Kaliszyk Using subst for identity definition.
2009-10-29 Cezary Kaliszyk Lifting of the 3 lemmas in LamEx
2009-10-29 Cezary Kaliszyk Fixed wrong CARD definition and removed the "Does not work anymore" comment.
2009-10-29 Christian Urban merged
2009-10-28 Christian Urban updated some definitions; had to give sometimes different names; somewhere I introduced a bug, since not everything is working anymore (needs fixing!)
2009-10-28 Christian Urban ported all constant definitions to new scheme
2009-10-28 Christian Urban fixed the definition of alpha; this *breaks* some of the experiments
2009-10-28 Cezary Kaliszyk disambiguate ===> syntax
2009-10-28 Cezary Kaliszyk More cleaning in Lam code
2009-10-28 Cezary Kaliszyk cleaned FSet
2009-10-28 Cezary Kaliszyk Some cleaning
2009-10-28 Cezary Kaliszyk Cleaning the unnecessary theorems in 'IntEx'.
2009-10-28 Cezary Kaliszyk Fix also in the general procedure.
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 merged
2009-10-28 Christian Urban added infrastructure for defining lifted constants
2009-10-28 Cezary Kaliszyk First experiments with Lambda
2009-10-28 Cezary Kaliszyk Fixed mistake in const generation, will postpone this.
2009-10-28 Cezary Kaliszyk More finshed proofs and cleaning
2009-10-28 Cezary Kaliszyk Proof of append_rsp
2009-10-28 Christian Urban merged
2009-10-28 Christian Urban added a function for matching types
2009-10-27 Cezary Kaliszyk Manual conversion of equality to equivalence allows lifting append_assoc.
2009-10-27 Cezary Kaliszyk Simplfied interface to repabs_injection.
2009-10-27 Cezary Kaliszyk map_append lifted automatically.
2009-10-27 Cezary Kaliszyk Manually lifted Map_Append.
2009-10-27 Cezary Kaliszyk Merged
2009-10-27 Cezary Kaliszyk Fixed APPLY_RSP vs Cong in the InjRepAbs tactic.
2009-10-27 Christian Urban tuned
2009-10-27 Christian Urban merged
2009-10-27 Christian Urban added equiv-thm to the quot_info
2009-10-27 Cezary Kaliszyk Simplifying FSet with new functions.
2009-10-27 Christian Urban added an example about lambda-terms
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
(0) -480 +480 +1000 tip