Sun, 29 Aug 2010 01:45:07 +0800 |
Christian Urban |
added fs-instance proofs
|
file |
diff |
annotate
|
Sun, 29 Aug 2010 01:17:36 +0800 |
Christian Urban |
added proofs for fsupp properties
|
file |
diff |
annotate
|
Sun, 29 Aug 2010 00:09:45 +0800 |
Christian Urban |
proved supports lemmas
|
file |
diff |
annotate
|
Fri, 27 Aug 2010 03:37:17 +0800 |
Christian Urban |
"isabelle make test" makes all major examples....they work up to supp theorems (excluding)
|
file |
diff |
annotate
|
Fri, 27 Aug 2010 02:03:52 +0800 |
Christian Urban |
corrected bug with fv-function generation (that was the problem with recursive binders)
|
file |
diff |
annotate
|
Thu, 26 Aug 2010 02:08:00 +0800 |
Christian Urban |
cleaned up (almost completely) the examples
|
file |
diff |
annotate
|
Wed, 25 Aug 2010 23:16:42 +0800 |
Christian Urban |
cleaning of unused files and code
|
file |
diff |
annotate
|
Wed, 25 Aug 2010 22:55:42 +0800 |
Christian Urban |
automatic lifting
|
file |
diff |
annotate
|
Wed, 25 Aug 2010 09:02:06 +0800 |
Christian Urban |
can now deal with type variables in nominal datatype definitions
|
file |
diff |
annotate
|
Sun, 22 Aug 2010 14:02:49 +0800 |
Christian Urban |
updated to new Isabelle
|
file |
diff |
annotate
|
Sun, 22 Aug 2010 11:00:53 +0800 |
Christian Urban |
updated to new Isabelle
|
file |
diff |
annotate
|
Sat, 21 Aug 2010 20:07:36 +0800 |
Christian Urban |
moved lifting code from Lift.thy to nominal_dt_quot.ML
|
file |
diff |
annotate
|
Sat, 21 Aug 2010 17:55:42 +0800 |
Christian Urban |
nominal_datatypes with type variables do not work
|
file |
diff |
annotate
|
Sat, 21 Aug 2010 16:20:10 +0800 |
Christian Urban |
changed parser so that the binding mode is indicated as "bind (list)", "bind (set)" or "bind (res)"; if only "bind" is given, then bind (list) is assumed as default
|
file |
diff |
annotate
|
Wed, 18 Aug 2010 00:23:42 +0800 |
Christian Urban |
put everything in a "timeit"
|
file |
diff |
annotate
|
Wed, 18 Aug 2010 00:19:15 +0800 |
Christian Urban |
improved runtime slightly, by constructing an explicit size measure for the function definitions
|
file |
diff |
annotate
|
Tue, 17 Aug 2010 18:17:53 +0800 |
Christian Urban |
more tuning of the code
|
file |
diff |
annotate
|
Tue, 17 Aug 2010 17:52:25 +0800 |
Christian Urban |
improved code
|
file |
diff |
annotate
|
Tue, 17 Aug 2010 07:11:45 +0800 |
Christian Urban |
can also lift the various eqvt lemmas for bn, fv, fv_bn and size
|
file |
diff |
annotate
|
Tue, 17 Aug 2010 06:50:49 +0800 |
Christian Urban |
also able to lift the bn_defs
|
file |
diff |
annotate
|
Tue, 17 Aug 2010 06:39:27 +0800 |
Christian Urban |
added rsp-lemmas for alpha_bns
|
file |
diff |
annotate
|
Mon, 16 Aug 2010 17:39:16 +0800 |
Christian Urban |
modified the code for class instantiations (with help from Florian)
|
file |
diff |
annotate
|
Sun, 15 Aug 2010 14:00:28 +0800 |
Christian Urban |
defined qperms and qsizes
|
file |
diff |
annotate
|
Sun, 15 Aug 2010 11:03:13 +0800 |
Christian Urban |
simplified code
|
file |
diff |
annotate
|
Sat, 14 Aug 2010 23:33:23 +0800 |
Christian Urban |
improved code
|
file |
diff |
annotate
|
Sat, 14 Aug 2010 16:54:41 +0800 |
Christian Urban |
more experiments with lifting
|
file |
diff |
annotate
|
Thu, 12 Aug 2010 21:29:35 +0800 |
Christian Urban |
updated to Isabelle 12th Aug
|
file |
diff |
annotate
|
Wed, 11 Aug 2010 19:53:57 +0800 |
Christian Urban |
rsp for constructors
|
file |
diff |
annotate
|
Sun, 08 Aug 2010 10:12:38 +0800 |
Christian Urban |
proved rsp-helper lemmas of size functions
|
file |
diff |
annotate
|
Sat, 31 Jul 2010 01:24:39 +0100 |
Christian Urban |
introduced a general alpha_prove method
|
file |
diff |
annotate
|
Fri, 30 Jul 2010 00:40:32 +0100 |
Christian Urban |
equivariance for size
|
file |
diff |
annotate
|
Thu, 29 Jul 2010 10:16:33 +0100 |
Christian Urban |
helper lemmas for rsp-lemmas
|
file |
diff |
annotate
|
Tue, 27 Jul 2010 09:09:02 +0200 |
Christian Urban |
fixed order of fold_union to make alpha and fv agree
|
file |
diff |
annotate
|
Thu, 22 Jul 2010 08:30:50 +0200 |
Christian Urban |
updated to new Isabelle; made FSet more "quiet"
|
file |
diff |
annotate
|
Fri, 16 Jul 2010 02:38:19 +0100 |
Christian Urban |
more on the paper
|
file |
diff |
annotate
|
Wed, 07 Jul 2010 09:34:00 +0100 |
Christian Urban |
more on the paper
|
file |
diff |
annotate
|
Mon, 28 Jun 2010 16:22:28 +0100 |
Christian Urban |
more quotient-definitions
|
file |
diff |
annotate
|
Mon, 28 Jun 2010 15:23:56 +0100 |
Christian Urban |
slight cleaning
|
file |
diff |
annotate
|
Sun, 27 Jun 2010 21:41:21 +0100 |
Christian Urban |
fixed according to changes in quotient
|
file |
diff |
annotate
|
Thu, 24 Jun 2010 21:35:11 +0100 |
Christian Urban |
added definition of the quotient types
|
file |
diff |
annotate
|
Wed, 23 Jun 2010 06:54:48 +0100 |
Christian Urban |
deleted compose-lemmas in Abs (not needed anymore)
|
file |
diff |
annotate
|
Wed, 23 Jun 2010 06:45:03 +0100 |
Christian Urban |
deleted equivp_hack
|
file |
diff |
annotate
|
Tue, 22 Jun 2010 18:07:53 +0100 |
Christian Urban |
proved eqvip theorems for alphas
|
file |
diff |
annotate
|
Tue, 22 Jun 2010 13:31:42 +0100 |
Christian Urban |
cleaned up the FSet (noise was introduced by error)
|
file |
diff |
annotate
|
Tue, 22 Jun 2010 13:05:00 +0100 |
Christian Urban |
prove that alpha implies alpha_bn (needed for rsp proofs)
|
file |
diff |
annotate
|
Fri, 11 Jun 2010 03:02:42 +0200 |
Christian Urban |
also symmetry
|
file |
diff |
annotate
|
Thu, 10 Jun 2010 14:53:28 +0200 |
Christian Urban |
premerge
|
file |
diff |
annotate
|
Wed, 09 Jun 2010 15:14:16 +0200 |
Christian Urban |
transitivity proofs done
|
file |
diff |
annotate
|
Mon, 07 Jun 2010 11:43:01 +0200 |
Christian Urban |
work on transitivity proof
|
file |
diff |
annotate
|
Thu, 03 Jun 2010 11:48:44 +0200 |
Christian Urban |
fixed problem with eqvt proofs
|
file |
diff |
annotate
|
Wed, 02 Jun 2010 11:37:51 +0200 |
Christian Urban |
fixed problem with bn_info
|
file |
diff |
annotate
|
Tue, 01 Jun 2010 15:21:01 +0200 |
Christian Urban |
equivariance done
|
file |
diff |
annotate
|
Tue, 01 Jun 2010 15:01:05 +0200 |
Christian Urban |
smaller code for raw-eqvt proofs
|
file |
diff |
annotate
|
Mon, 31 May 2010 19:57:29 +0200 |
Christian Urban |
all raw definitions are defined using function
|
file |
diff |
annotate
|
Thu, 27 May 2010 18:37:52 +0200 |
Christian Urban |
intermediate state
|
file |
diff |
annotate
|
Wed, 26 May 2010 15:37:56 +0200 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Wed, 26 May 2010 15:34:54 +0200 |
Christian Urban |
added FSet to the correct paper
|
file |
diff |
annotate
|
Tue, 25 May 2010 00:24:41 +0100 |
Christian Urban |
added slides
|
file |
diff |
annotate
|
Mon, 24 May 2010 21:11:33 +0100 |
Christian Urban |
tuned
|
file |
diff |
annotate
|
Mon, 24 May 2010 20:50:15 +0100 |
Christian Urban |
tuned
|
file |
diff |
annotate
|
Mon, 24 May 2010 20:02:37 +0100 |
Christian Urban |
alpha works now
|
file |
diff |
annotate
|
Sun, 23 May 2010 02:15:24 +0100 |
Christian Urban |
started to work on alpha
|
file |
diff |
annotate
|
Sat, 22 May 2010 13:51:47 +0100 |
Christian Urban |
properly exported bn_descr
|
file |
diff |
annotate
|
Fri, 21 May 2010 11:40:18 +0100 |
Christian Urban |
hving a working fv-definition without the export
|
file |
diff |
annotate
|
Fri, 21 May 2010 05:58:23 +0100 |
Christian Urban |
tuned
|
file |
diff |
annotate
|
Thu, 20 May 2010 21:23:53 +0100 |
Christian Urban |
new fv/fv_bn function (supp breaks now); exported raw perms and raw funs into separate ML-files
|
file |
diff |
annotate
|
Fri, 21 May 2010 10:42:53 +0200 |
Cezary Kaliszyk |
Renamings
|
file |
diff |
annotate
|
Mon, 17 May 2010 16:25:45 +0100 |
Christian Urban |
minor tuning
|
file |
diff |
annotate
|
Mon, 17 May 2010 12:46:51 +0100 |
Christian Urban |
slight tuning
|
file |
diff |
annotate
|
Mon, 17 May 2010 12:00:54 +0100 |
Christian Urban |
somewhat simplified the main parsing function; failed to move a Note-statement to define_raw_perms
|
file |
diff |
annotate
|
Sun, 16 May 2010 12:41:27 +0100 |
Christian Urban |
moved the exporting part into the parser (this is still a hack); re-added CoreHaskell again to the examples - there seems to be a problem with the variable name pat
|
file |
diff |
annotate
|
Thu, 13 May 2010 15:58:02 +0100 |
Christian Urban |
made out of STEPS a configuration value so that it can be set individually in each file
|
file |
diff |
annotate
|
Thu, 13 May 2010 10:34:59 +0100 |
Christian Urban |
added term4 back to the examples
|
file |
diff |
annotate
|
Wed, 12 May 2010 16:33:50 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Wed, 12 May 2010 16:33:25 +0100 |
Christian Urban |
moved the data-transformation into the parser
|
file |
diff |
annotate
|
Wed, 12 May 2010 16:39:10 +0200 |
Cezary Kaliszyk |
Move alpha_eqvt to unused.
|
file |
diff |
annotate
|
Wed, 12 May 2010 16:32:44 +0200 |
Cezary Kaliszyk |
Use equivariance instead of alpha_eqvt
|
file |
diff |
annotate
|
Wed, 12 May 2010 14:47:52 +0100 |
Christian Urban |
ingnored parameters in equivariance; added a proper interface to be called from ML
|
file |
diff |
annotate
|
Wed, 12 May 2010 13:43:48 +0100 |
Christian Urban |
properly exported defined bn-functions
|
file |
diff |
annotate
|
Tue, 11 May 2010 18:20:25 +0200 |
Cezary Kaliszyk |
Include raw permutation definitions in eqvt
|
file |
diff |
annotate
|
Mon, 10 May 2010 15:11:05 +0200 |
Cezary Kaliszyk |
Parser changes for compound relations
|
file |
diff |
annotate
|
Thu, 06 May 2010 14:14:30 +0200 |
Cezary Kaliszyk |
mem => member
|
file |
diff |
annotate
|
Tue, 04 May 2010 14:38:07 +0100 |
Christian Urban |
increased step counter so that all steps go through
|
file |
diff |
annotate
|
Tue, 04 May 2010 14:33:50 +0100 |
Christian Urban |
fixed my error with define_raw_fv
|
file |
diff |
annotate
|
Tue, 04 May 2010 14:25:22 +0100 |
Christian Urban |
tuned and added some comments to the code; added also an exception for early exit of the nominal2_cmd function
|
file |
diff |
annotate
|
Tue, 04 May 2010 06:24:54 +0100 |
Christian Urban |
roll back of the last commit (there was a difference)
|
file |
diff |
annotate
|
Tue, 04 May 2010 06:02:45 +0100 |
Christian Urban |
to my best knowledge the number of datatypes is equal to the length of the dt_descr; so we can save one argument in define_raw_perm
|
file |
diff |
annotate
|
Mon, 03 May 2010 15:13:15 +0200 |
Cezary Kaliszyk |
Comment
|
file |
diff |
annotate
|
Mon, 03 May 2010 14:30:37 +0200 |
Cezary Kaliszyk |
Register only non-looping rules in eq_iff
|
file |
diff |
annotate
|
Mon, 03 May 2010 13:42:44 +0200 |
Cezary Kaliszyk |
NewParser
|
file |
diff |
annotate
|
Mon, 03 May 2010 12:24:27 +0200 |
Cezary Kaliszyk |
Introduce eq_iff_simp to match the one from Parser.
|
file |
diff |
annotate
|
Mon, 03 May 2010 11:43:08 +0200 |
Cezary Kaliszyk |
Cheat support equations in new parser
|
file |
diff |
annotate
|
Mon, 03 May 2010 10:15:23 +0200 |
Cezary Kaliszyk |
Add explicit cheats in NewParser and comment out the examples for outside use.
|
file |
diff |
annotate
|
Mon, 03 May 2010 09:57:05 +0200 |
Cezary Kaliszyk |
Fix Datatype_Aux calls in NewParser.
|
file |
diff |
annotate
|
Sun, 02 May 2010 16:02:27 +0100 |
Christian Urban |
tried to add some comments in the huge(!) nominal2_cmd function
|
file |
diff |
annotate
|
Sun, 02 May 2010 14:06:26 +0100 |
Christian Urban |
attempted to remove dependency on (old) Fv and (old) Parser; lifting still uses Fv.thy; the examples do not work at the moment (with equivp proofs failing)
|
file |
diff |
annotate
|
Sat, 01 May 2010 09:15:46 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Sat, 01 May 2010 09:14:25 +0100 |
Christian Urban |
tuned
|
file |
diff |
annotate
|
Fri, 30 Apr 2010 15:45:39 +0200 |
Cezary Kaliszyk |
NewParser with Parser functionality, but some cheats included since the order of datayupes is wrong.
|
file |
diff |
annotate
|
Fri, 30 Apr 2010 14:48:13 +0200 |
Cezary Kaliszyk |
Merged nominal_datatype into NewParser until eqvts
|
file |
diff |
annotate
|
Fri, 30 Apr 2010 13:57:59 +0200 |
Cezary Kaliszyk |
more parser/new parser synchronization.
|
file |
diff |
annotate
|
Fri, 30 Apr 2010 10:31:32 +0200 |
Cezary Kaliszyk |
Change signature of fv and alpha generation.
|
file |
diff |
annotate
|
Thu, 29 Apr 2010 17:52:19 +0200 |
Cezary Kaliszyk |
New Alpha.
|
file |
diff |
annotate
|
Thu, 29 Apr 2010 16:18:38 +0200 |
Cezary Kaliszyk |
Fixing the definitions in the Parser.
|
file |
diff |
annotate
|
Thu, 29 Apr 2010 10:59:08 +0200 |
Cezary Kaliszyk |
Include support of unknown datatypes in new fv
|
file |
diff |
annotate
|
Wed, 28 Apr 2010 08:22:20 +0200 |
Christian Urban |
simpliied and moved the remaining lemmas about the atom-function to Nominal2_Base
|
file |
diff |
annotate
|
Wed, 28 Apr 2010 07:27:28 +0200 |
Christian Urban |
use sort at_base instead of at
|
file |
diff |
annotate
|
Tue, 27 Apr 2010 23:11:40 +0200 |
Christian Urban |
added some further problemetic tests
|
file |
diff |
annotate
|
Tue, 27 Apr 2010 22:45:50 +0200 |
Christian Urban |
some tuning
|
file |
diff |
annotate
|
Tue, 27 Apr 2010 19:01:22 +0200 |
Cezary Kaliszyk |
Rewrote FV code and included the function package.
|
file |
diff |
annotate
|
Sun, 25 Apr 2010 08:06:43 +0200 |
Christian Urban |
added definition of raw-permutations to the new-parser
|
file |
diff |
annotate
|
Sun, 25 Apr 2010 07:54:28 +0200 |
Christian Urban |
tuned
|
file |
diff |
annotate
|
Sun, 25 Apr 2010 01:31:22 +0200 |
Christian Urban |
slight tuning
|
file |
diff |
annotate
|
Sat, 24 Apr 2010 10:00:33 +0200 |
Christian Urban |
added a comment about a function where I am not sure who wrote it.
|
file |
diff |
annotate
|
Sat, 24 Apr 2010 09:49:23 +0200 |
Christian Urban |
merged
|
file |
diff |
annotate
|