Sun, 06 Dec 2009 04:03:08 +0100 |
Christian Urban |
working on lambda_prs with examples; polished code of clean_tac
|
file |
diff |
annotate
|
Sun, 06 Dec 2009 00:19:45 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Sun, 06 Dec 2009 00:13:35 +0100 |
Christian Urban |
added new example for Ints; regularise does not work in all instances
|
file |
diff |
annotate
|
Sat, 05 Dec 2009 23:26:08 +0100 |
Cezary Kaliszyk |
Proved foldl_rsp and ho_map_rsp
|
file |
diff |
annotate
|
Sat, 05 Dec 2009 22:38:42 +0100 |
Christian Urban |
moved all_prs and ex_prs out from the conversion into the simplifier
|
file |
diff |
annotate
|
Sat, 05 Dec 2009 22:05:09 +0100 |
Cezary Kaliszyk |
Added nil_rsp and cons_rsp to quotient_rsp; simplified IntEx.
|
file |
diff |
annotate
|
Sat, 05 Dec 2009 21:50:31 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Sat, 05 Dec 2009 21:47:48 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Sat, 05 Dec 2009 21:45:56 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Sat, 05 Dec 2009 21:44:01 +0100 |
Christian Urban |
simpler version of clean_tac
|
file |
diff |
annotate
|
Sat, 05 Dec 2009 21:45:39 +0100 |
Cezary Kaliszyk |
Handling of respects in the fast inj_repabs_tac; includes respects with quotient assumptions.
|
file |
diff |
annotate
|
Sat, 05 Dec 2009 21:28:24 +0100 |
Cezary Kaliszyk |
Solutions to IntEx tests.
|
file |
diff |
annotate
|
Sat, 05 Dec 2009 16:26:18 +0100 |
Christian Urban |
made some slight simplifications to the examples
|
file |
diff |
annotate
|
Sat, 05 Dec 2009 13:49:35 +0100 |
Christian Urban |
added three examples to IntEx for testing ideas - regularisation and injection seem to be not quite right yet
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 21:42:55 +0100 |
Christian Urban |
not yet quite functional treatment of constants
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 16:40:23 +0100 |
Cezary Kaliszyk |
More code cleaning and renaming: moved rsp and prs lemmas from Int to QuotList
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 15:50:57 +0100 |
Cezary Kaliszyk |
Even more name changes and cleaning
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 15:41:09 +0100 |
Cezary Kaliszyk |
More code cleaning and name changes
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 15:18:33 +0100 |
Cezary Kaliszyk |
More name changes
|
file |
diff |
annotate
|
Thu, 03 Dec 2009 15:03:31 +0100 |
Christian Urban |
removed quot argument...not all examples work anymore
|
file |
diff |
annotate
|
Thu, 03 Dec 2009 14:02:05 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Thu, 03 Dec 2009 14:00:43 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Thu, 03 Dec 2009 13:45:52 +0100 |
Cezary Kaliszyk |
Updated the examples
|
file |
diff |
annotate
|
Thu, 03 Dec 2009 11:34:34 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Thu, 03 Dec 2009 11:33:24 +0100 |
Christian Urban |
deleted some dead code
|
file |
diff |
annotate
|
Wed, 02 Dec 2009 23:31:30 +0100 |
Christian Urban |
deleted now obsolete argument rty everywhere
|
file |
diff |
annotate
|
Wed, 02 Dec 2009 17:15:36 +0100 |
Cezary Kaliszyk |
More experiments with higher order quotients and theorems with non-lifted constants.
|
file |
diff |
annotate
|
Tue, 01 Dec 2009 12:16:45 +0100 |
Cezary Kaliszyk |
Cleaning 'aps'.
|
file |
diff |
annotate
|
Mon, 30 Nov 2009 11:53:20 +0100 |
Cezary Kaliszyk |
Code cleaning.
|
file |
diff |
annotate
|
Sun, 29 Nov 2009 23:59:37 +0100 |
Christian Urban |
tried to improve the inj_repabs_trm function but left the new part commented out
|
file |
diff |
annotate
|
Sun, 29 Nov 2009 08:48:06 +0100 |
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.
|
file |
diff |
annotate
|
Sun, 29 Nov 2009 03:59:18 +0100 |
Christian Urban |
introduced a global list of respectfulness lemmas; the attribute is [quot_rsp]
|
file |
diff |
annotate
|
Sat, 28 Nov 2009 14:45:22 +0100 |
Christian Urban |
removed old inj_repabs_tac; kept only the one with (selective) debugging information
|
file |
diff |
annotate
|
Sat, 28 Nov 2009 14:33:04 +0100 |
Christian Urban |
renamed r_mk_comb_tac to inj_repabs_tac
|
file |
diff |
annotate
|
Sat, 28 Nov 2009 05:43:18 +0100 |
Cezary Kaliszyk |
Merged and tested that all works.
|
file |
diff |
annotate
|
Sat, 28 Nov 2009 05:29:30 +0100 |
Cezary Kaliszyk |
Finished and tested the new regularize
|
file |
diff |
annotate
|
Sat, 28 Nov 2009 04:46:03 +0100 |
Christian Urban |
fixed examples in IntEx and FSet
|
file |
diff |
annotate
|
Sat, 28 Nov 2009 04:37:04 +0100 |
Christian Urban |
fixed previous commit
|
file |
diff |
annotate
|
Sat, 28 Nov 2009 02:54:24 +0100 |
Christian Urban |
annotated a proof with all steps and simplified LAMBDA_RES_TAC
|
file |
diff |
annotate
|
Fri, 27 Nov 2009 10:04:49 +0100 |
Cezary Kaliszyk |
Simplifying arguments; got rid of trans2_thm.
|
file |
diff |
annotate
|
Fri, 27 Nov 2009 08:15:23 +0100 |
Cezary Kaliszyk |
Removing arguments of tactics: absrep, rel_refl, reps_same are computed.
|
file |
diff |
annotate
|
Fri, 27 Nov 2009 07:00:14 +0100 |
Cezary Kaliszyk |
Minor cleaning
|
file |
diff |
annotate
|
Fri, 27 Nov 2009 02:55:56 +0100 |
Christian Urban |
introduced a separate lemma for id_simps
|
file |
diff |
annotate
|
Fri, 27 Nov 2009 02:35:50 +0100 |
Christian Urban |
deleted obsolete qenv code
|
file |
diff |
annotate
|
Fri, 27 Nov 2009 02:23:49 +0100 |
Christian Urban |
renamed REGULARIZE to be regularize
|
file |
diff |
annotate
|
Wed, 25 Nov 2009 21:48:32 +0100 |
Cezary Kaliszyk |
applic_prs
|
file |
diff |
annotate
|
Wed, 25 Nov 2009 11:41:42 +0100 |
Cezary Kaliszyk |
Removed unused things from QuotMain.
|
file |
diff |
annotate
|
Wed, 25 Nov 2009 10:39:53 +0100 |
Cezary Kaliszyk |
cleaning in MyInt
|
file |
diff |
annotate
|
Wed, 25 Nov 2009 03:45:44 +0100 |
Christian Urban |
fixed the problem with generalising variables; at the moment it is quite a hack
|
file |
diff |
annotate
|
Tue, 24 Nov 2009 15:15:10 +0100 |
Christian Urban |
added a prepare_tac
|
file |
diff |
annotate
|
Tue, 24 Nov 2009 14:19:54 +0100 |
Cezary Kaliszyk |
Moved cleaning to QuotMain
|
file |
diff |
annotate
|
Tue, 24 Nov 2009 14:16:57 +0100 |
Cezary Kaliszyk |
New cleaning tactic
|
file |
diff |
annotate
|
Tue, 24 Nov 2009 13:46:36 +0100 |
Christian Urban |
explicit phases for the cleaning
|
file |
diff |
annotate
|
Tue, 24 Nov 2009 01:36:50 +0100 |
Christian Urban |
addded a tactic, which sets up the three goals of the `algorithm'
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 20:10:39 +0100 |
Cezary Kaliszyk |
Finished temporary goal-directed lift_theorem wrapper.
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 15:47:14 +0100 |
Cezary Kaliszyk |
Fixes for atomize
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 15:08:09 +0100 |
Cezary Kaliszyk |
lift_thm with a goal.
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 14:40:53 +0100 |
Cezary Kaliszyk |
Fixes for new code
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 13:55:31 +0100 |
Cezary Kaliszyk |
Moved new repabs_inj code to QuotMain
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 13:46:14 +0100 |
Cezary Kaliszyk |
New repabs behaves the same way as old one.
|
file |
diff |
annotate
|