Wed, 02 Dec 2009 14:37:21 +0100 |
Cezary Kaliszyk |
Lifting to 2 different types :)
|
file |
diff |
annotate
|
Wed, 02 Dec 2009 14:11:46 +0100 |
Cezary Kaliszyk |
New APPLY_RSP which finally does automatic partial lifting :). Doesn't support same relation yet.
|
file |
diff |
annotate
|
Wed, 02 Dec 2009 12:07:54 +0100 |
Cezary Kaliszyk |
Fixed unlam for non-abstractions and updated list_induct_part proof.
|
file |
diff |
annotate
|
Wed, 02 Dec 2009 11:30:40 +0100 |
Cezary Kaliszyk |
Removed the use of 'rty' from APPLY_RSP, finally LF proofs go automatically.
|
file |
diff |
annotate
|
Wed, 02 Dec 2009 10:56:35 +0100 |
Cezary Kaliszyk |
The conversion approach works.
|
file |
diff |
annotate
|
Wed, 02 Dec 2009 10:30:20 +0100 |
Cezary Kaliszyk |
Trying a conversion based approach.
|
file |
diff |
annotate
|
Wed, 02 Dec 2009 09:23:48 +0100 |
Cezary Kaliszyk |
A bit of progress; but the object-logic vs meta-logic distinction is troublesome.
|
file |
diff |
annotate
|
Tue, 01 Dec 2009 19:18:43 +0100 |
Cezary Kaliszyk |
back in working state
|
file |
diff |
annotate
|
Tue, 01 Dec 2009 19:01:51 +0100 |
Cezary Kaliszyk |
clean
|
file |
diff |
annotate
|
Tue, 01 Dec 2009 18:41:01 +0100 |
Christian Urban |
added a make_inst test
|
file |
diff |
annotate
|
Tue, 01 Dec 2009 18:22:48 +0100 |
Cezary Kaliszyk |
Transformation of QUOT_TRUE assumption by any given function
|
file |
diff |
annotate
|
Tue, 01 Dec 2009 16:27:42 +0100 |
Christian Urban |
QUOT_TRUE joke
|
file |
diff |
annotate
|
Tue, 01 Dec 2009 14:04:00 +0100 |
Cezary Kaliszyk |
more cleaning
|
file |
diff |
annotate
|
Tue, 01 Dec 2009 12:16:45 +0100 |
Cezary Kaliszyk |
Cleaning 'aps'.
|
file |
diff |
annotate
|
Mon, 30 Nov 2009 15:32:14 +0100 |
Cezary Kaliszyk |
clean_tac rewrites the definitions the other way
|
file |
diff |
annotate
|
Mon, 30 Nov 2009 12:14:20 +0100 |
Cezary Kaliszyk |
More code cleaning
|
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 09:38:07 +0100 |
Cezary Kaliszyk |
Removed unnecessary HOL_ss which proved one of the subgoals.
|
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 19:14:12 +0100 |
Christian Urban |
improved pattern matching inside the inj_repabs_tacs
|
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 13:54:48 +0100 |
Christian Urban |
renamed LAMBDA_RES_TAC and WEAK_LAMBDA_RES_TAC to lower case names
|
file |
diff |
annotate
|
Sat, 28 Nov 2009 05:49:16 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Sat, 28 Nov 2009 05:47:13 +0100 |
Christian Urban |
more simplification
|
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 02:54:24 +0100 |
Christian Urban |
annotated a proof with all steps and simplified LAMBDA_RES_TAC
|
file |
diff |
annotate
|
Fri, 27 Nov 2009 13:59:52 +0100 |
Christian Urban |
replaced FIRST' (map rtac list) with resolve_tac list
|
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
|
Thu, 26 Nov 2009 20:32:56 +0100 |
Cezary Kaliszyk |
Merge Again
|
file |
diff |
annotate
|
Thu, 26 Nov 2009 20:32:33 +0100 |
Cezary Kaliszyk |
Merged
|
file |
diff |
annotate
|
Thu, 26 Nov 2009 20:18:36 +0100 |
Christian Urban |
tuned comments
|
file |
diff |
annotate
|
Thu, 26 Nov 2009 19:51:31 +0100 |
Christian Urban |
some diagnostic code for r_mk_comb
|
file |
diff |
annotate
|
Thu, 26 Nov 2009 16:23:24 +0100 |
Christian Urban |
introduced a new property for Ball and ===> on the left
|
file |
diff |
annotate
|
Thu, 26 Nov 2009 13:46:00 +0100 |
Christian Urban |
changed left-res
|
file |
diff |
annotate
|
Thu, 26 Nov 2009 10:32:31 +0100 |
Cezary Kaliszyk |
Fixed FSet after merge.
|
file |
diff |
annotate
|
Thu, 26 Nov 2009 03:18:38 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Thu, 26 Nov 2009 02:31:00 +0100 |
Christian Urban |
test with monos
|
file |
diff |
annotate
|
Wed, 25 Nov 2009 21:48:32 +0100 |
Cezary Kaliszyk |
applic_prs
|
file |
diff |
annotate
|
Wed, 25 Nov 2009 15:20:10 +0100 |
Christian Urban |
reordered the code
|
file |
diff |
annotate
|
Wed, 25 Nov 2009 14:25:29 +0100 |
Cezary Kaliszyk |
Moved exception handling to QuotMain and cleaned FSet.
|
file |
diff |
annotate
|
Wed, 25 Nov 2009 14:15:34 +0100 |
Cezary Kaliszyk |
Finished manual lifting of list_induct_part :)
|
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:34:03 +0100 |
Cezary Kaliszyk |
lambda_prs and cleaning the existing examples.
|
file |
diff |
annotate
|
Wed, 25 Nov 2009 03:47:07 +0100 |
Christian Urban |
merged
|
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 20:13:16 +0100 |
Cezary Kaliszyk |
Ho-matching failures...
|
file |
diff |
annotate
|
Tue, 24 Nov 2009 17:00:53 +0100 |
Cezary Kaliszyk |
Conversion
|
file |
diff |
annotate
|
Tue, 24 Nov 2009 16:20:34 +0100 |
Cezary Kaliszyk |
The non-working procedure_tac.
|
file |
diff |
annotate
|
Tue, 24 Nov 2009 15:18:00 +0100 |
Cezary Kaliszyk |
Fixes to the tactic after quotient_tac changed.
|
file |
diff |
annotate
|
Tue, 24 Nov 2009 08:36:28 +0100 |
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.
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 23:09:03 +0100 |
Christian Urban |
fixed the error by a temporary fix (the data of the eqivalence relation should be only its name)
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 21:56:30 +0100 |
Cezary Kaliszyk |
Another not-typechecking regularized term.
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 21:48:44 +0100 |
Cezary Kaliszyk |
domain_type in regularizing equality
|
file |
diff |
annotate
|