IntEx.thy
Sat, 28 Nov 2009 14:45:22 +0100 Christian Urban removed old inj_repabs_tac; kept only the one with (selective) debugging information
Sat, 28 Nov 2009 14:33:04 +0100 Christian Urban renamed r_mk_comb_tac to inj_repabs_tac
Sat, 28 Nov 2009 05:43:18 +0100 Cezary Kaliszyk Merged and tested that all works.
Sat, 28 Nov 2009 05:29:30 +0100 Cezary Kaliszyk Finished and tested the new regularize
Sat, 28 Nov 2009 04:46:03 +0100 Christian Urban fixed examples in IntEx and FSet
Sat, 28 Nov 2009 04:37:04 +0100 Christian Urban fixed previous commit
Sat, 28 Nov 2009 02:54:24 +0100 Christian Urban annotated a proof with all steps and simplified LAMBDA_RES_TAC
Fri, 27 Nov 2009 10:04:49 +0100 Cezary Kaliszyk Simplifying arguments; got rid of trans2_thm.
Fri, 27 Nov 2009 08:15:23 +0100 Cezary Kaliszyk Removing arguments of tactics: absrep, rel_refl, reps_same are computed.
Fri, 27 Nov 2009 07:00:14 +0100 Cezary Kaliszyk Minor cleaning
Fri, 27 Nov 2009 02:55:56 +0100 Christian Urban introduced a separate lemma for id_simps
Fri, 27 Nov 2009 02:35:50 +0100 Christian Urban deleted obsolete qenv code
Fri, 27 Nov 2009 02:23:49 +0100 Christian Urban renamed REGULARIZE to be regularize
Wed, 25 Nov 2009 21:48:32 +0100 Cezary Kaliszyk applic_prs
Wed, 25 Nov 2009 11:41:42 +0100 Cezary Kaliszyk Removed unused things from QuotMain.
Wed, 25 Nov 2009 10:39:53 +0100 Cezary Kaliszyk cleaning in MyInt
Wed, 25 Nov 2009 03:45:44 +0100 Christian Urban fixed the problem with generalising variables; at the moment it is quite a hack
Tue, 24 Nov 2009 15:15:10 +0100 Christian Urban added a prepare_tac
Tue, 24 Nov 2009 14:19:54 +0100 Cezary Kaliszyk Moved cleaning to QuotMain
Tue, 24 Nov 2009 14:16:57 +0100 Cezary Kaliszyk New cleaning tactic
Tue, 24 Nov 2009 13:46:36 +0100 Christian Urban explicit phases for the cleaning
Tue, 24 Nov 2009 01:36:50 +0100 Christian Urban addded a tactic, which sets up the three goals of the `algorithm'
Mon, 23 Nov 2009 20:10:39 +0100 Cezary Kaliszyk Finished temporary goal-directed lift_theorem wrapper.
Mon, 23 Nov 2009 15:47:14 +0100 Cezary Kaliszyk Fixes for atomize
Mon, 23 Nov 2009 15:08:09 +0100 Cezary Kaliszyk lift_thm with a goal.
Mon, 23 Nov 2009 14:40:53 +0100 Cezary Kaliszyk Fixes for new code
Mon, 23 Nov 2009 13:55:31 +0100 Cezary Kaliszyk Moved new repabs_inj code to QuotMain
Mon, 23 Nov 2009 13:46:14 +0100 Cezary Kaliszyk New repabs behaves the same way as old one.
Mon, 23 Nov 2009 13:24:12 +0100 Christian Urban code review with Cezary
Sun, 22 Nov 2009 00:01:06 +0100 Christian Urban a little tuning of comments
Sat, 21 Nov 2009 23:23:01 +0100 Christian Urban slight tuning
Sat, 21 Nov 2009 14:45:25 +0100 Christian Urban some debugging code, but cannot find the place where the cprems_of exception is raised
Sat, 21 Nov 2009 14:18:31 +0100 Christian Urban tried to prove the repabs_inj lemma, but failed for the moment
Sat, 21 Nov 2009 13:14:35 +0100 Christian Urban my first version of repabs injection
Sat, 21 Nov 2009 10:58:08 +0100 Christian Urban tunded
Sat, 21 Nov 2009 02:49:39 +0100 Christian Urban simplified get_fun so that it uses directly rty and qty, instead of qenv
Fri, 20 Nov 2009 13:03:01 +0100 Christian Urban started regularize of rtrm/qtrm version; looks quite promising
Thu, 19 Nov 2009 14:17:10 +0100 Christian Urban updated to new Isabelle
Wed, 18 Nov 2009 23:52:48 +0100 Christian Urban fixed the storage of qconst definitions
Thu, 12 Nov 2009 12:07:33 +0100 Christian Urban looking up data in quot_info works now (needs qualified string)
Thu, 12 Nov 2009 02:18:36 +0100 Christian Urban added a container for quotient constants (does not work yet though)
Wed, 11 Nov 2009 11:59:22 +0100 Christian Urban updated to new Theory_Data and to new Isabelle
Wed, 11 Nov 2009 10:22:47 +0100 Cezary Kaliszyk Removed 'Toplevel.program' for polyml 5.3
Thu, 05 Nov 2009 13:47:04 +0100 Christian Urban removed typing information from get_fun in quotient_def; *potentially* dangerous
Thu, 05 Nov 2009 09:55:21 +0100 Christian Urban merged
Wed, 04 Nov 2009 13:33:13 +0100 Cezary Kaliszyk Experiments with lifting partially applied constants.
Wed, 04 Nov 2009 11:08:05 +0100 Cezary Kaliszyk Experiments in Int
Wed, 04 Nov 2009 10:43:33 +0100 Christian Urban fixed definition of PLUS
Wed, 04 Nov 2009 10:31:20 +0100 Christian Urban simplified the quotient_def code
Tue, 03 Nov 2009 16:51:33 +0100 Christian Urban simplified the quotient_def code; type of the defined constant must now be given; for-part eliminated
Mon, 02 Nov 2009 18:16:19 +0100 Christian Urban slightly saner way of parsing the quotient_def
Mon, 02 Nov 2009 15:39:25 +0100 Christian Urban merged
Mon, 02 Nov 2009 15:38:49 +0100 Christian Urban changed Type.typ_match to Sign.typ_match
Mon, 02 Nov 2009 15:38:03 +0100 Cezary Kaliszyk Fixes after optimization and preparing for a general FORALL_PRS
Fri, 30 Oct 2009 11:25:29 +0100 Cezary Kaliszyk Cleaning of the interface to lift.
Wed, 28 Oct 2009 18:08:38 +0100 Cezary Kaliszyk disambiguate ===> syntax
Wed, 28 Oct 2009 16:16:38 +0100 Cezary Kaliszyk Cleaning the unnecessary theorems in 'IntEx'.
Wed, 28 Oct 2009 16:06:19 +0100 Cezary Kaliszyk merge
Wed, 28 Oct 2009 16:05:59 +0100 Cezary Kaliszyk Fixes
Wed, 28 Oct 2009 15:48:38 +0100 Christian Urban updated all definitions
less more (0) -60 tip