Nominal/Ex/Lambda.thy
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 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
Sun, 05 Jun 2011 21:14:23 +0100 Christian Urban added an option for an invariant (at the moment only a stub)
Sat, 04 Jun 2011 09:07:50 +0900 Cezary Kaliszyk Finish and test the locale approach
Fri, 03 Jun 2011 12:46:23 +0100 Christian Urban recursion combinator inside a locale
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
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 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:17:22 +0100 Christian Urban functions involving if and case do not throw exceptions anymore; but eqvt_at assumption has now a precondition
Wed, 25 May 2011 21:38:50 +0200 Christian Urban added eq_iff and distinct lemmas of nominal datatypes to the simplifier
Sat, 14 May 2011 10:16:16 +0100 Christian Urban added a problem with inductive_cases (reported by Randy)
Tue, 03 May 2011 15:39:30 +0100 Christian Urban added two mutual recursive inductive definitions
Tue, 03 May 2011 13:09:08 +0100 Christian Urban proved that lfp is equivariant (that simplifies equivariance proofs of inductively defined predicates)
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:41:52 +0100 Christian Urban introduced framework for finetuning eqvt-rules; this solves problem with permute_pure called in nominal_inductive
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.
Tue, 01 Feb 2011 09:07:55 +0900 Cezary Kaliszyk Only one of the subgoals is needed
Tue, 25 Jan 2011 18:58:26 +0100 Christian Urban made eqvt-proof explicit in the function definitions
Wed, 19 Jan 2011 19:41:50 +0100 Christian Urban added obtain_fresh lemma; tuned Lambda.thy
Wed, 19 Jan 2011 18:56:28 +0100 Christian Urban ported some of the old proofs to serve as testcases
Wed, 19 Jan 2011 07:06:47 +0100 Christian Urban defined height as a function that returns an integer
Tue, 18 Jan 2011 19:27:30 +0100 Christian Urban defined properly substitution
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
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 12:37:37 +0000 Christian Urban removed old testing code from Lambda.thy
Sun, 09 Jan 2011 04:28:24 +0000 Christian Urban solved subgoals for depth and subst function
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 14:02:10 +0000 Christian Urban tuned
Fri, 31 Dec 2010 15:37:04 +0000 Christian Urban changed res keyword to set+ for restrictions; comment by a referee
Tue, 28 Dec 2010 19:51:25 +0000 Christian Urban automated all strong induction lemmas
Wed, 22 Dec 2010 09:13:25 +0000 Christian Urban properly exported strong exhaust theorem; cleaned up some examples
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, 29 Sep 2010 16:49:13 -0400 Christian Urban simplified exhaust proofs
Wed, 29 Sep 2010 04:42:37 -0400 Christian Urban test with induct_schema for simpler strong_ind proofs
Sun, 29 Aug 2010 13:36:03 +0800 Christian Urban renamed NewParser to Nominal2
Fri, 27 Aug 2010 13:57:00 +0800 Christian Urban make copies of the "old" files
Fri, 27 Aug 2010 03:37:17 +0800 Christian Urban "isabelle make test" makes all major examples....they work up to supp theorems (excluding)
Thu, 26 Aug 2010 02:08:00 +0800 Christian Urban cleaned up (almost completely) the examples
Wed, 25 Aug 2010 22:55:42 +0800 Christian Urban automatic lifting
Wed, 25 Aug 2010 11:58:37 +0800 Christian Urban now every lemma lifts (even with type variables)
Wed, 25 Aug 2010 09:02:06 +0800 Christian Urban can now deal with type variables in nominal datatype definitions
Sat, 21 Aug 2010 17:55:42 +0800 Christian Urban nominal_datatypes with type variables do not work
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
Mon, 07 Jun 2010 11:43:01 +0200 Christian Urban work on transitivity proof
Fri, 21 May 2010 17:17:51 +0200 Cezary Kaliszyk Match_Lam defined on Quotient Level.
Fri, 21 May 2010 11:55:22 +0200 Cezary Kaliszyk More on Function-defined subst.
Fri, 21 May 2010 10:47:45 +0200 Cezary Kaliszyk merge
Fri, 21 May 2010 10:43:14 +0200 Cezary Kaliszyk Renamings.
Fri, 21 May 2010 10:47:07 +0200 Cezary Kaliszyk merge (non-trival)
Fri, 21 May 2010 10:45:29 +0200 Cezary Kaliszyk Previously uncommited direct subst definition changes.
Fri, 21 May 2010 10:44:07 +0200 Cezary Kaliszyk Function experiments
Wed, 19 May 2010 12:29:08 +0200 Cezary Kaliszyk more subst experiments
Wed, 19 May 2010 11:29:42 +0200 Cezary Kaliszyk More subst experminets
Tue, 18 May 2010 17:56:41 +0200 Cezary Kaliszyk more on subst
Tue, 18 May 2010 17:17:54 +0200 Cezary Kaliszyk Single variable substitution
Tue, 18 May 2010 17:06:21 +0200 Cezary Kaliszyk subst fix
Tue, 18 May 2010 15:58:52 +0200 Cezary Kaliszyk subst experiments
Wed, 12 May 2010 16:59:53 +0100 Christian Urban fixed the examples for the new eqvt-procedure....temporarily disabled Manual/Term4.thy
Tue, 11 May 2010 18:20:25 +0200 Cezary Kaliszyk Include raw permutation definitions in eqvt
Tue, 11 May 2010 17:16:57 +0200 Cezary Kaliszyk Declare alpha_gen_eqvt as eqvt and change the proofs that used 'eqvts[symmetric]'
Sun, 09 May 2010 12:26:10 +0100 Christian Urban cleaned up a bit the examples; added equivariance to all examples
Tue, 04 May 2010 11:22:22 +0200 Cezary Kaliszyk Move 2 more to NewParser
Mon, 26 Apr 2010 20:17:41 +0200 Christian Urban some changes to the paper
Mon, 26 Apr 2010 08:19:11 +0200 Christian Urban eliminated command so that all compiles
Mon, 26 Apr 2010 08:08:20 +0200 Christian Urban changed theorem_i to theorem....requires new Isabelle
Sun, 25 Apr 2010 09:13:16 +0200 Christian Urban tuned and cleaned
Fri, 16 Apr 2010 16:29:11 +0200 Christian Urban automatic proofs for equivariance of alphas
Fri, 16 Apr 2010 11:09:32 +0200 Cezary Kaliszyk Finished proof in Lambda.thy
Fri, 16 Apr 2010 10:46:50 +0200 Christian Urban attempt to manual prove eqvt for alpha
Fri, 16 Apr 2010 10:18:16 +0200 Christian Urban some tuning of eqvt-infrastructure
Wed, 14 Apr 2010 22:23:52 +0200 Christian Urban deleted offending [eqvt]-attribute in Abs; Lambda works again, but there is now a problem in CoreHaskell
Wed, 14 Apr 2010 16:05:58 +0200 Christian Urban tuned and removed dead code
Wed, 14 Apr 2010 14:41:54 +0200 Christian Urban added a library for basic nominal functions; separated nominal_eqvt file
Wed, 14 Apr 2010 13:21:11 +0200 Christian Urban first working version of the automatic equivariance procedure
Wed, 14 Apr 2010 10:29:34 +0200 Christian Urban preliminary tests
Tue, 13 Apr 2010 07:40:54 +0200 Christian Urban made everything to compile
Tue, 13 Apr 2010 00:53:32 +0200 Christian Urban some small tunings (incompleted work in Lambda.thy)
Mon, 12 Apr 2010 17:44:26 +0200 Christian Urban early ott paper
Mon, 12 Apr 2010 13:34:54 +0200 Christian Urban implemented in thmdecls the case where eqvt-lemmas are of the form _ ==> _
Sun, 11 Apr 2010 22:48:49 +0200 Christian Urban fixed bug in thmdecls with destructing Trueprop; some initial infrastructure for eqvt-theorems of the form _ ==> _
Sun, 11 Apr 2010 18:11:13 +0200 Christian Urban a few tests
Fri, 09 Apr 2010 21:51:01 +0200 Christian Urban changed the eqvt-tac to move only outermost permutations inside; added tracing infrastructure for the eqvt-tac
Fri, 09 Apr 2010 11:08:05 +0200 Christian Urban renamed ExLam to Lambda and completed the proof of the strong ind principle; tuned paper
less more (0) tip