Wed, 15 Jun 2011 09:50:53 +0900 Cezary Kaliszyk Some TODOs
Wed, 15 Jun 2011 09:31:59 +0900 Cezary Kaliszyk merge
Wed, 15 Jun 2011 09:25:36 +0900 Cezary Kaliszyk TypeSchemes work with 'default'.
Tue, 14 Jun 2011 19:11:44 +0100 Christian Urban tuned some proofs
Tue, 14 Jun 2011 14:07:07 +0100 Christian Urban fixed the problem when giving a complex default-term; the fundef lemmas in Nominal_Base were not general enough
Tue, 14 Jun 2011 11:43:06 +0100 Christian Urban tuned
Fri, 10 Jun 2011 15:52:17 +0900 Cezary Kaliszyk Move working examples before non-working ones
Fri, 10 Jun 2011 15:45:49 +0900 Cezary Kaliszyk Optimized proofs and removed some garbage.
Fri, 10 Jun 2011 15:31:14 +0900 Cezary Kaliszyk merge
Fri, 10 Jun 2011 15:30:09 +0900 Cezary Kaliszyk Slightly modify fcb for list1 and put in common place.
Fri, 10 Jun 2011 09:00:24 +0900 Cezary Kaliszyk Experiments with Let
Thu, 09 Jun 2011 15:34:51 +0900 Cezary Kaliszyk Eval can be defined with additional freshness
Thu, 09 Jun 2011 15:03:58 +0900 Cezary Kaliszyk Minor simplification
Thu, 09 Jun 2011 11:10:41 +0900 Cezary Kaliszyk abs_res_fcb will be enough to finish the multiple-recursive proof, if we have a working 'default'.
Thu, 09 Jun 2011 09:44:51 +0900 Cezary Kaliszyk More experiments with 'default'
Wed, 08 Jun 2011 21:44:03 +0900 Cezary Kaliszyk Finished the proof with the invariant
Wed, 08 Jun 2011 21:32:35 +0900 Cezary Kaliszyk Issue with 'default'
Wed, 08 Jun 2011 12:30:56 +0100 Christian Urban merged
Wed, 08 Jun 2011 12:30:46 +0100 Christian Urban merged
Wed, 08 Jun 2011 08:44:01 +0100 Christian Urban using the option "default" the function package allows one to give an explicit default value
Wed, 08 Jun 2011 17:52:06 +0900 Cezary Kaliszyk Simpler proof of TypeSchemes/substs
Wed, 08 Jun 2011 17:25:54 +0900 Cezary Kaliszyk Simplify fcb_res
Wed, 08 Jun 2011 09:56:39 +0900 Cezary Kaliszyk FCB for res binding and simplified proof of subst for type schemes
Wed, 08 Jun 2011 07:06:20 +0900 Cezary Kaliszyk Simplify ln-trans proof
Wed, 08 Jun 2011 07:02:52 +0900 Cezary Kaliszyk cbvs can be easily defined without an invariant
Tue, 07 Jun 2011 20:58:00 +0100 Christian Urban defined the "count-bound-variables-occurences" function which has an accumulator like trans
Tue, 07 Jun 2011 17:45:38 +0100 Christian Urban merged
Tue, 07 Jun 2011 23:42:12 +0900 Cezary Kaliszyk remove garbage (proofs that assumes the invariant outside function)
Tue, 07 Jun 2011 23:38:39 +0900 Cezary Kaliszyk Proof of trans with invariant
Tue, 07 Jun 2011 23:22:58 +0900 Cezary Kaliszyk Testing invariant in Lambda_F_T
Tue, 07 Jun 2011 10:40:06 +0100 Christian Urban cleaned ups a bit the examples with the invariant framework; exported nominal_function_config datatype into separate structure and file
Tue, 07 Jun 2011 08:52:59 +0100 Christian Urban fixed problem with earlier commit about nominal_function_common; added facility for specifying an invariant - added a definition of frees_set which need a finiteness invariant
Mon, 06 Jun 2011 13:11:04 +0100 Christian Urban slightly stronger property in fundef_ex_prop
Sun, 05 Jun 2011 21:14:23 +0100 Christian Urban added an option for an invariant (at the moment only a stub)
Sun, 05 Jun 2011 16:58:18 +0100 Christian Urban added a more general lemma fro fundef_ex1
Sat, 04 Jun 2011 14:50:57 +0900 Cezary Kaliszyk Trying the induction on the graph
Sat, 04 Jun 2011 09:07:50 +0900 Cezary Kaliszyk Finish and test the locale approach
Fri, 03 Jun 2011 22:31:44 +0900 Cezary Kaliszyk FiniteSupp precondition in the function is enough to get rid of completeness obligationss
Fri, 03 Jun 2011 12:46:23 +0100 Christian Urban recursion combinator inside a locale
Fri, 03 Jun 2011 18:33:11 +0900 Cezary Kaliszyk merge
Fri, 03 Jun 2011 18:32:22 +0900 Cezary Kaliszyk F for lambda used to define translation to locally nameless
Thu, 02 Jun 2011 16:15:18 +0100 Christian Urban typo
Thu, 02 Jun 2011 15:35:33 +0100 Christian Urban removed dead code
Thu, 02 Jun 2011 22:24:33 +0900 Cezary Kaliszyk finished the missing obligations
Thu, 02 Jun 2011 12:14:03 +0100 Christian Urban merged
Thu, 02 Jun 2011 12:09:31 +0100 Christian Urban a test with a recursion combinator defined on top of nominal_primrec
Thu, 02 Jun 2011 16:41:09 +0900 Cezary Kaliszyk Use FCB to simplify proof
Thu, 02 Jun 2011 10:11:50 +0900 Cezary Kaliszyk merge
Thu, 02 Jun 2011 10:09:23 +0900 Cezary Kaliszyk Remove SMT
Wed, 01 Jun 2011 22:55:14 +0100 Christian Urban hopefully final fix for ho-functions
Wed, 01 Jun 2011 21:03:30 +0100 Christian Urban first test to fix the problem with free variables
Wed, 01 Jun 2011 16:13:42 +0900 Cezary Kaliszyk proved subst for All constructor in type schemes.
Wed, 01 Jun 2011 13:41:30 +0900 Cezary Kaliszyk DB translation using index; easier to reason about.
Wed, 01 Jun 2011 13:35:37 +0900 Cezary Kaliszyk Problem: free variables in the goal
Wed, 01 Jun 2011 11:01:39 +0900 Cezary Kaliszyk fixed previous commit
Wed, 01 Jun 2011 10:59:07 +0900 Cezary Kaliszyk equivariance of db_trans
Tue, 31 May 2011 12:22:28 +0100 Christian Urban fixed the problem with cps-like functions
Tue, 31 May 2011 14:12:31 +0900 Cezary Kaliszyk DeBruijn translation in a simplifier friendly way
Tue, 31 May 2011 13:25:35 +0900 Cezary Kaliszyk map_term can be defined when equivariance is assumed
Tue, 31 May 2011 13:21:00 +0900 Cezary Kaliszyk map_term is not a function the way it is defined
Tue, 31 May 2011 12:59:10 +0900 Cezary Kaliszyk Defined translation from nominal to de-Bruijn; with a freshness condition for the lambda case.
Tue, 31 May 2011 12:54:21 +0900 Cezary Kaliszyk Simple eqvt proofs with perm_simps for clarity
Tue, 31 May 2011 00:36:16 +0100 Christian Urban tuned last commit
Tue, 31 May 2011 00:17:22 +0100 Christian Urban functions involving if and case do not throw exceptions anymore; but eqvt_at assumption has now a precondition
Thu, 26 May 2011 06:36:29 +0200 Christian Urban updated to new Isabelle
Wed, 25 May 2011 21:38:50 +0200 Christian Urban added eq_iff and distinct lemmas of nominal datatypes to the simplifier
Tue, 24 May 2011 19:39:38 +0200 Christian Urban more on slides
Sun, 22 May 2011 10:20:18 +0200 Christian Urban added slides for copenhagen
Sat, 14 May 2011 10:16:16 +0100 Christian Urban added a problem with inductive_cases (reported by Randy)
Fri, 13 May 2011 14:50:17 +0100 Christian Urban misc
Tue, 10 May 2011 17:10:22 +0100 Christian Urban made the subtyping work again
Tue, 10 May 2011 07:47:06 +0100 Christian Urban updated to new Isabelle (> 9 May)
Mon, 09 May 2011 04:49:58 +0100 Christian Urban merged
Tue, 03 May 2011 15:39:30 +0100 Christian Urban added two mutual recursive inductive definitions
Tue, 03 May 2011 13:25:02 +0100 Christian Urban deleted two functions from the API
Tue, 03 May 2011 13:09:08 +0100 Christian Urban proved that lfp is equivariant (that simplifies equivariance proofs of inductively defined predicates)
Mon, 09 May 2011 04:46:43 +0100 Christian Urban more on pearl-paper
Wed, 04 May 2011 15:27:04 +0800 Christian Urban more on pearl-paper
Mon, 02 May 2011 13:01:02 +0800 Christian Urban updated Quotient paper so that it compiles again
Thu, 28 Apr 2011 11:51:01 +0800 Christian Urban merged
Thu, 28 Apr 2011 11:44:36 +0800 Christian Urban added slides for beijing
Fri, 22 Apr 2011 00:18:25 +0800 Christian Urban more to the pearl paper
Tue, 19 Apr 2011 13:03:08 +0100 Christian Urban updated to snapshot Isabelle 19 April
Mon, 18 Apr 2011 15:57:45 +0100 Christian Urban merged
Mon, 18 Apr 2011 15:56:07 +0100 Christian Urban added permute_pure back into the nominal_inductive procedure; updated to Isabelle 17 April
Fri, 15 Apr 2011 15:20:56 +0900 Cezary Kaliszyk New way of forward elimination of Abs1_eq and simplifications of the function obligation proofs.
Wed, 13 Apr 2011 13:44:25 +0100 Christian Urban merged
Wed, 13 Apr 2011 13:41:52 +0100 Christian Urban introduced framework for finetuning eqvt-rules; this solves problem with permute_pure called in nominal_inductive
Tue, 12 Apr 2011 15:46:35 +0800 Christian Urban shanghai slides
Mon, 11 Apr 2011 02:25:25 +0100 Christian Urban pictures for slides
Mon, 11 Apr 2011 02:04:11 +0100 Christian Urban Shanghai slides
Sun, 10 Apr 2011 14:13:55 +0800 Christian Urban more paper
Sun, 10 Apr 2011 07:41:52 +0800 Christian Urban eqvt of supp and fresh is proved using equivariance infrastructure
Sun, 10 Apr 2011 04:07:15 +0800 Christian Urban more paper
Sat, 09 Apr 2011 13:44:49 +0800 Christian Urban more on the paper
Sat, 09 Apr 2011 00:29:40 +0100 Christian Urban tuned paper
Sat, 09 Apr 2011 00:28:53 +0100 Christian Urban tuned paper
Sat, 09 Apr 2011 02:10:49 +0800 Christian Urban typo
Fri, 08 Apr 2011 14:23:28 +0800 Christian Urban more on paper
Fri, 08 Apr 2011 03:47:50 +0800 Christian Urban eqvt_lambda without eta-expansion
Wed, 06 Apr 2011 13:47:08 +0100 Christian Urban changed default preprocessor that does not catch variables only occuring on the right
Thu, 31 Mar 2011 15:25:35 +0200 Christian Urban final version of slides
Wed, 30 Mar 2011 22:27:26 +0200 Christian Urban more on the slides
Wed, 30 Mar 2011 08:11:36 +0200 Christian Urban tuned IsaMakefile
Tue, 29 Mar 2011 23:52:14 +0200 Christian Urban rearranged directories and updated to new Isabelle
Wed, 16 Mar 2011 21:14:43 +0100 Christian Urban precise path to LaTeXsugar
Wed, 16 Mar 2011 21:07:50 +0100 Christian Urban a lit bit more on the pearl-jv paper
Wed, 16 Mar 2011 20:42:14 +0100 Christian Urban ported changes from function package....needs Isabelle 16 March or above
Tue, 15 Mar 2011 00:40:39 +0100 Christian Urban more on the pearl paper
Mon, 14 Mar 2011 16:35:59 +0100 Christian Urban equivariance for All and Ex can be proved in terms of their definition
Fri, 11 Mar 2011 08:51:39 +0000 Christian Urban more on the paper
Tue, 08 Mar 2011 09:07:49 +0000 Christian Urban merged
Tue, 08 Mar 2011 09:07:27 +0000 Christian Urban more on the pearl paper
Wed, 02 Mar 2011 16:07:56 +0900 Cezary Kaliszyk distinct names at toplevel
Wed, 02 Mar 2011 12:49:01 +0900 Cezary Kaliszyk merge
Wed, 02 Mar 2011 12:48:00 +0900 Cezary Kaliszyk Pairing function
Wed, 02 Mar 2011 00:06:28 +0000 Christian Urban updated pearl papers
Tue, 01 Mar 2011 00:14:02 +0000 Christian Urban a bit more tuning
Mon, 28 Feb 2011 16:47:13 +0000 Christian Urban included old test cases for perm_simp into ROOT.ML file
Mon, 28 Feb 2011 15:21:10 +0000 Christian Urban split the library into a basics file; merged Nominal_Eqvt into Nominal_Base
Fri, 25 Feb 2011 21:23:30 +0000 Christian Urban some slight polishing
Thu, 24 Feb 2011 18:50:02 +0000 Christian Urban merged
Thu, 24 Feb 2011 16:26:11 +0000 Christian Urban added a lemma about fresh_star and Abs
Wed, 23 Feb 2011 11:11:02 +0900 Cezary Kaliszyk Reduce the definition of trans to FCB; test that FCB can be proved with simp rules.
Sat, 19 Feb 2011 09:31:22 +0900 Cezary Kaliszyk typeschemes/subst
Thu, 17 Feb 2011 17:02:25 +0900 Cezary Kaliszyk further experiments with typeschemes subst
Thu, 17 Feb 2011 12:01:08 +0900 Cezary Kaliszyk Finished the proof of a function that invents fresh variable names.
Wed, 16 Feb 2011 14:44:33 +0000 Christian Urban added eqvt for length
Wed, 16 Feb 2011 14:03:26 +0000 Christian Urban added eqvt lemmas for filter and distinct
Mon, 07 Feb 2011 16:00:24 +0000 Christian Urban added eqvt for cartesian products
Mon, 07 Feb 2011 15:59:37 +0000 Christian Urban cleaned up the experiments so that the tests go through
Sat, 05 Feb 2011 07:39:00 +0900 Cezary Kaliszyk merge
Sat, 05 Feb 2011 07:38:22 +0900 Cezary Kaliszyk Experiments defining a function on Let
Fri, 04 Feb 2011 04:45:04 +0000 Christian Urban updated TODO
Fri, 04 Feb 2011 03:52:38 +0000 Christian Urban Lambda.thy which works with Nominal_Isabelle2011
Thu, 03 Feb 2011 02:57:04 +0000 Christian Urban merged
Thu, 03 Feb 2011 02:51:57 +0000 Christian Urban removed diagnostic code
Tue, 01 Feb 2011 09:07:55 +0900 Cezary Kaliszyk Only one of the subgoals is needed
Tue, 01 Feb 2011 08:57:50 +0900 Cezary Kaliszyk Experiments with substitution on set+
Tue, 01 Feb 2011 08:48:14 +0900 Cezary Kaliszyk More properties that relate abs_res and abs_set. Also abs_res with less binders.
Sun, 30 Jan 2011 12:09:23 +0900 Cezary Kaliszyk alpha_res implies alpha_set :)
Sun, 30 Jan 2011 09:57:37 +0900 Cezary Kaliszyk Showing that the binders difference is fresh for the left side solves the goal for 'set'.
Sat, 29 Jan 2011 14:26:47 +0900 Cezary Kaliszyk Experiments with functions
Thu, 27 Jan 2011 20:19:13 +0100 Christian Urban some experiments
Thu, 27 Jan 2011 04:24:17 +0100 Christian Urban the proofs with eqvt_at
Tue, 25 Jan 2011 18:58:26 +0100 Christian Urban made eqvt-proof explicit in the function definitions
Tue, 25 Jan 2011 02:51:44 +0900 Cezary Kaliszyk merge
Tue, 25 Jan 2011 02:46:05 +0900 Cezary Kaliszyk minor
Tue, 25 Jan 2011 02:42:15 +0900 Cezary Kaliszyk Down as infixr
Sat, 22 Jan 2011 23:24:20 -0600 Christian Urban added some slides
Sun, 23 Jan 2011 03:29:22 +0100 Christian Urban added Tutorial6
Sat, 22 Jan 2011 18:59:48 -0600 Christian Urban cleaning up
Sat, 22 Jan 2011 16:37:00 -0600 Christian Urban merged
Sat, 22 Jan 2011 16:36:21 -0600 Christian Urban cleaned up Tutorial 3 with solutions
Sun, 23 Jan 2011 07:32:28 +0900 Cezary Kaliszyk Missing val.simps
Sun, 23 Jan 2011 07:17:35 +0900 Cezary Kaliszyk merge
Sun, 23 Jan 2011 07:15:59 +0900 Cezary Kaliszyk Tutorial 4s
Sat, 22 Jan 2011 16:04:40 -0600 Christian Urban cleaned up and solution section
Sat, 22 Jan 2011 15:07:36 -0600 Christian Urban cleaned up tutorial1...added solution file
Sat, 22 Jan 2011 12:46:01 -0600 Christian Urban better version of Tutorial 1
Fri, 21 Jan 2011 22:58:03 +0100 Christian Urban better flow of proofs and definitions and proof
Fri, 21 Jan 2011 22:23:44 +0100 Christian Urban separated type preservation and progress into a separate file
Fri, 21 Jan 2011 22:02:34 +0100 Christian Urban substitution lemma in separate file
Fri, 21 Jan 2011 21:58:51 +0100 Christian Urban added unbind example
Fri, 21 Jan 2011 00:55:28 +0100 Christian Urban a bit tuning
Thu, 20 Jan 2011 23:19:30 +0100 Christian Urban first split of tutorrial theory
Wed, 19 Jan 2011 23:58:12 +0100 Christian Urban added a very rough version of the tutorial; all seems to work
Wed, 19 Jan 2011 19:41:50 +0100 Christian Urban added obtain_fresh lemma; tuned Lambda.thy
Wed, 19 Jan 2011 19:06:52 +0100 Christian Urban base file for the tutorial (contains definitions for heigt, subst and beta-reduction)
Wed, 19 Jan 2011 18:56:28 +0100 Christian Urban ported some of the old proofs to serve as testcases
Wed, 19 Jan 2011 18:07:29 +0100 Christian Urban added eqvt and supp lemma for removeAll (function from List.thy)
Wed, 19 Jan 2011 17:54:50 +0100 Christian Urban theory name as it should be
Wed, 19 Jan 2011 17:54:06 +0100 Christian Urban removed diagnostic code
Wed, 19 Jan 2011 17:11:10 +0100 Christian Urban added Minimal file to test things
Wed, 19 Jan 2011 07:06:47 +0100 Christian Urban defined height as a function that returns an integer
Tue, 18 Jan 2011 21:28:07 +0100 Christian Urban deleted diagnostic code
Tue, 18 Jan 2011 21:26:58 +0100 Christian Urban some tryes about substitution over type-schemes
Tue, 18 Jan 2011 19:27:30 +0100 Christian Urban defined properly substitution
Tue, 18 Jan 2011 18:04:40 +0100 Christian Urban derived stronger Abs_eq_iff2 theorems
Tue, 18 Jan 2011 17:30:47 +0100 Christian Urban made alpha_abs_set_stronger1 stronger
Tue, 18 Jan 2011 17:19:50 +0100 Christian Urban removed finiteness assumption from set_rename_perm
Tue, 18 Jan 2011 22:11:49 +0900 Cezary Kaliszyk alpha_abs_set_stronger1
Tue, 18 Jan 2011 21:12:25 +0900 Cezary Kaliszyk alpha_abs_let_stronger is not true in the same form
Tue, 18 Jan 2011 11:02:57 +0100 Christian Urban the function translating lambda terms to locally nameless lambda terms; still needs a stronger abs_eq_iff lemma...at the moment only proved for restrictions
Tue, 18 Jan 2011 06:55:18 +0100 Christian Urban modified the renaming_perm lemmas
Mon, 17 Jan 2011 17:20:21 +0100 Christian Urban added a translation function from lambda-terms to deBruijn terms (equivariance fails at the moment)
Mon, 17 Jan 2011 15:12:03 +0100 Christian Urban added a few examples of functions to Lambda.thy
Mon, 17 Jan 2011 14:37:18 +0100 Christian Urban exported nominal function code to external file
Mon, 17 Jan 2011 12:37:37 +0000 Christian Urban removed old testing code from Lambda.thy
Mon, 17 Jan 2011 12:34:11 +0000 Christian Urban moved high level code from LamTest into the main libraries.
Mon, 17 Jan 2011 12:33:37 +0000 Christian Urban eliminated tracing code; added flag so that equivariance is only proved for the function graph, not the relation
Sat, 15 Jan 2011 21:16:15 +0000 Christian Urban subst also works now
Sat, 15 Jan 2011 20:24:16 +0000 Christian Urban nominal_function works now completely for frees and depth; still a propbelm with subst; no unproved assumptions
Fri, 14 Jan 2011 14:22:25 +0000 Christian Urban strengthened renaming lemmas
Thu, 13 Jan 2011 12:12:47 +0000 Christian Urban added eqvt_lemmas for subset and psubset
Mon, 10 Jan 2011 11:36:55 +0000 Christian Urban a few lemmas about freshness for at and at_base
Mon, 10 Jan 2011 08:51:51 +0000 Christian Urban added a property about finite support in the presense of eqvt_at
Sun, 09 Jan 2011 05:38:53 +0000 Christian Urban instantiated fundef_ex1_eqvt_at theorem with the indction hypothesis
Sun, 09 Jan 2011 04:28:24 +0000 Christian Urban solved subgoals for depth and subst function
Sun, 09 Jan 2011 01:17:44 +0000 Christian Urban added eqvt_at premises in function definition - however not proved at the moment
Fri, 07 Jan 2011 05:40:31 +0000 Christian Urban added one further lemma about equivariance of THE_default
Fri, 07 Jan 2011 05:06:25 +0000 Christian Urban equivariance of THE_default under the uniqueness assumption
Fri, 07 Jan 2011 02:30:00 +0000 Christian Urban derived equivariance for the function graph and function relation
Thu, 06 Jan 2011 23:06:45 +0000 Christian Urban a modified function package where, as a test, True has been injected into the compatibility condictions
Thu, 06 Jan 2011 20:25:40 +0000 Christian Urban removed last traces of debugging code
Thu, 06 Jan 2011 19:57:57 +0000 Christian Urban removed debugging code abd introduced a guarded tracing function
Thu, 06 Jan 2011 14:53:38 +0000 Christian Urban moved Weakening up....it does not compile when put at the last position
Thu, 06 Jan 2011 14:02:10 +0000 Christian Urban tuned
Thu, 06 Jan 2011 13:31:44 +0000 Christian Urban added weakening to the test cases
Thu, 06 Jan 2011 13:28:40 +0000 Christian Urban cleaned up weakening proof and added a version with finit sets
Thu, 06 Jan 2011 13:28:19 +0000 Christian Urban same
Thu, 06 Jan 2011 13:28:04 +0000 Christian Urban some further lemmas for fsets
Thu, 06 Jan 2011 11:00:16 +0000 Christian Urban made sure the raw datatypes and raw functions do not get any mixfix syntax
Wed, 05 Jan 2011 17:33:43 +0000 Christian Urban exported the code into a separate file
Wed, 05 Jan 2011 16:51:27 +0000 Christian Urban strong rule inductions; as an example the weakening lemma works
Tue, 04 Jan 2011 13:47:38 +0000 Christian Urban final version of the ESOP paper; used set+ instead of res as requested by one reviewer
Mon, 03 Jan 2011 16:21:12 +0000 Christian Urban file with most of the strong rule induction development
Mon, 03 Jan 2011 16:19:27 +0000 Christian Urban simple cases for string rule inductions
Fri, 31 Dec 2010 15:37:04 +0000 Christian Urban changed res keyword to set+ for restrictions; comment by a referee
Fri, 31 Dec 2010 13:31:39 +0000 Christian Urban added proper case names for all induct and exhaust theorems
Fri, 31 Dec 2010 12:12:59 +0000 Christian Urban added small example for strong inductions; functions still need a sorry
Thu, 30 Dec 2010 10:00:09 +0000 Christian Urban removed local fix for bug in induction_schema; added setup method for strong inductions
Tue, 28 Dec 2010 19:51:25 +0000 Christian Urban automated all strong induction lemmas
Tue, 28 Dec 2010 00:20:50 +0000 Christian Urban proper application of induction_schema and strong_exhaust rules; needs local fix in induction_schema.ML
Sun, 26 Dec 2010 16:35:16 +0000 Christian Urban generated goals for strong induction theorems.
Thu, 23 Dec 2010 01:05:05 +0000 Christian Urban test with strong inductions
Thu, 23 Dec 2010 00:46:06 +0000 Christian Urban moved all strong_exhaust code to nominal_dt_quot; tuned examples
Thu, 23 Dec 2010 00:22:41 +0000 Christian Urban moved generic functions into nominal_library
Wed, 22 Dec 2010 23:12:51 +0000 Christian Urban slight tuning
Wed, 22 Dec 2010 22:30:43 +0000 Christian Urban slight tuning
Wed, 22 Dec 2010 21:13:44 +0000 Christian Urban tuned examples
Wed, 22 Dec 2010 21:13:32 +0000 Christian Urban added fold_right which produces the correct term for left-infix operators
Wed, 22 Dec 2010 12:47:09 +0000 Christian Urban updated to Isabelle 22 December
Wed, 22 Dec 2010 12:17:49 +0000 Christian Urban a bit tuning
Wed, 22 Dec 2010 10:32:01 +0000 Christian Urban corrected premises of strong exhausts theorems
Wed, 22 Dec 2010 09:13:25 +0000 Christian Urban properly exported strong exhaust theorem; cleaned up some examples
Tue, 21 Dec 2010 10:28:08 +0000 Christian Urban all examples for strong exhausts work; recursive binders need to be treated differently; still unclean version with lots of diagnostic code
Sun, 19 Dec 2010 07:50:37 +0000 Christian Urban one interesting case done
Sun, 19 Dec 2010 07:43:32 +0000 Christian Urban a stronger statement for at_set_avoiding
Fri, 17 Dec 2010 01:01:44 +0000 Christian Urban tuned
Fri, 17 Dec 2010 00:39:27 +0000 Christian Urban tuned
Thu, 16 Dec 2010 08:42:48 +0000 Christian Urban simple cases for strong inducts done; infrastructure for the difficult ones is there
Thu, 16 Dec 2010 02:25:35 +0000 Christian Urban added theorem-rewriter conversion
Tue, 14 Dec 2010 14:23:40 +0000 Christian Urban freshness theorem in strong exhausts; (temporarily includes a cheat_tac to make all tests go through)
Sun, 12 Dec 2010 22:09:11 +0000 Christian Urban created strong_exhausts terms
Sun, 12 Dec 2010 00:10:40 +0000 Christian Urban moved setify and listify functions into the library; introduced versions that have a type argument
Fri, 10 Dec 2010 19:01:44 +0000 Christian Urban updated
Thu, 09 Dec 2010 18:12:42 +0000 Christian Urban a bit more tuning of the paper
Thu, 09 Dec 2010 17:10:08 +0000 Christian Urban brought the paper to 20 pages plus one page appendix
Wed, 08 Dec 2010 17:07:08 +0000 Christian Urban first tests about exhaust
Wed, 08 Dec 2010 13:16:25 +0000 Christian Urban moved some code into the nominal_library
Wed, 08 Dec 2010 13:05:04 +0000 Christian Urban moved definition of raw bn-functions into nominal_dt_rawfuns
Wed, 08 Dec 2010 12:37:25 +0000 Christian Urban kept the nested structure of constructors (belonging to one datatype)
Tue, 07 Dec 2010 19:16:09 +0000 Christian Urban moved general theorems into the libraries
Tue, 07 Dec 2010 14:27:39 +0000 Christian Urban automated permute_bn theorems
Tue, 07 Dec 2010 14:27:21 +0000 Christian Urban updated to changes in Isabelle
Mon, 06 Dec 2010 17:11:54 +0000 Christian Urban deleted nominal_dt_supp.ML
Mon, 06 Dec 2010 17:11:34 +0000 Christian Urban moved code from nominal_dt_supp to nominal_dt_quot
Mon, 06 Dec 2010 16:35:42 +0000 Christian Urban automated alpha_perm_bn theorems
Mon, 06 Dec 2010 14:24:17 +0000 Christian Urban ordered raw_bn_info to agree with the order of the raw_bn_functions; started alpha_bn proof
Fri, 03 Dec 2010 13:51:07 +0000 Christian Urban updated to Isabelle 2nd December
Mon, 29 Nov 2010 08:01:09 +0000 Christian Urban isarfied some of the high-level proofs
Mon, 29 Nov 2010 05:17:41 +0000 Christian Urban added abs_rename_res lemma
Mon, 29 Nov 2010 05:10:02 +0000 Christian Urban completed proofs in Foo2
Sun, 28 Nov 2010 16:37:34 +0000 Christian Urban completed the strong exhausts rules for Foo2 using general lemmas
Sat, 27 Nov 2010 23:00:16 +0000 Christian Urban tuned proof to reduce number of warnings
Sat, 27 Nov 2010 22:55:29 +0000 Christian Urban disabled the Foo examples, because of heavy work
Fri, 26 Nov 2010 22:43:26 +0000 Christian Urban slightly simplified the Foo2 tests and hint at a general lemma
Fri, 26 Nov 2010 19:03:23 +0000 Christian Urban completely different method fro deriving the exhaust lemma
Fri, 26 Nov 2010 10:53:55 +0000 Christian Urban merged
Thu, 25 Nov 2010 01:18:24 +0000 Christian Urban merged
Wed, 24 Nov 2010 02:36:21 +0000 Christian Urban added example from the F-ing paper by Rossberg, Russo and Dreyer
Wed, 24 Nov 2010 01:08:48 +0000 Christian Urban implemented concrete suggestion of 3rd reviewer
Fri, 26 Nov 2010 12:17:24 +0900 Cezary Kaliszyk missing freshness assumptions
Thu, 25 Nov 2010 15:06:45 +0900 Cezary Kaliszyk foo2 strong induction
Wed, 24 Nov 2010 17:44:50 +0900 Cezary Kaliszyk foo2 full exhausts
Wed, 24 Nov 2010 16:59:26 +0900 Cezary Kaliszyk Foo2 strong_exhaust for first variable.
Mon, 22 Nov 2010 16:16:25 +0900 Cezary Kaliszyk single rename in let2
Mon, 22 Nov 2010 16:14:47 +0900 Cezary Kaliszyk current isabelle
Sun, 21 Nov 2010 02:17:19 +0000 Christian Urban added example Foo2.thy
Mon, 15 Nov 2010 20:54:01 +0000 Christian Urban tuned example
Mon, 15 Nov 2010 09:52:29 +0000 Christian Urban proved that bn functions return a finite set
Mon, 15 Nov 2010 08:17:11 +0000 Christian Urban added a test for the various shallow binders
Mon, 15 Nov 2010 01:10:02 +0000 Christian Urban fixed bug in fv function where a shallow binder binds lists of names
Sun, 14 Nov 2010 16:34:47 +0000 Christian Urban merged Nominal-General directory into Nominal; renamed Abs.thy to Nominal2_Abs.thy
Sun, 14 Nov 2010 12:09:14 +0000 Christian Urban deleted special Nominal2_FSet theory
Sun, 14 Nov 2010 11:46:39 +0000 Christian Urban moved rest of the lemmas from Nominal2_FSet to the TypeScheme example
Sun, 14 Nov 2010 11:05:22 +0000 Christian Urban moved most material fron Nominal2_FSet into the Nominal_Base theory
Sun, 14 Nov 2010 10:02:30 +0000 Christian Urban tuned example
Sun, 14 Nov 2010 01:00:56 +0000 Christian Urban lifted permute_bn simp rules
Sat, 13 Nov 2010 22:23:26 +0000 Christian Urban lifted permute_bn constants
Sat, 13 Nov 2010 10:25:03 +0000 Christian Urban respectfulness for permute_bn functions
Fri, 12 Nov 2010 01:20:53 +0000 Christian Urban automated permute_bn functions (raw ones first)
Wed, 10 Nov 2010 13:46:21 +0000 Christian Urban adapted to changes by Florian on the quotient package and removed local fix for function package
Wed, 10 Nov 2010 13:40:46 +0000 Christian Urban expanded the paper by uncommenting the comments and adding the appendix
Sun, 07 Nov 2010 11:22:31 +0000 Christian Urban fixed locally the problem with the function package; all tests work again
Sat, 06 Nov 2010 06:18:41 +0000 Christian Urban added a test about subtyping; disabled two tests, because of problem with function package
Fri, 05 Nov 2010 15:21:10 +0000 Christian Urban small typo
Fri, 29 Oct 2010 15:37:24 +0100 Christian Urban squeezed qpaper to 6 pages
Fri, 29 Oct 2010 14:25:50 +0900 Cezary Kaliszyk Qpaper / Move examples to commented out appendix
Thu, 28 Oct 2010 15:16:43 +0900 Cezary Kaliszyk Unanonymize qpaper
Thu, 28 Oct 2010 14:12:30 +0900 Cezary Kaliszyk FSet changes for Qpaper
Thu, 28 Oct 2010 14:03:46 +0900 Cezary Kaliszyk Remove FSet and use the one from Isabelle
Tue, 19 Oct 2010 15:08:24 +0100 Christian Urban took out comment about map-types / adapted to recent changes
Tue, 19 Oct 2010 10:10:41 +0100 Christian Urban use definitions instead of functions
Mon, 18 Oct 2010 12:15:44 +0100 Christian Urban tuned
Mon, 18 Oct 2010 11:51:22 +0100 Christian Urban used functions instead of definitions
Mon, 18 Oct 2010 09:42:51 +0100 Christian Urban added missing style file
Mon, 18 Oct 2010 14:13:28 +0900 Cezary Kaliszyk Use the generalized compositional quotient theorem
Sun, 17 Oct 2010 21:40:23 +0100 Christian Urban fixed typo
Sun, 17 Oct 2010 15:53:37 +0100 Christian Urban all tests work again
Sun, 17 Oct 2010 15:28:05 +0100 Christian Urban some tuning
Sun, 17 Oct 2010 13:35:52 +0100 Christian Urban naming scheme is now *_fset (not f*_)
Fri, 15 Oct 2010 23:45:54 +0100 Christian Urban more cleaning
Fri, 15 Oct 2010 17:37:44 +0100 Christian Urban further tuning
Fri, 15 Oct 2010 16:01:03 +0100 Christian Urban renamed fminus_raw to diff_list
Fri, 15 Oct 2010 15:58:48 +0100 Christian Urban renamed fcard_raw to card_list
Fri, 15 Oct 2010 15:56:16 +0100 Christian Urban slight update
Fri, 15 Oct 2010 15:47:20 +0100 Christian Urban Further reorganisation and cleaning
Fri, 15 Oct 2010 14:11:23 +0100 Christian Urban further cleaning
Fri, 15 Oct 2010 13:28:39 +0100 Christian Urban typo
Fri, 15 Oct 2010 16:32:34 +0900 Cezary Kaliszyk FSet: stronger fact in Isabelle.
Fri, 15 Oct 2010 16:23:26 +0900 Cezary Kaliszyk FSet synchronizing
Fri, 15 Oct 2010 15:52:40 +0900 Cezary Kaliszyk Synchronizing FSet further.
Fri, 15 Oct 2010 15:24:19 +0900 Cezary Kaliszyk Partially merging changes from Isabelle
Thu, 14 Oct 2010 17:32:06 +0100 Christian Urban fixed the typo in the abstract and the problem with append (the type of map_k
Thu, 14 Oct 2010 15:58:34 +0100 Christian Urban changed format of the pearl paper
Thu, 14 Oct 2010 11:09:52 +0100 Christian Urban deleted some unused lemmas
Thu, 14 Oct 2010 04:14:22 +0100 Christian Urban major reorganisation of fset (renamed fset_to_set to fset, changed the definition of list_eq and fcard_raw)
Wed, 13 Oct 2010 22:55:58 +0100 Christian Urban more on the pearl paper
Tue, 12 Oct 2010 13:06:18 +0100 Christian Urban added a section about abstractions
Tue, 12 Oct 2010 10:07:48 +0100 Christian Urban tiny work on the pearl paper
Fri, 08 Oct 2010 23:53:51 +0100 Christian Urban tuned
Fri, 08 Oct 2010 23:49:18 +0100 Christian Urban added apendix to paper detailing one proof
Fri, 08 Oct 2010 15:37:11 +0100 Christian Urban minor
Fri, 08 Oct 2010 15:35:14 +0100 Christian Urban minor
Fri, 08 Oct 2010 13:41:54 +0100 Christian Urban down to 20 pages
Thu, 07 Oct 2010 14:23:32 +0900 Cezary Kaliszyk minor
Wed, 06 Oct 2010 21:32:44 +0100 Christian Urban down to 21 pages and changed strong induction section
Wed, 06 Oct 2010 08:13:09 +0100 Christian Urban tuned
Wed, 06 Oct 2010 08:09:40 +0100 Christian Urban down to 22 pages
Tue, 05 Oct 2010 21:48:31 +0100 Christian Urban down to 23 pages
Tue, 05 Oct 2010 08:43:49 +0100 Christian Urban down to 24 pages and a bit
Tue, 05 Oct 2010 07:30:37 +0100 Christian Urban llncs and more sqeezing
Mon, 04 Oct 2010 12:39:57 +0100 Christian Urban first part of sqeezing everything into 20 pages (at the moment we have 26)
Mon, 04 Oct 2010 07:25:37 +0100 Christian Urban changed to llncs
Fri, 01 Oct 2010 07:11:47 -0400 Christian Urban merged
Fri, 01 Oct 2010 07:09:59 -0400 Christian Urban minor experiments
Thu, 30 Sep 2010 07:43:46 -0400 Christian Urban merged
Wed, 29 Sep 2010 16:49:13 -0400 Christian Urban simplified exhaust proofs
Fri, 01 Oct 2010 15:44:50 +0900 Cezary Kaliszyk Made the paper to compile with the renamings.
Wed, 29 Sep 2010 09:51:57 -0400 Christian Urban merged
Wed, 29 Sep 2010 09:47:26 -0400 Christian Urban worked example Foo1 with induct_schema
Wed, 29 Sep 2010 07:39:06 -0400 Christian Urban merged
Wed, 29 Sep 2010 06:45:01 -0400 Christian Urban use also induct_schema for the Let-example (permute_bn is used)
Wed, 29 Sep 2010 04:42:37 -0400 Christian Urban test with induct_schema for simpler strong_ind proofs
Wed, 29 Sep 2010 16:36:31 +0900 Cezary Kaliszyk substitution definition with 'next_name'.
Tue, 28 Sep 2010 08:21:47 -0400 Christian Urban merged
Tue, 28 Sep 2010 05:56:11 -0400 Christian Urban added Foo1 to explore a contrived example
Mon, 27 Sep 2010 12:19:17 -0400 Christian Urban added postprocessed fresh-lemmas for constructors
Mon, 27 Sep 2010 09:51:15 -0400 Christian Urban post-processed eq_iff and supp threormes according to the fv-supp equality
Mon, 27 Sep 2010 04:56:49 -0400 Christian Urban more consistent naming in Abs.thy
Mon, 27 Sep 2010 04:56:28 -0400 Christian Urban some experiments
Mon, 27 Sep 2010 04:10:36 -0400 Christian Urban added simp rules for prod_fv and prod_alpha
Sun, 26 Sep 2010 17:57:30 -0400 Christian Urban a few more words about Ott
Sat, 25 Sep 2010 08:38:04 -0400 Christian Urban lifted size_thms and exported them as <name>.size
Sat, 25 Sep 2010 08:28:45 -0400 Christian Urban cleaned up two examples
Sat, 25 Sep 2010 02:53:39 +0200 Christian Urban added example about datatypes
Thu, 23 Sep 2010 05:28:40 +0200 Christian Urban updated to Isabelle 22 Sept
Wed, 22 Sep 2010 23:17:25 +0200 Christian Urban removed dead code
Wed, 22 Sep 2010 18:13:26 +0200 Christian Urban fixed
Wed, 22 Sep 2010 14:19:48 +0800 Christian Urban made supp proofs more robust by not using the standard induction; renamed some example files
Mon, 20 Sep 2010 21:52:45 +0800 Christian Urban introduced a general procedure for structural inductions; simplified reflexivity proof
Sat, 18 Sep 2010 06:09:43 +0800 Christian Urban updated to Isabelle Sept 16
Sat, 18 Sep 2010 05:13:42 +0800 Christian Urban updated to Isabelle Sept 13
Sun, 12 Sep 2010 22:46:40 +0800 Christian Urban tuned code
Sat, 11 Sep 2010 05:56:49 +0800 Christian Urban tuned (to conform with indentation policy of Markus)
Fri, 10 Sep 2010 09:17:40 +0800 Christian Urban supp-proofs work except for CoreHaskell and Modules (induct is probably not finding the correct instance)
Sun, 05 Sep 2010 07:00:19 +0800 Christian Urban generated inducts rule by Project_Rule.projections
Sun, 05 Sep 2010 06:42:53 +0800 Christian Urban added the definition supp_rel (support w.r.t. a relation)
Sat, 04 Sep 2010 14:26:09 +0800 Christian Urban merged
Sat, 04 Sep 2010 07:39:38 +0800 Christian Urban got rid of Nominal2_Supp (is now in Nomina2_Base)
Sat, 04 Sep 2010 07:28:35 +0800 Christian Urban moved everything out of Nominal_Supp
Sat, 04 Sep 2010 06:48:14 +0800 Christian Urban renamed alpha_gen -> alpha_set and Abs -> Abs_set etc
(0) -1000 -384 +384 tip