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 14:16:41 +0100 |
Cezary Kaliszyk |
Move atomize_goal to QuotMain
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 14:05:02 +0100 |
Cezary Kaliszyk |
Removed second implementation of Regularize/Inject from FSet.
|
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
|
Mon, 23 Nov 2009 13:24:12 +0100 |
Christian Urban |
code review with Cezary
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 10:26:59 +0100 |
Cezary Kaliszyk |
The other branch does not seem to work...
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 10:04:35 +0100 |
Cezary Kaliszyk |
Fixes for recent changes.
|
file |
diff |
annotate
|
Fri, 13 Nov 2009 19:32:12 +0100 |
Cezary Kaliszyk |
Still don't know how to do the proof automatically.
|
file |
diff |
annotate
|
Thu, 12 Nov 2009 13:56:07 +0100 |
Cezary Kaliszyk |
merged
|
file |
diff |
annotate
|
Wed, 11 Nov 2009 22:30:43 +0100 |
Cezary Kaliszyk |
Lifting towards goal and manually finished the proof.
|
file |
diff |
annotate
|
Wed, 11 Nov 2009 10:22:47 +0100 |
Cezary Kaliszyk |
Removed 'Toplevel.program' for polyml 5.3
|
file |
diff |
annotate
|
Tue, 10 Nov 2009 17:43:05 +0100 |
Cezary Kaliszyk |
Atomizing a "goal" theorems.
|
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 17:42:20 +0100 |
Cezary Kaliszyk |
Minor changes
|
file |
diff |
annotate
|
Fri, 06 Nov 2009 11:01:22 +0100 |
Cezary Kaliszyk |
fold_rsp
|
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:47:41 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Thu, 05 Nov 2009 13:47:04 +0100 |
Christian Urban |
removed typing information from get_fun in quotient_def; *potentially* dangerous
|
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 09:38:34 +0100 |
Cezary Kaliszyk |
Infrastructure for polymorphic types
|
file |
diff |
annotate
|
Wed, 04 Nov 2009 11:08:05 +0100 |
Cezary Kaliszyk |
Experiments in Int
|
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 15:38:03 +0100 |
Cezary Kaliszyk |
Fixes after optimization and preparing for a general FORALL_PRS
|
file |
diff |
annotate
|
Mon, 02 Nov 2009 11:51:50 +0100 |
Cezary Kaliszyk |
Map does not fully work yet.
|
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 15:30:33 +0100 |
Christian Urban |
not sure what changed here
|
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 08:06:49 +0100 |
Cezary Kaliszyk |
Fixed wrong CARD definition and removed the "Does not work anymore" comment.
|
file |
diff |
annotate
|
Thu, 29 Oct 2009 07:29:12 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 20:01:20 +0100 |
Christian Urban |
updated some definitions; had to give sometimes different names; somewhere I introduced a bug, since not everything is working anymore (needs fixing!)
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 18:08:38 +0100 |
Cezary Kaliszyk |
disambiguate ===> syntax
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 17:17:21 +0100 |
Cezary Kaliszyk |
cleaned FSet
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 16:48:57 +0100 |
Cezary Kaliszyk |
Some cleaning
|
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 12:22:06 +0100 |
Cezary Kaliszyk |
Fixed mistake in const generation, will postpone this.
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 10:29:00 +0100 |
Cezary Kaliszyk |
More finshed proofs and cleaning
|
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:05:45 +0100 |
Cezary Kaliszyk |
Manual conversion of equality to equivalence allows lifting append_assoc.
|
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 16:15:56 +0100 |
Cezary Kaliszyk |
Manually lifted Map_Append.
|
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 12:20:57 +0100 |
Cezary Kaliszyk |
Simplifying FSet with new functions.
|
file |
diff |
annotate
|
Mon, 26 Oct 2009 15:31:53 +0100 |
Cezary Kaliszyk |
Simplifying Int and Working on map
|
file |
diff |
annotate
|