Tue, 09 Mar 2010 17:25:35 +0100 Cezary Kaliszyk All examples should work.
Tue, 09 Mar 2010 17:02:29 +0100 Cezary Kaliszyk Fix to get old alpha.
Tue, 09 Mar 2010 16:57:51 +0100 Cezary Kaliszyk Separate primrecs in Fv.
Tue, 09 Mar 2010 16:24:39 +0100 Cezary Kaliszyk A version of Fv that takes into account recursive and non-recursive bindings.
Tue, 09 Mar 2010 11:36:40 +0100 Cezary Kaliszyk Trying to prove that old alpha is the same as new recursive one. Lets still to do.
Tue, 09 Mar 2010 11:06:57 +0100 Cezary Kaliszyk fv_bi and alpha_bi
Tue, 09 Mar 2010 09:55:19 +0100 Christian Urban merged
Tue, 09 Mar 2010 09:54:58 +0100 Christian Urban added first test about new compat
Tue, 09 Mar 2010 09:38:49 +0100 Cezary Kaliszyk fv_compat
Tue, 09 Mar 2010 08:46:55 +0100 Christian Urban added another compat example
Mon, 08 Mar 2010 20:18:27 +0100 Christian Urban added a test-file for compatibility
Mon, 08 Mar 2010 16:11:42 +0100 Christian Urban added compat definitions to some examples
Mon, 08 Mar 2010 15:28:25 +0100 Cezary Kaliszyk Proper recognition of atoms and atom sets.
Mon, 08 Mar 2010 15:06:14 +0100 Christian Urban deleted comments about "weird"
Mon, 08 Mar 2010 15:01:26 +0100 Christian Urban merged
Mon, 08 Mar 2010 15:01:01 +0100 Christian Urban updated to new Isabelle
Mon, 08 Mar 2010 14:31:04 +0100 Cezary Kaliszyk Term5 written as nominal_datatype is the recursive let.
Mon, 08 Mar 2010 11:25:57 +0100 Cezary Kaliszyk With restricted_nominal=1, exp7 and exp8 work. Not sure about proving bn_rsp there.
Mon, 08 Mar 2010 11:12:15 +0100 Cezary Kaliszyk More fine-grained nominal restriction for debugging.
Mon, 08 Mar 2010 11:10:43 +0100 Cezary Kaliszyk Fix permutation addition.
Mon, 08 Mar 2010 10:33:55 +0100 Cezary Kaliszyk Update the comments
Mon, 08 Mar 2010 10:08:31 +0100 Cezary Kaliszyk Gather bindings with same binder, and generate only one permutation for them.
Mon, 08 Mar 2010 02:40:16 +0100 Cezary Kaliszyk Undo effects of simp.
Sun, 07 Mar 2010 21:30:57 +0100 Christian Urban merged
Sun, 07 Mar 2010 21:30:12 +0100 Christian Urban updated to renamings in Isabelle
Thu, 04 Mar 2010 15:56:58 +0100 Christian Urban merged
Thu, 04 Mar 2010 15:31:34 +0100 Christian Urban merged
Thu, 04 Mar 2010 15:31:21 +0100 Christian Urban more proofs in Abs and work on Core Haskell
Wed, 03 Mar 2010 19:10:40 +0100 Christian Urban added a lemma that permutations can be represented as sums of swapping
Fri, 05 Mar 2010 18:14:04 +0100 Cezary Kaliszyk Still unable to show supp=fv for let with one existential.
Fri, 05 Mar 2010 17:09:48 +0100 Cezary Kaliszyk Ported LF to the parser interface.
Fri, 05 Mar 2010 14:56:19 +0100 Cezary Kaliszyk merge
Fri, 05 Mar 2010 14:55:21 +0100 Cezary Kaliszyk Lift fv and bn eqvts; no need to lift alpha_eqvt.
Fri, 05 Mar 2010 13:04:47 +0100 Cezary Kaliszyk Not much progress about the single existential let case.
Fri, 05 Mar 2010 10:23:40 +0100 Cezary Kaliszyk Fixed LF for one quantifier over 2 premises.
Fri, 05 Mar 2010 09:41:22 +0100 Cezary Kaliszyk Trying to fix the proofs for the single existential... So far failed.
Thu, 04 Mar 2010 18:57:23 +0100 Cezary Kaliszyk Lift distinct.
Thu, 04 Mar 2010 15:55:53 +0100 Cezary Kaliszyk Added lifting of pseudo-injectivity, commented out the code again and enabled the weird examples.
Thu, 04 Mar 2010 15:15:44 +0100 Cezary Kaliszyk Lift BV,FV,Permutations and injection :).
Thu, 04 Mar 2010 12:00:11 +0100 Cezary Kaliszyk Comment out Weird and Phd until we have an idea how to handle multiple permutations. Transp that works for multiple existentials.
Thu, 04 Mar 2010 11:16:36 +0100 Cezary Kaliszyk A version that just leaves the supp/\supp goal. Obviously not true.
Thu, 04 Mar 2010 10:59:52 +0100 Cezary Kaliszyk Prove symp and transp of weird without the supp /\ supp = {} assumption.
Wed, 03 Mar 2010 17:51:47 +0100 Cezary Kaliszyk merge
Wed, 03 Mar 2010 17:49:34 +0100 Cezary Kaliszyk Experiments with proving weird transp
Wed, 03 Mar 2010 17:47:29 +0100 Cezary Kaliszyk Code for solving symp goals with multiple existentials.
Wed, 03 Mar 2010 15:28:25 +0100 Cezary Kaliszyk reflp for multiple quantifiers.
Wed, 03 Mar 2010 14:46:14 +0100 Christian Urban fixed mess in Test.thy
Wed, 03 Mar 2010 14:22:58 +0100 Cezary Kaliszyk Fix eqvt for multiple quantifiers.
Wed, 03 Mar 2010 12:48:05 +0100 Christian Urban only tuned
Wed, 03 Mar 2010 12:47:06 +0100 Christian Urban merged
Wed, 03 Mar 2010 12:45:55 +0100 Christian Urban start of paper - does not compile yet
Wed, 03 Mar 2010 11:50:25 +0100 Christian Urban added ACM style file for ICFP
Wed, 03 Mar 2010 11:42:15 +0100 Cezary Kaliszyk weird eqvt
Wed, 03 Mar 2010 10:39:43 +0100 Cezary Kaliszyk Add the supp intersection conditions.
Tue, 02 Mar 2010 21:43:27 +0100 Cezary Kaliszyk Comment out the part that does not work with 2 quantifiers.
Tue, 02 Mar 2010 21:10:04 +0100 Cezary Kaliszyk Fixes for the fv problem and alpha problem.
Tue, 02 Mar 2010 20:14:21 +0100 Christian Urban merged
Tue, 02 Mar 2010 20:11:56 +0100 Christian Urban preliinary test about alpha-weirdo
Tue, 02 Mar 2010 18:57:26 +0100 Christian Urban Another problem with permutations in alpha and possibly also in fv
Tue, 02 Mar 2010 18:48:20 +0100 Christian Urban potential problem with the phd-example, where two permutations are generated, but only one is used
Tue, 02 Mar 2010 19:48:44 +0100 Cezary Kaliszyk Some tests around Term4. Not sure how to fix the generated fv function.
Tue, 02 Mar 2010 17:48:56 +0100 Cezary Kaliszyk merge
Tue, 02 Mar 2010 17:48:41 +0100 Cezary Kaliszyk Porting from Lift to Parser; until defining the Quotient type.
Tue, 02 Mar 2010 17:11:58 +0100 Cezary Kaliszyk Add image_eqvt and atom_eqvt to eqvt bases.
Tue, 02 Mar 2010 17:11:19 +0100 Cezary Kaliszyk Include the raw eqvt lemmas.
Tue, 02 Mar 2010 16:04:48 +0100 Christian Urban merged
Tue, 02 Mar 2010 16:03:19 +0100 Christian Urban added some more examples from Peter Sewell's bestiary
Tue, 02 Mar 2010 15:13:00 +0100 Cezary Kaliszyk merge
Tue, 02 Mar 2010 15:12:50 +0100 Cezary Kaliszyk Minor
Tue, 02 Mar 2010 15:11:41 +0100 Cezary Kaliszyk Working bv_eqvt
Tue, 02 Mar 2010 15:10:47 +0100 Cezary Kaliszyk Moving wrappers out of Lift.
Tue, 02 Mar 2010 15:07:27 +0100 Christian Urban merged
Tue, 02 Mar 2010 15:05:50 +0100 Christian Urban added distinctness of perms
Tue, 02 Mar 2010 15:05:35 +0100 Christian Urban updated (added lemma about commuting permutations)
Tue, 02 Mar 2010 14:51:40 +0100 Cezary Kaliszyk Change type schemes to name set.
Tue, 02 Mar 2010 14:24:57 +0100 Cezary Kaliszyk More fixes for new alpha, the whole lift script should now work again.
Tue, 02 Mar 2010 13:28:54 +0100 Cezary Kaliszyk Length fix for nested recursions.
Tue, 02 Mar 2010 12:28:07 +0100 Cezary Kaliszyk Fix equivp.
Tue, 02 Mar 2010 11:04:49 +0100 Cezary Kaliszyk Fixed eqvt code.
Tue, 02 Mar 2010 08:58:28 +0100 Christian Urban most tests work - the ones that do not I commented out
Tue, 02 Mar 2010 08:49:04 +0100 Cezary Kaliszyk merge
Tue, 02 Mar 2010 08:48:35 +0100 Cezary Kaliszyk Add a check of fv_functions.
Tue, 02 Mar 2010 08:43:53 +0100 Christian Urban some tuning
Tue, 02 Mar 2010 08:42:10 +0100 Cezary Kaliszyk Link calls to Raw permutations, FV definition and alpha_definition into the parser.
Tue, 02 Mar 2010 06:43:09 +0100 Christian Urban merged
Tue, 02 Mar 2010 06:42:43 +0100 Christian Urban rawified the bind specs (ready to be used now)
Mon, 01 Mar 2010 21:50:40 +0100 Cezary Kaliszyk merge
Mon, 01 Mar 2010 21:50:24 +0100 Cezary Kaliszyk Trying to prove equivariance.
Mon, 01 Mar 2010 19:23:08 +0100 Christian Urban modified for new binding format - hope it is the intended one
Mon, 01 Mar 2010 16:55:41 +0100 Christian Urban further code-refactoring in the parser
Mon, 01 Mar 2010 16:04:03 +0100 Cezary Kaliszyk The new alpha-equivalence and testing in Trm2 and Trm5.
Mon, 01 Mar 2010 14:26:14 +0100 Christian Urban slight simplification of the raw-decl generation
Mon, 01 Mar 2010 11:40:48 +0100 Cezary Kaliszyk Example that shows that current alpha is wrong.
Mon, 01 Mar 2010 07:46:50 +0100 Christian Urban added example from my phd
Sat, 27 Feb 2010 11:54:59 +0100 Christian Urban streamlined parser
Fri, 26 Feb 2010 18:38:25 +0100 Christian Urban generated the "binding list" from the input; at the moment it is only printed out as tracing; does not yet include the "bind itself binders"
Fri, 26 Feb 2010 18:21:39 +0100 Cezary Kaliszyk More about the general lifting procedure.
Fri, 26 Feb 2010 16:22:47 +0100 Cezary Kaliszyk Update TODO
Fri, 26 Feb 2010 16:15:03 +0100 Cezary Kaliszyk Progress with general lifting procedure.
Fri, 26 Feb 2010 15:42:00 +0100 Cezary Kaliszyk RSP of perms can be shown in one go.
Fri, 26 Feb 2010 15:10:55 +0100 Cezary Kaliszyk Change in signature of prove_const_rsp for general lifting.
Fri, 26 Feb 2010 13:57:43 +0100 Cezary Kaliszyk Permutation and FV_Alpha interface change.
Fri, 26 Feb 2010 10:34:04 +0100 Cezary Kaliszyk To call quotient it is enough to export the alpha frees to proper constants and their respective equivp theorems.
Thu, 25 Feb 2010 15:41:23 +0100 Cezary Kaliszyk merge
Thu, 25 Feb 2010 15:40:09 +0100 Cezary Kaliszyk Preparing the generalized lifting procedure
Thu, 25 Feb 2010 14:20:40 +0100 Christian Urban merged
Thu, 25 Feb 2010 14:20:10 +0100 Christian Urban added ott-example about Leroy96
Thu, 25 Feb 2010 14:14:40 +0100 Cezary Kaliszyk Forgot to add one file.
Thu, 25 Feb 2010 14:14:08 +0100 Cezary Kaliszyk Split Terms into separate files and add them to tests.
Thu, 25 Feb 2010 12:32:15 +0100 Cezary Kaliszyk merge
Thu, 25 Feb 2010 12:30:50 +0100 Cezary Kaliszyk Move the eqvt code out of Terms and fixed induction for single-rule examples.
Thu, 25 Feb 2010 12:24:37 +0100 Christian Urban merged
Thu, 25 Feb 2010 11:51:34 +0100 Christian Urban a few simplifications
Thu, 25 Feb 2010 11:30:00 +0100 Christian Urban first attempt to make sense out of the core-haskell definition
Thu, 25 Feb 2010 12:15:11 +0100 Cezary Kaliszyk Code for proving eqvt, still in Terms.
Thu, 25 Feb 2010 09:41:14 +0100 Cezary Kaliszyk Use eqvt infrastructure.
Thu, 25 Feb 2010 09:22:29 +0100 Cezary Kaliszyk Simple function eqvt code.
Thu, 25 Feb 2010 08:40:52 +0100 Christian Urban added IsaMakefile...but so far included only a test for the parser
Thu, 25 Feb 2010 07:57:17 +0100 Christian Urban moved Quot package to Attic (still compiles there with "isabelle make")
Thu, 25 Feb 2010 07:48:57 +0100 Christian Urban merged
Thu, 25 Feb 2010 07:48:33 +0100 Christian Urban moved Nominal to "toplevel"
Thu, 25 Feb 2010 07:05:52 +0100 Cezary Kaliszyk Export perm_frees.
Wed, 24 Feb 2010 23:25:30 +0100 Cezary Kaliszyk Restructuring the code in Perm
Wed, 24 Feb 2010 18:38:49 +0100 Cezary Kaliszyk Simplified and finised eqvt proofs for t1 and t5
Wed, 24 Feb 2010 17:42:52 +0100 Cezary Kaliszyk merge
Wed, 24 Feb 2010 17:42:37 +0100 Cezary Kaliszyk Define lifted perms.
Wed, 24 Feb 2010 17:32:43 +0100 Christian Urban merged
Wed, 24 Feb 2010 17:32:22 +0100 Christian Urban parsing and definition of raw datatype and bv-function work (not very beautiful)
Wed, 24 Feb 2010 15:39:17 +0100 Cezary Kaliszyk With permute_rsp we can lift the instance proofs :).
Wed, 24 Feb 2010 15:36:07 +0100 Cezary Kaliszyk Note the instance proofs, since they can be easily lifted.
Wed, 24 Feb 2010 15:13:22 +0100 Cezary Kaliszyk More refactoring and removed references to the global simpset in Perm.
Wed, 24 Feb 2010 14:55:09 +0100 Cezary Kaliszyk Factor-out 'prove_perm_empty'; I plan to use it in defining permutations on the lifted type.
Wed, 24 Feb 2010 14:37:51 +0100 Cezary Kaliszyk Regularize finite support proof for trm1
Wed, 24 Feb 2010 14:09:34 +0100 Cezary Kaliszyk Made the fv-supp proof much more straightforward.
Wed, 24 Feb 2010 12:06:55 +0100 Cezary Kaliszyk Regularize the proofs about finite support.
Wed, 24 Feb 2010 11:28:34 +0100 Cezary Kaliszyk Respects of permute and constructors.
Wed, 24 Feb 2010 11:03:30 +0100 Cezary Kaliszyk Generate fv_rsp automatically.
Wed, 24 Feb 2010 10:59:31 +0100 Cezary Kaliszyk Define the constants automatically.
Wed, 24 Feb 2010 10:47:41 +0100 Cezary Kaliszyk Rename also the lifted types to non-capital.
Wed, 24 Feb 2010 10:44:38 +0100 Cezary Kaliszyk Use the infrastructure in LF. Much shorter :).
Wed, 24 Feb 2010 10:38:45 +0100 Cezary Kaliszyk Final synchronization of names.
Wed, 24 Feb 2010 10:25:59 +0100 Cezary Kaliszyk LF renaming part 3 (proper names of alpha equvalences)
Wed, 24 Feb 2010 10:08:54 +0100 Cezary Kaliszyk LF renaming part 2 (proper fv functions)
Wed, 24 Feb 2010 09:58:44 +0100 Cezary Kaliszyk merge
Wed, 24 Feb 2010 09:58:12 +0100 Cezary Kaliszyk LF renaming part1.
Wed, 24 Feb 2010 09:56:32 +0100 Christian Urban merged
Wed, 24 Feb 2010 09:56:12 +0100 Christian Urban parsing of function definitions almost works now; still an error with undefined constants
Tue, 23 Feb 2010 18:28:48 +0100 Cezary Kaliszyk merge
Tue, 23 Feb 2010 18:27:32 +0100 Cezary Kaliszyk rsp for bv; the only issue is that it requires an appropriate induction principle.
Tue, 23 Feb 2010 16:32:04 +0100 Christian Urban merged
Tue, 23 Feb 2010 16:31:40 +0100 Christian Urban declarartion of the raw datatype already works; raw binding functions throw an exception about mutual recursive types
Tue, 23 Feb 2010 16:12:30 +0100 Cezary Kaliszyk rsp infrastructure.
Tue, 23 Feb 2010 14:20:42 +0100 Cezary Kaliszyk merge
Tue, 23 Feb 2010 14:19:44 +0100 Cezary Kaliszyk Progress towards automatic rsp of constants and fv.
Tue, 23 Feb 2010 13:33:01 +0100 Christian Urban merged
Tue, 23 Feb 2010 13:32:35 +0100 Christian Urban "raw"-ified the term-constructors and types given in the specification
Tue, 23 Feb 2010 12:49:45 +0100 Cezary Kaliszyk Looking at proving the rsp rules automatically.
Tue, 23 Feb 2010 11:56:47 +0100 Cezary Kaliszyk Minor beutification.
Tue, 23 Feb 2010 11:22:06 +0100 Cezary Kaliszyk Define the quotient from ML
Tue, 23 Feb 2010 10:47:14 +0100 Cezary Kaliszyk All works in LF but will require renaming.
Tue, 23 Feb 2010 09:34:41 +0100 Cezary Kaliszyk Reordering in LF.
Tue, 23 Feb 2010 09:31:59 +0100 Cezary Kaliszyk Fixes for auxiliary datatypes.
Mon, 22 Feb 2010 18:09:44 +0100 Cezary Kaliszyk Fixed pseudo_injectivity for trm4
Mon, 22 Feb 2010 17:19:28 +0100 Cezary Kaliszyk Testing auto equivp code.
Mon, 22 Feb 2010 16:44:58 +0100 Cezary Kaliszyk A tactic for final equivp
Mon, 22 Feb 2010 16:16:04 +0100 Cezary Kaliszyk More equivp infrastructure.
Mon, 22 Feb 2010 15:41:30 +0100 Cezary Kaliszyk tactify transp
Mon, 22 Feb 2010 15:09:53 +0100 Cezary Kaliszyk export the reflp and symp tacs.
Mon, 22 Feb 2010 15:03:48 +0100 Cezary Kaliszyk Generalize atom_trans and atom_sym.
Mon, 22 Feb 2010 14:50:53 +0100 Cezary Kaliszyk Some progress about transp
Mon, 22 Feb 2010 13:41:13 +0100 Cezary Kaliszyk alpha-symmetric addons.
Mon, 22 Feb 2010 12:12:32 +0100 Cezary Kaliszyk alpha reflexivity
Mon, 22 Feb 2010 10:57:39 +0100 Cezary Kaliszyk Renaming.
Mon, 22 Feb 2010 10:39:05 +0100 Cezary Kaliszyk Added missing description.
Mon, 22 Feb 2010 10:16:13 +0100 Cezary Kaliszyk Added Brian's suggestion.
Mon, 22 Feb 2010 09:55:43 +0100 Cezary Kaliszyk Update TODO
Sun, 21 Feb 2010 22:39:11 +0100 Cezary Kaliszyk Removed bindings 'in itself' where possible.
Sat, 20 Feb 2010 06:31:03 +0100 Cezary Kaliszyk Some adaptation
Fri, 19 Feb 2010 17:50:43 +0100 Cezary Kaliszyk proof cleaning and standardizing.
Fri, 19 Feb 2010 16:45:24 +0100 Cezary Kaliszyk Automatic production and proving of pseudo-injectivity.
Fri, 19 Feb 2010 12:05:58 +0100 Cezary Kaliszyk Experiments for the pseudo-injectivity tactic.
Fri, 19 Feb 2010 10:26:38 +0100 Cezary Kaliszyk merge
Fri, 19 Feb 2010 10:17:35 +0100 Cezary Kaliszyk Constructing alpha_inj goal.
Thu, 18 Feb 2010 23:07:52 +0100 Christian Urban merged
Thu, 18 Feb 2010 23:07:28 +0100 Christian Urban start work with the parser
Thu, 18 Feb 2010 18:33:53 +0100 Cezary Kaliszyk Full alpha equivalence + testing in terms. Some differ but it seems the generated version is more correct.
Thu, 18 Feb 2010 15:03:09 +0100 Cezary Kaliszyk First (non-working) version of alpha-equivalence
Thu, 18 Feb 2010 13:36:38 +0100 Cezary Kaliszyk Description of the fv procedure.
Thu, 18 Feb 2010 12:06:59 +0100 Cezary Kaliszyk Testing auto constant lifting.
Thu, 18 Feb 2010 11:28:20 +0100 Cezary Kaliszyk Fix for new Isabelle (primrec)
Thu, 18 Feb 2010 11:19:16 +0100 Cezary Kaliszyk Automatic lifting of constants.
Thu, 18 Feb 2010 10:01:48 +0100 Cezary Kaliszyk Changed back to original version of trm5
Thu, 18 Feb 2010 10:00:58 +0100 Cezary Kaliszyk The alternate version of trm5 with additional binding. All proofs work the same.
Thu, 18 Feb 2010 09:46:38 +0100 Cezary Kaliszyk Code for handling atom sets.
Thu, 18 Feb 2010 08:43:13 +0100 Cezary Kaliszyk Replace Terms by Terms2.
Thu, 18 Feb 2010 08:37:45 +0100 Cezary Kaliszyk Fixed proofs in Terms2 and found a mistake in Terms.
Wed, 17 Feb 2010 17:51:35 +0100 Cezary Kaliszyk Terms2 with bindings for binders synchronized with bindings they are used in.
Wed, 17 Feb 2010 17:29:26 +0100 Cezary Kaliszyk Cleaning of proofs in Terms.
Wed, 17 Feb 2010 16:22:16 +0100 Cezary Kaliszyk Testing Fv
Wed, 17 Feb 2010 15:52:08 +0100 Cezary Kaliszyk Fix the strong induction principle.
Wed, 17 Feb 2010 15:45:03 +0100 Cezary Kaliszyk Reorder
Wed, 17 Feb 2010 15:28:50 +0100 Cezary Kaliszyk Add bindings of recursive types by free_variables.
Wed, 17 Feb 2010 15:20:22 +0100 Cezary Kaliszyk Bindings adapted to multiple defined datatypes.
Wed, 17 Feb 2010 15:00:04 +0100 Cezary Kaliszyk Reorganization
Wed, 17 Feb 2010 14:44:32 +0100 Cezary Kaliszyk Now should work.
Wed, 17 Feb 2010 14:35:06 +0100 Cezary Kaliszyk Some optimizations and fixes.
Wed, 17 Feb 2010 14:17:02 +0100 Cezary Kaliszyk Simplified format of bindings.
Wed, 17 Feb 2010 13:56:31 +0100 Cezary Kaliszyk Tested the Perm code; works everywhere in Terms.
Wed, 17 Feb 2010 13:54:35 +0100 Cezary Kaliszyk Wrapped the permutation code.
Wed, 17 Feb 2010 10:20:26 +0100 Cezary Kaliszyk Description of intended bindings.
Wed, 17 Feb 2010 10:12:01 +0100 Cezary Kaliszyk Code for generating the fv function, no bindings yet.
Wed, 17 Feb 2010 09:27:02 +0100 Cezary Kaliszyk merge
Wed, 17 Feb 2010 09:26:49 +0100 Cezary Kaliszyk indent
Wed, 17 Feb 2010 09:26:38 +0100 Cezary Kaliszyk merge
Wed, 17 Feb 2010 09:26:10 +0100 Cezary Kaliszyk Simplifying perm_eq
Tue, 16 Feb 2010 15:13:14 +0100 Cezary Kaliszyk merge
Tue, 16 Feb 2010 15:12:31 +0100 Cezary Kaliszyk indenting
Tue, 16 Feb 2010 15:12:49 +0100 Cezary Kaliszyk Minor
Tue, 16 Feb 2010 14:57:39 +0100 Cezary Kaliszyk Merge
Tue, 16 Feb 2010 14:57:22 +0100 Cezary Kaliszyk Ported Stefan's permutation code, still needs some localizing.
Mon, 15 Feb 2010 16:54:09 +0100 Cezary Kaliszyk merge
Mon, 15 Feb 2010 16:53:51 +0100 Cezary Kaliszyk Removed varifyT.
Mon, 15 Feb 2010 17:02:46 +0100 Christian Urban merged
Mon, 15 Feb 2010 17:02:26 +0100 Christian Urban 2-spaces rule (where it makes sense)
Mon, 15 Feb 2010 16:52:32 +0100 Cezary Kaliszyk merge
Mon, 15 Feb 2010 16:51:30 +0100 Cezary Kaliszyk Fixed the definition of less and finished the missing proof.
Mon, 15 Feb 2010 16:50:11 +0100 Christian Urban further tuning
Mon, 15 Feb 2010 16:37:48 +0100 Christian Urban small tuning
Mon, 15 Feb 2010 16:28:07 +0100 Christian Urban tuned the parsing and testing code in quotient_def.ML; cleaned out old stuff in AbsRepTest.thy
Mon, 15 Feb 2010 14:58:03 +0100 Cezary Kaliszyk der_bname -> derived_bname
Mon, 15 Feb 2010 14:51:17 +0100 Cezary Kaliszyk Names of files.
Mon, 15 Feb 2010 14:28:03 +0100 Cezary Kaliszyk Finished introducing the binding.
Mon, 15 Feb 2010 13:40:03 +0100 Cezary Kaliszyk Synchronize the commands.
Mon, 15 Feb 2010 12:23:02 +0100 Cezary Kaliszyk Passing the binding to quotient_def
Mon, 15 Feb 2010 12:15:14 +0100 Cezary Kaliszyk Added a binding to the parser.
Mon, 15 Feb 2010 10:25:17 +0100 Cezary Kaliszyk Second inline
Mon, 15 Feb 2010 10:11:26 +0100 Cezary Kaliszyk remove one-line wrapper.
Fri, 12 Feb 2010 16:27:25 +0100 Cezary Kaliszyk Undid the read_terms change; now compiles.
Fri, 12 Feb 2010 16:06:09 +0100 Cezary Kaliszyk merge
Fri, 12 Feb 2010 16:04:10 +0100 Cezary Kaliszyk renamed 'as' to 'is' everywhere.
Fri, 12 Feb 2010 15:50:43 +0100 Cezary Kaliszyk "is" defined as the keyword
Fri, 12 Feb 2010 15:06:20 +0100 Christian Urban moved "strange" lemma to quotient_tacs; marked a number of lemmas as unused; tuned
Fri, 12 Feb 2010 12:06:09 +0100 Cezary Kaliszyk The lattice instantiations are gone from Isabelle/Main, so
Thu, 11 Feb 2010 17:58:06 +0100 Cezary Kaliszyk the lam/bla example.
Thu, 11 Feb 2010 16:54:04 +0100 Cezary Kaliszyk Finished a working foo/bar.
Thu, 11 Feb 2010 16:05:15 +0100 Cezary Kaliszyk fv_foo is not regular.
Thu, 11 Feb 2010 15:08:45 +0100 Cezary Kaliszyk Testing foo/bar
Thu, 11 Feb 2010 14:23:26 +0100 Cezary Kaliszyk Even when bv = fv it still doesn't lift.
Thu, 11 Feb 2010 14:02:34 +0100 Cezary Kaliszyk Added the missing syntax file
Thu, 11 Feb 2010 14:00:00 +0100 Cezary Kaliszyk Notation available locally
Thu, 11 Feb 2010 10:06:02 +0100 Cezary Kaliszyk Main renaming + fixes for new Isabelle in IntEx2.
Thu, 11 Feb 2010 09:23:59 +0100 Cezary Kaliszyk Merging QuotBase into QuotMain.
Wed, 10 Feb 2010 21:39:40 +0100 Christian Urban removed dead code
Wed, 10 Feb 2010 20:35:54 +0100 Christian Urban cleaned a bit
Wed, 10 Feb 2010 17:22:18 +0100 Cezary Kaliszyk lowercase locale
Wed, 10 Feb 2010 17:10:52 +0100 Cezary Kaliszyk hg-added the added file.
(0) -1000 -256 +256 +1000 tip