Fri, 04 Dec 2009 15:04:05 +0100 |
Cezary Kaliszyk |
Naming 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 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 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:18:46 +0100 |
Cezary Kaliszyk |
Changing = to \<equiv> in case if we want to use simp.
|
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
|
Sat, 28 Nov 2009 05:29:30 +0100 |
Cezary Kaliszyk |
Finished and tested the new regularize
|
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
|
Fri, 27 Nov 2009 08:15:23 +0100 |
Cezary Kaliszyk |
Removing arguments of tactics: absrep, rel_refl, reps_same are computed.
|
file |
diff |
annotate
|
Thu, 26 Nov 2009 13:52:46 +0100 |
Christian Urban |
fixed QuotList
|
file |
diff |
annotate
|
Thu, 26 Nov 2009 13:46:00 +0100 |
Christian Urban |
changed left-res
|
file |
diff |
annotate
|
Thu, 26 Nov 2009 12:21:47 +0100 |
Cezary Kaliszyk |
Manually regularized akind_aty_atrm.induct
|
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
|
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
|
Wed, 28 Oct 2009 18:08:38 +0100 |
Cezary Kaliszyk |
disambiguate ===> syntax
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 14:59:24 +0100 |
Cezary Kaliszyk |
First experiments with Lambda
|
file |
diff |
annotate
|
Mon, 26 Oct 2009 10:20:20 +0100 |
Cezary Kaliszyk |
Finished COND_PRS proof.
|
file |
diff |
annotate
|
Mon, 26 Oct 2009 10:02:50 +0100 |
Cezary Kaliszyk |
Cleaning and fixing.
|
file |
diff |
annotate
|
Sun, 25 Oct 2009 01:15:03 +0200 |
Christian Urban |
proved the two lemmas in QuotScript (reformulated them without leading forall)
|
file |
diff |
annotate
|
Sat, 24 Oct 2009 14:00:18 +0200 |
Cezary Kaliszyk |
Finally completely lift the previously lifted theorems + clean some old stuff
|
file |
diff |
annotate
|
Sat, 24 Oct 2009 13:00:54 +0200 |
Cezary Kaliszyk |
More infrastructure for automatic lifting of theorems lifted before
|
file |
diff |
annotate
|
Sat, 24 Oct 2009 10:16:53 +0200 |
Cezary Kaliszyk |
More infrastructure for automatic lifting of theorems lifted before
|
file |
diff |
annotate
|
Sat, 24 Oct 2009 08:09:09 +0200 |
cek |
Better tactic and simplified the proof further
|
file |
diff |
annotate
|
Fri, 23 Oct 2009 16:01:13 +0200 |
Cezary Kaliszyk |
eqsubst_tac
|
file |
diff |
annotate
|
Thu, 22 Oct 2009 15:44:16 +0200 |
Cezary Kaliszyk |
Removed an assumption
|
file |
diff |
annotate
|
Thu, 22 Oct 2009 15:02:01 +0200 |
Cezary Kaliszyk |
The proof now including manually unfolded higher-order RES_FORALL_RSP.
|
file |
diff |
annotate
|
Thu, 22 Oct 2009 13:45:48 +0200 |
Cezary Kaliszyk |
The problems with 'abs' term.
|
file |
diff |
annotate
|
Sat, 17 Oct 2009 16:06:54 +0200 |
Cezary Kaliszyk |
Partial simplification of the proof
|
file |
diff |
annotate
|
Fri, 16 Oct 2009 17:05:52 +0200 |
Cezary Kaliszyk |
Symmetric version of REP_ABS_RSP
|
file |
diff |
annotate
|
Fri, 16 Oct 2009 16:51:01 +0200 |
Cezary Kaliszyk |
Progressing with the proof
|
file |
diff |
annotate
|
Thu, 15 Oct 2009 10:25:23 +0200 |
Cezary Kaliszyk |
A number of lemmas for REGULARIZE_TAC and regularizing card1.
|
file |
diff |
annotate
|
Wed, 14 Oct 2009 18:13:16 +0200 |
Cezary Kaliszyk |
Proving the proper RepAbs version
|
file |
diff |
annotate
|
Wed, 14 Oct 2009 16:23:32 +0200 |
Cezary Kaliszyk |
Manually regularized list_induct2
|
file |
diff |
annotate
|
Tue, 11 Aug 2009 12:29:15 +0200 |
Christian Urban |
initial commit
|
file |
diff |
annotate
|