Quot/Examples/IntEx.thy
2009-12-24 Christian Urban made the quotient_type definition more like typedef; now type variables need to be explicitly given
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
2009-12-19 Christian Urban on suggestion of Tobias renamed "quotient_def" to "quotient_definition"; needs new keyword file
2009-12-19 Christian Urban renamed "quotient" command to "quotient_type"; needs new keyword file to be installed
2009-12-19 Christian Urban with "isabelle make keywords" you can create automatically a "quot" keywordfile, provided all Logics are in place
2009-12-19 Christian Urban avoided global "open"s - replaced by local "open"s
2009-12-17 Christian Urban moved the QuotMain code into two ML-files
2009-12-11 Cezary Kaliszyk New syntax for definitions.
2009-12-10 Cezary Kaliszyk Moved 'int_induct' to IntEx to keep IntEx2 being just theory of integers in order.
2009-12-09 Cezary Kaliszyk Different syntax for definitions that allows overloading and retrieving of definitions by matching whole constants.
2009-12-09 Cezary Kaliszyk Temporarily repeated fun_map_tac 4 times. Cleaning for all examples work.
2009-12-08 Christian Urban implemented cleaning strategy with fun_map.simps on non-bounded variables; still a few rough edges
2009-12-08 Christian Urban decoupled QuotProd from QuotMain and also started new cleaning strategy
2009-12-08 Christian Urban proper formulation of all preservation theorems
2009-12-08 Christian Urban chnaged syntax to "lifting theorem"
2009-12-08 Christian Urban changed names of attributes
2009-12-08 Christian Urban added methods for the lifting_tac and the other tacs
2009-12-08 Cezary Kaliszyk Another lambda example theorem proved. Seems it starts working properly.
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-07 Christian Urban tuning of the code
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 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 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 directory re-arrangement
less more (0) tip