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
|
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:35:50 +0100 |
Christian Urban |
deleted obsolete qenv code
|
file |
diff |
annotate
|
Fri, 27 Nov 2009 02:23:49 +0100 |
Christian Urban |
renamed REGULARIZE to be regularize
|
file |
diff |
annotate
|
Wed, 25 Nov 2009 21:48:32 +0100 |
Cezary Kaliszyk |
applic_prs
|
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:39:53 +0100 |
Cezary Kaliszyk |
cleaning in MyInt
|
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 15:15:10 +0100 |
Christian Urban |
added a prepare_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 13:46:36 +0100 |
Christian Urban |
explicit phases for the cleaning
|
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 20:10:39 +0100 |
Cezary Kaliszyk |
Finished temporary goal-directed lift_theorem wrapper.
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 15:47:14 +0100 |
Cezary Kaliszyk |
Fixes for atomize
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 15:08:09 +0100 |
Cezary Kaliszyk |
lift_thm with a goal.
|
file |
diff |
annotate
|
Mon, 23 Nov 2009 14:40:53 +0100 |
Cezary Kaliszyk |
Fixes for new code
|
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: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
|
Sun, 22 Nov 2009 00:01:06 +0100 |
Christian Urban |
a little tuning of comments
|
file |
diff |
annotate
|
Sat, 21 Nov 2009 23:23:01 +0100 |
Christian Urban |
slight tuning
|
file |
diff |
annotate
|
Sat, 21 Nov 2009 14:45:25 +0100 |
Christian Urban |
some debugging code, but cannot find the place where the cprems_of exception is raised
|
file |
diff |
annotate
|
Sat, 21 Nov 2009 14:18:31 +0100 |
Christian Urban |
tried to prove the repabs_inj lemma, but failed for the moment
|
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 10:58:08 +0100 |
Christian Urban |
tunded
|
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
|
Wed, 18 Nov 2009 23:52:48 +0100 |
Christian Urban |
fixed the storage of qconst definitions
|
file |
diff |
annotate
|
Thu, 12 Nov 2009 12:07:33 +0100 |
Christian Urban |
looking up data in quot_info works now (needs qualified string)
|
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 11:59:22 +0100 |
Christian Urban |
updated to new Theory_Data and to new Isabelle
|
file |
diff |
annotate
|
Wed, 11 Nov 2009 10:22:47 +0100 |
Cezary Kaliszyk |
Removed 'Toplevel.program' for polyml 5.3
|
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 09:55:21 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Wed, 04 Nov 2009 13:33:13 +0100 |
Cezary Kaliszyk |
Experiments with lifting partially applied constants.
|
file |
diff |
annotate
|
Wed, 04 Nov 2009 11:08:05 +0100 |
Cezary Kaliszyk |
Experiments in Int
|
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
|
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
|
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:39:25 +0100 |
Christian Urban |
merged
|
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 15:38:03 +0100 |
Cezary Kaliszyk |
Fixes after optimization and preparing for a general FORALL_PRS
|
file |
diff |
annotate
|
Fri, 30 Oct 2009 11:25:29 +0100 |
Cezary Kaliszyk |
Cleaning of the interface to lift.
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 18:08:38 +0100 |
Cezary Kaliszyk |
disambiguate ===> syntax
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 16:16:38 +0100 |
Cezary Kaliszyk |
Cleaning the unnecessary theorems in 'IntEx'.
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 16:06:19 +0100 |
Cezary Kaliszyk |
merge
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 16:05:59 +0100 |
Cezary Kaliszyk |
Fixes
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 15:48:38 +0100 |
Christian Urban |
updated all definitions
|
file |
diff |
annotate
|
Wed, 28 Oct 2009 15:25:11 +0100 |
Christian Urban |
added infrastructure for defining lifted constants
|
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 14:59:00 +0100 |
Cezary Kaliszyk |
Fixed APPLY_RSP vs Cong in the InjRepAbs tactic.
|
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 11:03:38 +0100 |
Christian Urban |
merged
|
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 19:35:30 +0100 |
Cezary Kaliszyk |
Simplifying Int.
|
file |
diff |
annotate
|