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
|
Sat, 05 Dec 2009 00:06:27 +0100 |
Christian Urban |
tuned code
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 21:43:29 +0100 |
Christian Urban |
merged
|
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 19:47:58 +0100 |
Cezary Kaliszyk |
Changed FOCUS to SUBGOAL in rep_abs_rsp_tac; another 20% speedup :)
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 19:06:53 +0100 |
Cezary Kaliszyk |
Changing FOCUS to CSUBGOAL (part 1)
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 17:50:02 +0100 |
Cezary Kaliszyk |
Minor renames and moving
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 17:36:45 +0100 |
Cezary Kaliszyk |
Cleaning/review of QuotScript.
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 17:15:55 +0100 |
Cezary Kaliszyk |
More cleaning
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 16:53:11 +0100 |
Cezary Kaliszyk |
more name cleaning and removing
|
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 16:12:40 +0100 |
Cezary Kaliszyk |
Cleaning & Renaming coming from 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
|
Fri, 04 Dec 2009 14:35:36 +0100 |
Cezary Kaliszyk |
code cleaning and renaming
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 14:11:20 +0100 |
Cezary Kaliszyk |
merge
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 14:11:03 +0100 |
Cezary Kaliszyk |
Removed previous inj_repabs_tac
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 13:58:23 +0100 |
Christian Urban |
some tuning
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 12:21:15 +0100 |
Cezary Kaliszyk |
merge
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 12:20:49 +0100 |
Cezary Kaliszyk |
rep_abs_rsp_tac to replace the last use of instantiate_tac with matching and unification.
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 11:34:49 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 11:34:21 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 11:33:58 +0100 |
Cezary Kaliszyk |
Change equiv_trans2 to EQUALS_RSP, since we can prove it for any quotient type, not only for eqv relations.
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 11:06:43 +0100 |
Cezary Kaliszyk |
compose_tac instead of rtac to avoid unification; some code cleaning.
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 10:36:35 +0100 |
Cezary Kaliszyk |
Got to about 5 seconds for the longest proof. APPLY_RSP_TAC' solves the quotient internally without instantiation resulting in a faster proof.
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 10:12:17 +0100 |
Cezary Kaliszyk |
Using APPLY_RSP1; again a little bit faster.
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 09:33:32 +0100 |
Cezary Kaliszyk |
Fixes after big merge.
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 09:25:27 +0100 |
Cezary Kaliszyk |
The big merge; probably non-functional.
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 09:08:51 +0100 |
Cezary Kaliszyk |
Testing the new tactic everywhere
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 09:01:13 +0100 |
Cezary Kaliszyk |
First version of the deterministic rep-abs-inj-tac.
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 09:18:46 +0100 |
Cezary Kaliszyk |
Changing = to \<equiv> in case if we want to use simp.
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 09:10:31 +0100 |
Cezary Kaliszyk |
Even better: Completely got rid of the simps in both quotient_tac and inj_repabs_tac
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 08:19:56 +0100 |
Cezary Kaliszyk |
merge
|
file |
diff |
annotate
|
Fri, 04 Dec 2009 08:18:38 +0100 |
Cezary Kaliszyk |
Made your version work again with LIST_REL_EQ.
|
file |
diff |
annotate
|
Thu, 03 Dec 2009 19:06:14 +0100 |
Christian Urban |
the error occurs in APPLY_RSP_TAC where the wrong quotient (for LIST_REL) is applied
|
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 13:59:53 +0100 |
Christian Urban |
first version of internalised quotient theorems; added FIXME-TODO
|
file |
diff |
annotate
|
Thu, 03 Dec 2009 11:40:10 +0100 |
Christian Urban |
further dead code
|
file |
diff |
annotate
|
Thu, 03 Dec 2009 13:56:59 +0100 |
Cezary Kaliszyk |
Reintroduced varifyT; we still need it for permutation definition.
|
file |
diff |
annotate
|
Thu, 03 Dec 2009 12:33:05 +0100 |
Cezary Kaliszyk |
Fixed previous mistake
|
file |
diff |
annotate
|
Thu, 03 Dec 2009 12:31:05 +0100 |
Cezary Kaliszyk |
defs used automatically by clean_tac
|
file |
diff |
annotate
|
Thu, 03 Dec 2009 11:58:46 +0100 |
Cezary Kaliszyk |
removing unused code
|
file |
diff |
annotate
|
Thu, 03 Dec 2009 11:33:24 +0100 |
Christian Urban |
deleted some dead code
|
file |
diff |
annotate
|
Thu, 03 Dec 2009 11:28:19 +0100 |
Cezary Kaliszyk |
Included all_prs and ex_prs in the lambda_prs conversion.
|
file |
diff |
annotate
|
Thu, 03 Dec 2009 02:53:54 +0100 |
Christian Urban |
further simplification
|
file |
diff |
annotate
|
Thu, 03 Dec 2009 02:18:21 +0100 |
Christian Urban |
simplified lambda_prs_conv
|
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 23:11:50 +0100 |
Christian Urban |
deleted tests at the beginning of QuotMain
|
file |
diff |
annotate
|
Wed, 02 Dec 2009 20:54:59 +0100 |
Cezary Kaliszyk |
Experiments with OPTION_map
|
file |
diff |
annotate
|
Wed, 02 Dec 2009 17:16:44 +0100 |
Cezary Kaliszyk |
merge
|
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
|
Wed, 02 Dec 2009 16:12:41 +0100 |
Christian Urban |
merged
|
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 07:21:10 +0100 |
Cezary Kaliszyk |
Added tactic for dealing with QUOT_TRUE and introducing QUOT_TRUE.
|
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:51:14 +0100 |
Christian Urban |
fixed previous commit
|
file |
diff |
annotate
|
Tue, 01 Dec 2009 18:48:52 +0100 |
Christian Urban |
fixed problems with FOCUS
|
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:08:56 +0100 |
Cezary Kaliszyk |
Removed last HOL_ss
|
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:40:22 +0100 |
Cezary Kaliszyk |
merge
|
file |
diff |
annotate
|
Mon, 30 Nov 2009 15:36:49 +0100 |
Christian Urban |
cleaned inj_regabs_trm
|
file |
diff |
annotate
|
Mon, 30 Nov 2009 15:33:06 +0100 |
Cezary Kaliszyk |
merge
|
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 13:58:05 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Mon, 30 Nov 2009 12:26:08 +0100 |
Christian Urban |
added facilities to get all stored quotient data (equiv thms etc)
|
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
|
Mon, 30 Nov 2009 10:16:10 +0100 |
Cezary Kaliszyk |
Commented clean-tac
|
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 17:47:37 +0100 |
Christian Urban |
started functions for qid-insertion and fixed a bug in regularise
|
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
|
Sun, 29 Nov 2009 02:51:42 +0100 |
Christian Urban |
tuned
|
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 18:49:39 +0100 |
Christian Urban |
selective debugging of the inj_repabs_tac (at the moment for step 3 and 4 debugging information is printed)
|
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 14:15:05 +0100 |
Christian Urban |
tuning
|
file |
diff |
annotate
|
Sat, 28 Nov 2009 14:03:01 +0100 |
Christian Urban |
tuned comments
|
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 08:04:23 +0100 |
Cezary Kaliszyk |
Moved fast instantiation to QuotMain
|
file |
diff |
annotate
|
Sat, 28 Nov 2009 05:53:31 +0100 |
Christian Urban |
further proper merge
|
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 05:09:22 +0100 |
Christian Urban |
more tuning of the repabs-tactics
|
file |
diff |
annotate
|
Sat, 28 Nov 2009 04:37:30 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Sat, 28 Nov 2009 04:37:04 +0100 |
Christian Urban |
fixed previous commit
|
file |
diff |
annotate
|
Sat, 28 Nov 2009 04:02:54 +0100 |
Cezary Kaliszyk |
Cleaned all lemmas about regularisation of Ball and Bex and moved in one place. Second Ball simprox.
|
file |
diff |
annotate
|
Sat, 28 Nov 2009 03:17:22 +0100 |
Cezary Kaliszyk |
Merged comment
|
file |
diff |
annotate
|
Sat, 28 Nov 2009 03:06:22 +0100 |
Christian Urban |
some slight tuning of the apply-tactic
|
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:16:16 +0100 |
Cezary Kaliszyk |
More cleaning in QuotMain, identity handling.
|
file |
diff |
annotate
|
Fri, 27 Nov 2009 04:02:20 +0100 |
Christian Urban |
tuned
|
file |
diff |
annotate
|
Fri, 27 Nov 2009 03:56:18 +0100 |
Christian Urban |
some tuning
|
file |
diff |
annotate
|
Fri, 27 Nov 2009 03:33:30 +0100 |
Christian Urban |
simplified gen_frees_tac and properly named abstracted variables
|
file |
diff |
annotate
|
Fri, 27 Nov 2009 02:58:28 +0100 |
Christian Urban |
removed CHANGED'
|
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:45:54 +0100 |
Christian Urban |
renamed inj_REPABS to inj_repabs_trm
|
file |
diff |
annotate
|
Fri, 27 Nov 2009 02:44:11 +0100 |
Christian Urban |
tuned comments and moved slightly some code
|
file |
diff |
annotate
|
Fri, 27 Nov 2009 02:23:49 +0100 |
Christian Urban |
renamed REGULARIZE to be regularize
|
file |
diff |
annotate
|
Thu, 26 Nov 2009 21:16:59 +0100 |
Christian Urban |
more tuning
|
file |
diff |
annotate
|
Thu, 26 Nov 2009 21:04:17 +0100 |
Christian Urban |
deleted get_fun_old and stuff
|
file |
diff |
annotate
|
Thu, 26 Nov 2009 21:01:53 +0100 |
Christian Urban |
recommited changes of comments
|
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 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:43:12 +0100 |
Christian Urban |
polishing
|
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 12:27:28 +0100 |
Christian Urban |
comments tuning and slight reordering
|
file |
diff |
annotate
|
Wed, 25 Nov 2009 11:59:49 +0100 |
Cezary Kaliszyk |
Merge
|
file |
diff |
annotate
|
Wed, 25 Nov 2009 11:58:56 +0100 |
Cezary Kaliszyk |
More moving from QuotMain to UnusedQuotMain
|
file |
diff |
annotate
|
Wed, 25 Nov 2009 11:46:59 +0100 |
Christian Urban |
deleted some obsolete diagnostic code
|
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: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 19:09:29 +0100 |
Christian Urban |
changed unification to matching
|
file |
diff |
annotate
|
Tue, 24 Nov 2009 18:13:57 +0100 |
Christian Urban |
unification
|
file |
diff |
annotate
|
Tue, 24 Nov 2009 18:13:18 +0100 |
Cezary Kaliszyk |
Lambda & SOLVED' for new quotient_tac
|
file |
diff |
annotate
|
Tue, 24 Nov 2009 17:35:31 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Tue, 24 Nov 2009 16:10:31 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Tue, 24 Nov 2009 15:31:29 +0100 |
Christian Urban |
use error instead of raising our own exception
|
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 15:15:33 +0100 |
Christian Urban |
merged
|
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:41:47 +0100 |
Cezary Kaliszyk |
TRY' for clean_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 12:25:04 +0100 |
Cezary Kaliszyk |
Separate regularize_tac
|
file |
diff |
annotate
|
Tue, 24 Nov 2009 08:35:04 +0100 |
Cezary Kaliszyk |
More fixes for inj_REPABS
|
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 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:59:57 +0100 |
Christian Urban |
tuned some comments
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 21:48:44 +0100 |
Cezary Kaliszyk |
domain_type in regularizing equality
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 21:12:16 +0100 |
Cezary Kaliszyk |
More theorems lifted in the goal-directed way.
|
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 16:13:19 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 16:12:50 +0100 |
Christian Urban |
a version of inj_REPABS (needs to be looked at again later)
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 15:47:14 +0100 |
Cezary Kaliszyk |
Fixes for atomize
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 15:02:48 +0100 |
Christian Urban |
slight change in code layout
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 14:32:11 +0100 |
Cezary Kaliszyk |
Removing dead code
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 14:16:41 +0100 |
Cezary Kaliszyk |
Move atomize_goal to QuotMain
|
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:24:12 +0100 |
Christian Urban |
code review with Cezary
|
file |
diff |
annotate
|
Sun, 22 Nov 2009 00:01:06 +0100 |
Christian Urban |
a little tuning of comments
|
file |
diff |
annotate
|
Sat, 21 Nov 2009 13:14:35 +0100 |
Christian Urban |
my first version of repabs injection
|
file |
diff |
annotate
|
Sat, 21 Nov 2009 11:16:48 +0100 |
Christian Urban |
tuned
|
file |
diff |
annotate
|
Sat, 21 Nov 2009 03:12:50 +0100 |
Christian Urban |
tuned
|
file |
diff |
annotate
|
Sat, 21 Nov 2009 02:49:39 +0100 |
Christian Urban |
simplified get_fun so that it uses directly rty and qty, instead of qenv
|
file |
diff |
annotate
|
Fri, 20 Nov 2009 13:03:01 +0100 |
Christian Urban |
started regularize of rtrm/qtrm version; looks quite promising
|
file |
diff |
annotate
|
Thu, 19 Nov 2009 14:17:10 +0100 |
Christian Urban |
updated to new Isabelle
|
file |
diff |
annotate
|
Fri, 13 Nov 2009 16:44:36 +0100 |
Christian Urban |
added some tracing information to all phases of lifting to the function lift_thm
|
file |
diff |
annotate
|
Thu, 12 Nov 2009 13:56:07 +0100 |
Cezary Kaliszyk |
merged
|
file |
diff |
annotate
|
Thu, 12 Nov 2009 02:54:40 +0100 |
Christian Urban |
changed the quotdata to be a symtab table (needs fixing)
|
file |
diff |
annotate
|
Thu, 12 Nov 2009 02:18:36 +0100 |
Christian Urban |
added a container for quotient constants (does not work yet though)
|
file |
diff |
annotate
|
Wed, 11 Nov 2009 18:49:46 +0100 |
Cezary Kaliszyk |
Modifications while preparing the goal-directed version.
|
file |
diff |
annotate
|
Tue, 10 Nov 2009 09:32:16 +0100 |
Cezary Kaliszyk |
More code cleaning and commenting
|
file |
diff |
annotate
|
Mon, 09 Nov 2009 15:40:43 +0100 |
Cezary Kaliszyk |
Minor cleaning and removing of some 'handle _'.
|
file |
diff |
annotate
|
Mon, 09 Nov 2009 15:23:33 +0100 |
Cezary Kaliszyk |
Cleaning and commenting
|
file |
diff |
annotate
|
Mon, 09 Nov 2009 13:47:46 +0100 |
Cezary Kaliszyk |
Fixes for the other get_fun implementation.
|
file |
diff |
annotate
|
Fri, 06 Nov 2009 19:26:08 +0100 |
Christian Urban |
updated to new Isabelle version and added a new example file
|
file |
diff |
annotate
|
Fri, 06 Nov 2009 09:48:37 +0100 |
Christian Urban |
tuned the code in quotient and quotient_def
|
file |
diff |
annotate
|
Thu, 05 Nov 2009 16:43:57 +0100 |
Cezary Kaliszyk |
More functionality for lifting list.cases and list.recs.
|
file |
diff |
annotate
|
Thu, 05 Nov 2009 13:36:46 +0100 |
Cezary Kaliszyk |
Remaining fixes for polymorphic types. map_append now lifts properly with 'a list and 'b list.
|
file |
diff |
annotate
|
Thu, 05 Nov 2009 10:46:54 +0100 |
Christian Urban |
removed Simplifier.context
|
file |
diff |
annotate
|
Thu, 05 Nov 2009 09:55:21 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Thu, 05 Nov 2009 09:38:34 +0100 |
Cezary Kaliszyk |
Infrastructure for polymorphic types
|
file |
diff |
annotate
|
Wed, 04 Nov 2009 15:27:32 +0100 |
Cezary Kaliszyk |
Type instantiation in regularize
|
file |
diff |
annotate
|
Wed, 04 Nov 2009 14:03:46 +0100 |
Cezary Kaliszyk |
Description of regularize
|
file |
diff |
annotate
|
Wed, 04 Nov 2009 11:59:15 +0100 |
Christian Urban |
separated the quotient_def into a separate file
|
file |
diff |
annotate
|
Wed, 04 Nov 2009 10:43:33 +0100 |
Christian Urban |
fixed definition of PLUS
|
file |
diff |
annotate
|
Wed, 04 Nov 2009 10:31:20 +0100 |
Christian Urban |
simplified the quotient_def code
|
file |
diff |
annotate
|
Wed, 04 Nov 2009 09:52:31 +0100 |
Cezary Kaliszyk |
Lifting 'fold1.simps(2)' and some cleaning.
|
file |
diff |
annotate
|
Tue, 03 Nov 2009 17:30:43 +0100 |
Cezary Kaliszyk |
merge
|
file |
diff |
annotate
|
Tue, 03 Nov 2009 17:30:27 +0100 |
Cezary Kaliszyk |
applic_prs
|
file |
diff |
annotate
|
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
|
file |
diff |
annotate
|
Tue, 03 Nov 2009 16:17:19 +0100 |
Cezary Kaliszyk |
Automatic FORALL_PRS. 'list.induct' lifts automatically. Faster ALLEX_RSP
|
file |
diff |
annotate
|
Mon, 02 Nov 2009 18:26:55 +0100 |
Christian Urban |
split quotient.ML into two files
|
file |
diff |
annotate
|
Mon, 02 Nov 2009 18:16:19 +0100 |
Christian Urban |
slightly saner way of parsing the quotient_def
|
file |
diff |
annotate
|
Mon, 02 Nov 2009 15:38:49 +0100 |
Christian Urban |
changed Type.typ_match to Sign.typ_match
|
file |
diff |
annotate
|
Mon, 02 Nov 2009 14:57:56 +0100 |
Cezary Kaliszyk |
Optimization
|
file |
diff |
annotate
|
Mon, 02 Nov 2009 11:15:26 +0100 |
Cezary Kaliszyk |
Fixed quotdata_lookup.
|
file |
diff |
annotate
|
Mon, 02 Nov 2009 09:39:29 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Mon, 02 Nov 2009 09:33:48 +0100 |
Christian Urban |
fixed the problem with types in map
|
file |
diff |
annotate
|
Sat, 31 Oct 2009 11:20:55 +0100 |
Cezary Kaliszyk |
Automatic computation of application preservation and manually finished "alpha.induct". Slow...
|
file |
diff |
annotate
|
Fri, 30 Oct 2009 19:03:53 +0100 |
Cezary Kaliszyk |
Regularize for equalities and a better tactic. "alpha.cases" now lifts.
|
file |
diff |
annotate
|
Fri, 30 Oct 2009 18:31:06 +0100 |
Cezary Kaliszyk |
Regularization
|
file |
diff |
annotate
|
Fri, 30 Oct 2009 16:24:07 +0100 |
Cezary Kaliszyk |
Finally merged the code of the versions of regularize and tested examples.
|
file |
diff |
annotate
|
Fri, 30 Oct 2009 14:25:37 +0100 |
Cezary Kaliszyk |
Finding applications and duplicates filtered out in abstractions
|
file |
diff |
annotate
|
Fri, 30 Oct 2009 11:25:29 +0100 |
Cezary Kaliszyk |
Cleaning of the interface to lift.
|
file |
diff |
annotate
|
Thu, 29 Oct 2009 13:29:03 +0100 |
Cezary Kaliszyk |
Cleaning of 'map id' and 'prod_fun id id' in lower_defs.
|
file |
diff |
annotate
|
Thu, 29 Oct 2009 12:09:31 +0100 |
Cezary Kaliszyk |
Using subst for identity definition.
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 16:11:28 +0100 |
Cezary Kaliszyk |
Fix also in the general procedure.
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 16:05:59 +0100 |
Cezary Kaliszyk |
Fixes
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 15:25:36 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 15:25:11 +0100 |
Christian Urban |
added infrastructure for defining lifted constants
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 14:59:24 +0100 |
Cezary Kaliszyk |
First experiments with Lambda
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 10:17:07 +0100 |
Cezary Kaliszyk |
Proof of append_rsp
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 01:49:31 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 01:48:45 +0100 |
Christian Urban |
added a function for matching types
|
file |
diff |
annotate
|
Tue, 27 Oct 2009 18:02:35 +0100 |
Cezary Kaliszyk |
Simplfied interface to repabs_injection.
|
file |
diff |
annotate
|
Tue, 27 Oct 2009 17:08:47 +0100 |
Cezary Kaliszyk |
map_append lifted automatically.
|
file |
diff |
annotate
|
Tue, 27 Oct 2009 15:00:15 +0100 |
Cezary Kaliszyk |
Merged
|
file |
diff |
annotate
|
Tue, 27 Oct 2009 14:59:00 +0100 |
Cezary Kaliszyk |
Fixed APPLY_RSP vs Cong in the InjRepAbs tactic.
|
file |
diff |
annotate
|
Tue, 27 Oct 2009 14:46:38 +0100 |
Christian Urban |
tuned
|
file |
diff |
annotate
|
Tue, 27 Oct 2009 14:14:30 +0100 |
Christian Urban |
added equiv-thm to the quot_info
|
file |
diff |
annotate
|
Tue, 27 Oct 2009 11:27:53 +0100 |
Christian Urban |
made quotients compatiple with Nominal; updated keyword file
|
file |
diff |
annotate
|
Tue, 27 Oct 2009 09:01:12 +0100 |
Cezary Kaliszyk |
Completely cleaned Int.
|
file |
diff |
annotate
|
Tue, 27 Oct 2009 07:46:52 +0100 |
Cezary Kaliszyk |
Further reordering in Int code.
|
file |
diff |
annotate
|
Mon, 26 Oct 2009 14:18:26 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Mon, 26 Oct 2009 13:33:28 +0100 |
Cezary Kaliszyk |
Symmetry of integer addition
|
file |
diff |
annotate
|
Mon, 26 Oct 2009 11:55:36 +0100 |
Cezary Kaliszyk |
Finished the code for adding lower defs, and more things moved to QuotMain
|
file |
diff |
annotate
|
Mon, 26 Oct 2009 10:02:50 +0100 |
Cezary Kaliszyk |
Cleaning and fixing.
|
file |
diff |
annotate
|
Sun, 25 Oct 2009 23:44:41 +0100 |
Christian Urban |
added code for declaring map-functions
|
file |
diff |
annotate
|
Sun, 25 Oct 2009 00:14:40 +0200 |
Christian Urban |
added data-storage about the quotients
|
file |
diff |
annotate
|
Sat, 24 Oct 2009 18:17:38 +0200 |
Christian Urban |
changed the definitions of liftet constants to use fun_maps
|
file |
diff |
annotate
|
Sat, 24 Oct 2009 16:09:05 +0200 |
Christian Urban |
moved the map_funs setup into QuotMain
|
file |
diff |
annotate
|
Sat, 24 Oct 2009 08:34:14 +0200 |
cek |
Undid wrong merge
|
file |
diff |
annotate
|
Sat, 24 Oct 2009 08:24:26 +0200 |
cek |
Cleaning the mess
|
file |
diff |
annotate
|
Sat, 24 Oct 2009 01:33:29 +0200 |
Christian Urban |
fixed problem with incorrect ABS/REP name
|
file |
diff |
annotate
|