FSet.thy
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 Cezary Kaliszyk Conversion
2009-11-24 Cezary Kaliszyk The non-working procedure_tac.
2009-11-24 Cezary Kaliszyk Fixes to the tactic after quotient_tac changed.
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-23 Christian Urban fixed the error by a temporary fix (the data of the eqivalence relation should be only its name)
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 Move atomize_goal to QuotMain
2009-11-23 Cezary Kaliszyk Removed second implementation of Regularize/Inject from FSet.
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-13 Cezary Kaliszyk Still don't know how to do the proof automatically.
2009-11-12 Cezary Kaliszyk merged
2009-11-11 Cezary Kaliszyk Lifting towards goal and manually finished the proof.
2009-11-11 Cezary Kaliszyk Removed 'Toplevel.program' for polyml 5.3
2009-11-10 Cezary Kaliszyk Atomizing a "goal" theorems.
2009-11-09 Cezary Kaliszyk Fixes for the other get_fun implementation.
2009-11-06 Cezary Kaliszyk Minor changes
2009-11-06 Cezary Kaliszyk fold_rsp
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 Cezary Kaliszyk Infrastructure for polymorphic types
2009-11-04 Cezary Kaliszyk Experiments in Int
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 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-02 Cezary Kaliszyk Fixes after optimization and preparing for a general FORALL_PRS
2009-11-02 Cezary Kaliszyk Map does not fully work yet.
2009-11-02 Cezary Kaliszyk Fixed quotdata_lookup.
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 Cezary Kaliszyk Finally merged the code of the versions of regularize and tested examples.
2009-10-30 Christian Urban not sure what changed here
2009-10-30 Cezary Kaliszyk Finding applications and duplicates filtered out in abstractions
2009-10-30 Cezary Kaliszyk Cleaning of the interface to lift.
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 Cezary Kaliszyk disambiguate ===> syntax
2009-10-28 Cezary Kaliszyk cleaned FSet
2009-10-28 Cezary Kaliszyk Some cleaning
2009-10-28 Cezary Kaliszyk Fixes
2009-10-28 Christian Urban merged
2009-10-28 Christian Urban added infrastructure for defining lifted constants
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 Fixed APPLY_RSP vs Cong in the InjRepAbs tactic.
2009-10-27 Cezary Kaliszyk Simplifying FSet with new functions.
2009-10-26 Cezary Kaliszyk Simplifying Int and Working on map
2009-10-26 Cezary Kaliszyk Finished the code for adding lower defs, and more things moved to QuotMain
2009-10-26 Cezary Kaliszyk Making all the definitions from the original ones
2009-10-26 Cezary Kaliszyk Cleaning and fixing.
2009-10-24 Christian Urban proved the two lemmas in QuotScript (reformulated them without leading forall)
2009-10-24 Christian Urban changed the definitions of liftet constants to use fun_maps
2009-10-24 Cezary Kaliszyk Finally lifted induction, with some manually added simplification lemmas.
2009-10-24 cek Merge
2009-10-24 Cezary Kaliszyk Preparing infrastructire for LAMBDA_PRS
2009-10-24 Christian Urban moved the map_funs setup into QuotMain
2009-10-24 Cezary Kaliszyk Finally completely lift the previously lifted theorems + clean some old stuff
2009-10-24 Cezary Kaliszyk More infrastructure for automatic lifting of theorems lifted before
2009-10-24 Cezary Kaliszyk More infrastructure for automatic lifting of theorems lifted before
2009-10-24 cek Cleaning the mess
2009-10-24 cek Merge
2009-10-24 cek Better tactic and simplified the proof further
2009-10-23 Christian Urban fixed problem with incorrect ABS/REP name
2009-10-23 Cezary Kaliszyk Stronger tactic, simpler proof.
2009-10-23 Cezary Kaliszyk Split Finite Set example into separate file
less more (0) tip