| 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 |