| Thu, 16 Jun 2011 20:56:30 +0900 | Cezary Kaliszyk | Added the CPS translation experiments. CPS1 comes with all the proofs, CPS2,3 just have the function and need eqvt_rhs to finish the obligations. | changeset | files | 
| Thu, 16 Jun 2011 12:12:25 +0100 | Christian Urban | added a test that every function must be of pt-sort | changeset | files | 
| Thu, 16 Jun 2011 11:03:01 +0100 | Christian Urban | all tests work again | changeset | files | 
| Wed, 15 Jun 2011 22:36:59 +0100 | Christian Urban | added size-lemmas to simplifier; as a result termination can be proved by the standard lexicographic_order method | changeset | files | 
| Wed, 15 Jun 2011 12:52:48 +0100 | Christian Urban | added an abstract | changeset | files | 
| Wed, 15 Jun 2011 12:32:40 +0100 | Christian Urban | added a stub for function paper; "isabelle make fnpaper" | changeset | files | 
| Wed, 15 Jun 2011 11:06:48 +0900 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 15 Jun 2011 11:06:31 +0900 | Cezary Kaliszyk | one TODO and one Problem? | changeset | files | 
| Wed, 15 Jun 2011 09:51:26 +0900 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 15 Jun 2011 09:50:53 +0900 | Cezary Kaliszyk | Some TODOs | changeset | files | 
| Wed, 15 Jun 2011 09:31:59 +0900 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 15 Jun 2011 09:25:36 +0900 | Cezary Kaliszyk | TypeSchemes work with 'default'. | changeset | files | 
| Tue, 14 Jun 2011 19:11:44 +0100 | Christian Urban | tuned some proofs | changeset | files | 
| 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 | changeset | files | 
| Tue, 14 Jun 2011 11:43:06 +0100 | Christian Urban | tuned | changeset | files | 
| Fri, 10 Jun 2011 15:52:17 +0900 | Cezary Kaliszyk | Move working examples before non-working ones | changeset | files | 
| Fri, 10 Jun 2011 15:45:49 +0900 | Cezary Kaliszyk | Optimized proofs and removed some garbage. | changeset | files | 
| Fri, 10 Jun 2011 15:31:14 +0900 | Cezary Kaliszyk | merge | changeset | files | 
| Fri, 10 Jun 2011 15:30:09 +0900 | Cezary Kaliszyk | Slightly modify fcb for list1 and put in common place. | changeset | files | 
| Fri, 10 Jun 2011 09:00:24 +0900 | Cezary Kaliszyk | Experiments with Let | changeset | files | 
| Thu, 09 Jun 2011 15:34:51 +0900 | Cezary Kaliszyk | Eval can be defined with additional freshness | changeset | files | 
| Thu, 09 Jun 2011 15:03:58 +0900 | Cezary Kaliszyk | Minor simplification | changeset | files | 
| 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'. | changeset | files | 
| Thu, 09 Jun 2011 09:44:51 +0900 | Cezary Kaliszyk | More experiments with 'default' | changeset | files | 
| Wed, 08 Jun 2011 21:44:03 +0900 | Cezary Kaliszyk | Finished the proof with the invariant | changeset | files | 
| Wed, 08 Jun 2011 21:32:35 +0900 | Cezary Kaliszyk | Issue with 'default' | changeset | files | 
| Wed, 08 Jun 2011 12:30:56 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 08 Jun 2011 12:30:46 +0100 | Christian Urban | merged | changeset | files | 
| 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 | changeset | files | 
| Wed, 08 Jun 2011 17:52:06 +0900 | Cezary Kaliszyk | Simpler proof of TypeSchemes/substs | changeset | files | 
| Wed, 08 Jun 2011 17:25:54 +0900 | Cezary Kaliszyk | Simplify fcb_res | changeset | files | 
| Wed, 08 Jun 2011 09:56:39 +0900 | Cezary Kaliszyk | FCB for res binding and simplified proof of subst for type schemes | changeset | files | 
| Wed, 08 Jun 2011 07:06:20 +0900 | Cezary Kaliszyk | Simplify ln-trans proof | changeset | files | 
| Wed, 08 Jun 2011 07:02:52 +0900 | Cezary Kaliszyk | cbvs can be easily defined without an invariant | changeset | files | 
| Tue, 07 Jun 2011 20:58:00 +0100 | Christian Urban | defined the "count-bound-variables-occurences" function which has an accumulator like trans | changeset | files | 
| Tue, 07 Jun 2011 17:45:38 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 07 Jun 2011 23:42:12 +0900 | Cezary Kaliszyk | remove garbage (proofs that assumes the invariant outside function) | changeset | files | 
| Tue, 07 Jun 2011 23:38:39 +0900 | Cezary Kaliszyk | Proof of trans with invariant | changeset | files | 
| Tue, 07 Jun 2011 23:22:58 +0900 | Cezary Kaliszyk | Testing invariant in Lambda_F_T | changeset | files | 
| 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 | changeset | files | 
| 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 | changeset | files | 
| Mon, 06 Jun 2011 13:11:04 +0100 | Christian Urban | slightly stronger property in fundef_ex_prop | changeset | files | 
| Sun, 05 Jun 2011 21:14:23 +0100 | Christian Urban | added an option for an invariant (at the moment only a stub) | changeset | files | 
| Sun, 05 Jun 2011 16:58:18 +0100 | Christian Urban | added a more general lemma fro fundef_ex1 | changeset | files | 
| Sat, 04 Jun 2011 14:50:57 +0900 | Cezary Kaliszyk | Trying the induction on the graph | changeset | files | 
| Sat, 04 Jun 2011 09:07:50 +0900 | Cezary Kaliszyk | Finish and test the locale approach | changeset | files | 
| Fri, 03 Jun 2011 22:31:44 +0900 | Cezary Kaliszyk | FiniteSupp precondition in the function is enough to get rid of completeness obligationss | changeset | files | 
| Fri, 03 Jun 2011 12:46:23 +0100 | Christian Urban | recursion combinator inside a locale | changeset | files | 
| Fri, 03 Jun 2011 18:33:11 +0900 | Cezary Kaliszyk | merge | changeset | files | 
| Fri, 03 Jun 2011 18:32:22 +0900 | Cezary Kaliszyk | F for lambda used to define translation to locally nameless | changeset | files | 
| Thu, 02 Jun 2011 16:15:18 +0100 | Christian Urban | typo | changeset | files | 
| Thu, 02 Jun 2011 15:35:33 +0100 | Christian Urban | removed dead code | changeset | files | 
| Thu, 02 Jun 2011 22:24:33 +0900 | Cezary Kaliszyk | finished the missing obligations | changeset | files | 
| Thu, 02 Jun 2011 12:14:03 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 02 Jun 2011 12:09:31 +0100 | Christian Urban | a test with a recursion combinator defined on top of nominal_primrec | changeset | files | 
| Thu, 02 Jun 2011 16:41:09 +0900 | Cezary Kaliszyk | Use FCB to simplify proof | changeset | files | 
| Thu, 02 Jun 2011 10:11:50 +0900 | Cezary Kaliszyk | merge | changeset | files | 
| Thu, 02 Jun 2011 10:09:23 +0900 | Cezary Kaliszyk | Remove SMT | changeset | files | 
| Wed, 01 Jun 2011 22:55:14 +0100 | Christian Urban | hopefully final fix for ho-functions | changeset | files | 
| Wed, 01 Jun 2011 21:03:30 +0100 | Christian Urban | first test to fix the problem with free variables | changeset | files | 
| Wed, 01 Jun 2011 16:13:42 +0900 | Cezary Kaliszyk | proved subst for All constructor in type schemes. | changeset | files | 
| Wed, 01 Jun 2011 13:41:30 +0900 | Cezary Kaliszyk | DB translation using index; easier to reason about. | changeset | files | 
| Wed, 01 Jun 2011 13:35:37 +0900 | Cezary Kaliszyk | Problem: free variables in the goal | changeset | files | 
| Wed, 01 Jun 2011 11:01:39 +0900 | Cezary Kaliszyk | fixed previous commit | changeset | files | 
| Wed, 01 Jun 2011 10:59:07 +0900 | Cezary Kaliszyk | equivariance of db_trans | changeset | files | 
| Tue, 31 May 2011 12:22:28 +0100 | Christian Urban | fixed the problem with cps-like functions | changeset | files | 
| Tue, 31 May 2011 14:12:31 +0900 | Cezary Kaliszyk | DeBruijn translation in a simplifier friendly way | changeset | files | 
| Tue, 31 May 2011 13:25:35 +0900 | Cezary Kaliszyk | map_term can be defined when equivariance is assumed | changeset | files | 
| Tue, 31 May 2011 13:21:00 +0900 | Cezary Kaliszyk | map_term is not a function the way it is defined | changeset | files | 
| 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. | changeset | files | 
| Tue, 31 May 2011 12:54:21 +0900 | Cezary Kaliszyk | Simple eqvt proofs with perm_simps for clarity | changeset | files | 
| Tue, 31 May 2011 00:36:16 +0100 | Christian Urban | tuned last commit | changeset | files | 
| 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 | changeset | files | 
| Thu, 26 May 2011 06:36:29 +0200 | Christian Urban | updated to new Isabelle | changeset | files | 
| Wed, 25 May 2011 21:38:50 +0200 | Christian Urban | added eq_iff and distinct lemmas of nominal datatypes to the simplifier | changeset | files | 
| Tue, 24 May 2011 19:39:38 +0200 | Christian Urban | more on slides | changeset | files | 
| Sun, 22 May 2011 10:20:18 +0200 | Christian Urban | added slides for copenhagen | changeset | files | 
| Sat, 14 May 2011 10:16:16 +0100 | Christian Urban | added a problem with inductive_cases (reported by Randy) | changeset | files | 
| Fri, 13 May 2011 14:50:17 +0100 | Christian Urban | misc | changeset | files | 
| Tue, 10 May 2011 17:10:22 +0100 | Christian Urban | made the subtyping work again | changeset | files | 
| Tue, 10 May 2011 07:47:06 +0100 | Christian Urban | updated to new Isabelle (> 9 May) | changeset | files | 
| Mon, 09 May 2011 04:49:58 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 03 May 2011 15:39:30 +0100 | Christian Urban | added two mutual recursive inductive definitions | changeset | files | 
| Tue, 03 May 2011 13:25:02 +0100 | Christian Urban | deleted two functions from the API | changeset | files | 
| Tue, 03 May 2011 13:09:08 +0100 | Christian Urban | proved that lfp is equivariant (that simplifies equivariance proofs of inductively defined predicates) | changeset | files | 
| Mon, 09 May 2011 04:46:43 +0100 | Christian Urban | more on pearl-paper | changeset | files | 
| Wed, 04 May 2011 15:27:04 +0800 | Christian Urban | more on pearl-paper | changeset | files | 
| Mon, 02 May 2011 13:01:02 +0800 | Christian Urban | updated Quotient paper so that it compiles again | changeset | files | 
| Thu, 28 Apr 2011 11:51:01 +0800 | Christian Urban | merged | changeset | files | 
| Thu, 28 Apr 2011 11:44:36 +0800 | Christian Urban | added slides for beijing | changeset | files | 
| Fri, 22 Apr 2011 00:18:25 +0800 | Christian Urban | more to the pearl paper | changeset | files | 
| Tue, 19 Apr 2011 13:03:08 +0100 | Christian Urban | updated to snapshot Isabelle 19 April | changeset | files | 
| Mon, 18 Apr 2011 15:57:45 +0100 | Christian Urban | merged | changeset | files | 
| Mon, 18 Apr 2011 15:56:07 +0100 | Christian Urban | added permute_pure back into the nominal_inductive procedure; updated to Isabelle 17 April | changeset | files | 
| 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. | changeset | files | 
| Wed, 13 Apr 2011 13:44:25 +0100 | Christian Urban | merged | changeset | files | 
| 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 | changeset | files | 
| Tue, 12 Apr 2011 15:46:35 +0800 | Christian Urban | shanghai slides | changeset | files | 
| Mon, 11 Apr 2011 02:25:25 +0100 | Christian Urban | pictures for slides | changeset | files | 
| Mon, 11 Apr 2011 02:04:11 +0100 | Christian Urban | Shanghai slides | changeset | files | 
| Sun, 10 Apr 2011 14:13:55 +0800 | Christian Urban | more paper | changeset | files | 
| Sun, 10 Apr 2011 07:41:52 +0800 | Christian Urban | eqvt of supp and fresh is proved using equivariance infrastructure | changeset | files | 
| Sun, 10 Apr 2011 04:07:15 +0800 | Christian Urban | more paper | changeset | files | 
| Sat, 09 Apr 2011 13:44:49 +0800 | Christian Urban | more on the paper | changeset | files | 
| Sat, 09 Apr 2011 00:29:40 +0100 | Christian Urban | tuned paper | changeset | files | 
| Sat, 09 Apr 2011 00:28:53 +0100 | Christian Urban | tuned paper | changeset | files | 
| Sat, 09 Apr 2011 02:10:49 +0800 | Christian Urban | typo | changeset | files | 
| Fri, 08 Apr 2011 14:23:28 +0800 | Christian Urban | more on paper | changeset | files | 
| Fri, 08 Apr 2011 03:47:50 +0800 | Christian Urban | eqvt_lambda without eta-expansion | changeset | files | 
| Wed, 06 Apr 2011 13:47:08 +0100 | Christian Urban | changed default preprocessor that does not catch variables only occuring on the right | changeset | files | 
| Thu, 31 Mar 2011 15:25:35 +0200 | Christian Urban | final version of slides | changeset | files | 
| Wed, 30 Mar 2011 22:27:26 +0200 | Christian Urban | more on the slides | changeset | files | 
| Wed, 30 Mar 2011 08:11:36 +0200 | Christian Urban | tuned IsaMakefile | changeset | files | 
| Tue, 29 Mar 2011 23:52:14 +0200 | Christian Urban | rearranged directories and updated to new Isabelle | changeset | files | 
| Wed, 16 Mar 2011 21:14:43 +0100 | Christian Urban | precise path to LaTeXsugar | changeset | files | 
| Wed, 16 Mar 2011 21:07:50 +0100 | Christian Urban | a lit bit more on the pearl-jv paper | changeset | files | 
| Wed, 16 Mar 2011 20:42:14 +0100 | Christian Urban | ported changes from function package....needs Isabelle 16 March or above | changeset | files | 
| Tue, 15 Mar 2011 00:40:39 +0100 | Christian Urban | more on the pearl paper | changeset | files | 
| Mon, 14 Mar 2011 16:35:59 +0100 | Christian Urban | equivariance for All and Ex can be proved in terms of their definition | changeset | files | 
| Fri, 11 Mar 2011 08:51:39 +0000 | Christian Urban | more on the paper | changeset | files | 
| Tue, 08 Mar 2011 09:07:49 +0000 | Christian Urban | merged | changeset | files | 
| Tue, 08 Mar 2011 09:07:27 +0000 | Christian Urban | more on the pearl paper | changeset | files | 
| Wed, 02 Mar 2011 16:07:56 +0900 | Cezary Kaliszyk | distinct names at toplevel | changeset | files | 
| Wed, 02 Mar 2011 12:49:01 +0900 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 02 Mar 2011 12:48:00 +0900 | Cezary Kaliszyk | Pairing function | changeset | files | 
| Wed, 02 Mar 2011 00:06:28 +0000 | Christian Urban | updated pearl papers | changeset | files | 
| Tue, 01 Mar 2011 00:14:02 +0000 | Christian Urban | a bit more tuning | changeset | files | 
| Mon, 28 Feb 2011 16:47:13 +0000 | Christian Urban | included old test cases for perm_simp into ROOT.ML file | changeset | files | 
| Mon, 28 Feb 2011 15:21:10 +0000 | Christian Urban | split the library into a basics file; merged Nominal_Eqvt into Nominal_Base | changeset | files | 
| Fri, 25 Feb 2011 21:23:30 +0000 | Christian Urban | some slight polishing | changeset | files | 
| Thu, 24 Feb 2011 18:50:02 +0000 | Christian Urban | merged | changeset | files | 
| Thu, 24 Feb 2011 16:26:11 +0000 | Christian Urban | added a lemma about fresh_star and Abs | changeset | files | 
| 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. | changeset | files | 
| Sat, 19 Feb 2011 09:31:22 +0900 | Cezary Kaliszyk | typeschemes/subst | changeset | files | 
| Thu, 17 Feb 2011 17:02:25 +0900 | Cezary Kaliszyk | further experiments with typeschemes subst | changeset | files | 
| Thu, 17 Feb 2011 12:01:08 +0900 | Cezary Kaliszyk | Finished the proof of a function that invents fresh variable names. | changeset | files | 
| Wed, 16 Feb 2011 14:44:33 +0000 | Christian Urban | added eqvt for length | changeset | files | 
| Wed, 16 Feb 2011 14:03:26 +0000 | Christian Urban | added eqvt lemmas for filter and distinct | changeset | files | 
| Mon, 07 Feb 2011 16:00:24 +0000 | Christian Urban | added eqvt for cartesian products | changeset | files | 
| Mon, 07 Feb 2011 15:59:37 +0000 | Christian Urban | cleaned up the experiments so that the tests go through | changeset | files | 
| Sat, 05 Feb 2011 07:39:00 +0900 | Cezary Kaliszyk | merge | changeset | files | 
| Sat, 05 Feb 2011 07:38:22 +0900 | Cezary Kaliszyk | Experiments defining a function on Let | changeset | files | 
| Fri, 04 Feb 2011 04:45:04 +0000 | Christian Urban | updated TODO | changeset | files | 
| Fri, 04 Feb 2011 03:52:38 +0000 | Christian Urban | Lambda.thy which works with Nominal_Isabelle2011 | changeset | files | 
| Thu, 03 Feb 2011 02:57:04 +0000 | Christian Urban | merged | changeset | files | 
| Thu, 03 Feb 2011 02:51:57 +0000 | Christian Urban | removed diagnostic code | changeset | files | 
| Tue, 01 Feb 2011 09:07:55 +0900 | Cezary Kaliszyk | Only one of the subgoals is needed | changeset | files | 
| Tue, 01 Feb 2011 08:57:50 +0900 | Cezary Kaliszyk | Experiments with substitution on set+ | changeset | files | 
| 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. | changeset | files | 
| Sun, 30 Jan 2011 12:09:23 +0900 | Cezary Kaliszyk | alpha_res implies alpha_set :) | changeset | files | 
| 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'. | changeset | files | 
| Sat, 29 Jan 2011 14:26:47 +0900 | Cezary Kaliszyk | Experiments with functions | changeset | files | 
| Thu, 27 Jan 2011 20:19:13 +0100 | Christian Urban | some experiments | changeset | files | 
| Thu, 27 Jan 2011 04:24:17 +0100 | Christian Urban | the proofs with eqvt_at | changeset | files | 
| Tue, 25 Jan 2011 18:58:26 +0100 | Christian Urban | made eqvt-proof explicit in the function definitions | changeset | files | 
| Tue, 25 Jan 2011 02:51:44 +0900 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 25 Jan 2011 02:46:05 +0900 | Cezary Kaliszyk | minor | changeset | files | 
| Tue, 25 Jan 2011 02:42:15 +0900 | Cezary Kaliszyk | Down as infixr | changeset | files | 
| Sat, 22 Jan 2011 23:24:20 -0600 | Christian Urban | added some slides | changeset | files | 
| Sun, 23 Jan 2011 03:29:22 +0100 | Christian Urban | added Tutorial6 | changeset | files | 
| Sat, 22 Jan 2011 18:59:48 -0600 | Christian Urban | cleaning up | changeset | files | 
| Sat, 22 Jan 2011 16:37:00 -0600 | Christian Urban | merged | changeset | files | 
| Sat, 22 Jan 2011 16:36:21 -0600 | Christian Urban | cleaned up Tutorial 3 with solutions | changeset | files | 
| Sun, 23 Jan 2011 07:32:28 +0900 | Cezary Kaliszyk | Missing val.simps | changeset | files | 
| Sun, 23 Jan 2011 07:17:35 +0900 | Cezary Kaliszyk | merge | changeset | files | 
| Sun, 23 Jan 2011 07:15:59 +0900 | Cezary Kaliszyk | Tutorial 4s | changeset | files | 
| Sat, 22 Jan 2011 16:04:40 -0600 | Christian Urban | cleaned up and solution section | changeset | files | 
| Sat, 22 Jan 2011 15:07:36 -0600 | Christian Urban | cleaned up tutorial1...added solution file | changeset | files | 
| Sat, 22 Jan 2011 12:46:01 -0600 | Christian Urban | better version of Tutorial 1 | changeset | files | 
| Fri, 21 Jan 2011 22:58:03 +0100 | Christian Urban | better flow of proofs and definitions and proof | changeset | files | 
| Fri, 21 Jan 2011 22:23:44 +0100 | Christian Urban | separated type preservation and progress into a separate file | changeset | files | 
| Fri, 21 Jan 2011 22:02:34 +0100 | Christian Urban | substitution lemma in separate file | changeset | files | 
| Fri, 21 Jan 2011 21:58:51 +0100 | Christian Urban | added unbind example | changeset | files | 
| Fri, 21 Jan 2011 00:55:28 +0100 | Christian Urban | a bit tuning | changeset | files | 
| Thu, 20 Jan 2011 23:19:30 +0100 | Christian Urban | first split of tutorrial theory | changeset | files | 
| Wed, 19 Jan 2011 23:58:12 +0100 | Christian Urban | added a very rough version of the tutorial; all seems to work | changeset | files | 
| Wed, 19 Jan 2011 19:41:50 +0100 | Christian Urban | added obtain_fresh lemma; tuned Lambda.thy | changeset | files | 
| Wed, 19 Jan 2011 19:06:52 +0100 | Christian Urban | base file for the tutorial (contains definitions for heigt, subst and beta-reduction) | changeset | files | 
| Wed, 19 Jan 2011 18:56:28 +0100 | Christian Urban | ported some of the old proofs to serve as testcases | changeset | files | 
| Wed, 19 Jan 2011 18:07:29 +0100 | Christian Urban | added eqvt and supp lemma for removeAll (function from List.thy) | changeset | files | 
| Wed, 19 Jan 2011 17:54:50 +0100 | Christian Urban | theory name as it should be | changeset | files | 
| Wed, 19 Jan 2011 17:54:06 +0100 | Christian Urban | removed diagnostic code | changeset | files | 
| Wed, 19 Jan 2011 17:11:10 +0100 | Christian Urban | added Minimal file to test things | changeset | files | 
| Wed, 19 Jan 2011 07:06:47 +0100 | Christian Urban | defined height as a function that returns an integer | changeset | files | 
| Tue, 18 Jan 2011 21:28:07 +0100 | Christian Urban | deleted diagnostic code | changeset | files | 
| Tue, 18 Jan 2011 21:26:58 +0100 | Christian Urban | some tryes about substitution over type-schemes | changeset | files | 
| Tue, 18 Jan 2011 19:27:30 +0100 | Christian Urban | defined properly substitution | changeset | files | 
| Tue, 18 Jan 2011 18:04:40 +0100 | Christian Urban | derived stronger Abs_eq_iff2 theorems | changeset | files | 
| Tue, 18 Jan 2011 17:30:47 +0100 | Christian Urban | made alpha_abs_set_stronger1 stronger | changeset | files | 
| Tue, 18 Jan 2011 17:19:50 +0100 | Christian Urban | removed finiteness assumption from set_rename_perm | changeset | files | 
| Tue, 18 Jan 2011 22:11:49 +0900 | Cezary Kaliszyk | alpha_abs_set_stronger1 | changeset | files | 
| Tue, 18 Jan 2011 21:12:25 +0900 | Cezary Kaliszyk | alpha_abs_let_stronger is not true in the same form | changeset | files | 
| 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 | changeset | files | 
| Tue, 18 Jan 2011 06:55:18 +0100 | Christian Urban | modified the renaming_perm lemmas | changeset | files | 
| 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) | changeset | files | 
| Mon, 17 Jan 2011 15:12:03 +0100 | Christian Urban | added a few examples of functions to Lambda.thy | changeset | files | 
| Mon, 17 Jan 2011 14:37:18 +0100 | Christian Urban | exported nominal function code to external file | changeset | files | 
| Mon, 17 Jan 2011 12:37:37 +0000 | Christian Urban | removed old testing code from Lambda.thy | changeset | files | 
| Mon, 17 Jan 2011 12:34:11 +0000 | Christian Urban | moved high level code from LamTest into the main libraries. | changeset | files | 
| 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 | changeset | files | 
| Sat, 15 Jan 2011 21:16:15 +0000 | Christian Urban | subst also works now | changeset | files | 
| 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 | changeset | files | 
| Fri, 14 Jan 2011 14:22:25 +0000 | Christian Urban | strengthened renaming lemmas | changeset | files | 
| Thu, 13 Jan 2011 12:12:47 +0000 | Christian Urban | added eqvt_lemmas for subset and psubset | changeset | files | 
| Mon, 10 Jan 2011 11:36:55 +0000 | Christian Urban | a few lemmas about freshness for at and at_base | changeset | files | 
| Mon, 10 Jan 2011 08:51:51 +0000 | Christian Urban | added a property about finite support in the presense of eqvt_at | changeset | files | 
| Sun, 09 Jan 2011 05:38:53 +0000 | Christian Urban | instantiated fundef_ex1_eqvt_at theorem with the indction hypothesis | changeset | files | 
| Sun, 09 Jan 2011 04:28:24 +0000 | Christian Urban | solved subgoals for depth and subst function | changeset | files | 
| Sun, 09 Jan 2011 01:17:44 +0000 | Christian Urban | added eqvt_at premises in function definition - however not proved at the moment | changeset | files | 
| Fri, 07 Jan 2011 05:40:31 +0000 | Christian Urban | added one further lemma about equivariance of THE_default | changeset | files | 
| Fri, 07 Jan 2011 05:06:25 +0000 | Christian Urban | equivariance of THE_default under the uniqueness assumption | changeset | files | 
| Fri, 07 Jan 2011 02:30:00 +0000 | Christian Urban | derived equivariance for the function graph and function relation | changeset | files | 
| 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 | changeset | files | 
| Thu, 06 Jan 2011 20:25:40 +0000 | Christian Urban | removed last traces of debugging code | changeset | files | 
| Thu, 06 Jan 2011 19:57:57 +0000 | Christian Urban | removed debugging code abd introduced a guarded tracing function | changeset | files | 
| Thu, 06 Jan 2011 14:53:38 +0000 | Christian Urban | moved Weakening up....it does not compile when put at the last position | changeset | files | 
| Thu, 06 Jan 2011 14:02:10 +0000 | Christian Urban | tuned | changeset | files | 
| Thu, 06 Jan 2011 13:31:44 +0000 | Christian Urban | added weakening to the test cases | changeset | files | 
| Thu, 06 Jan 2011 13:28:40 +0000 | Christian Urban | cleaned up weakening proof and added a version with finit sets | changeset | files | 
| Thu, 06 Jan 2011 13:28:19 +0000 | Christian Urban | same | changeset | files | 
| Thu, 06 Jan 2011 13:28:04 +0000 | Christian Urban | some further lemmas for fsets | changeset | files | 
| Thu, 06 Jan 2011 11:00:16 +0000 | Christian Urban | made sure the raw datatypes and raw functions do not get any mixfix syntax | changeset | files | 
| Wed, 05 Jan 2011 17:33:43 +0000 | Christian Urban | exported the code into a separate file | changeset | files | 
| Wed, 05 Jan 2011 16:51:27 +0000 | Christian Urban | strong rule inductions; as an example the weakening lemma works | changeset | files | 
| 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 | changeset | files | 
| Mon, 03 Jan 2011 16:21:12 +0000 | Christian Urban | file with most of the strong rule induction development | changeset | files | 
| Mon, 03 Jan 2011 16:19:27 +0000 | Christian Urban | simple cases for string rule inductions | changeset | files | 
| Fri, 31 Dec 2010 15:37:04 +0000 | Christian Urban | changed res keyword to set+ for restrictions; comment by a referee | changeset | files | 
| Fri, 31 Dec 2010 13:31:39 +0000 | Christian Urban | added proper case names for all induct and exhaust theorems | changeset | files | 
| Fri, 31 Dec 2010 12:12:59 +0000 | Christian Urban | added small example for strong inductions; functions still need a sorry | changeset | files | 
| Thu, 30 Dec 2010 10:00:09 +0000 | Christian Urban | removed local fix for bug in induction_schema; added setup method for strong inductions | changeset | files | 
| Tue, 28 Dec 2010 19:51:25 +0000 | Christian Urban | automated all strong induction lemmas | changeset | files | 
| 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 | changeset | files | 
| Sun, 26 Dec 2010 16:35:16 +0000 | Christian Urban | generated goals for strong induction theorems. | changeset | files | 
| Thu, 23 Dec 2010 01:05:05 +0000 | Christian Urban | test with strong inductions | changeset | files | 
| Thu, 23 Dec 2010 00:46:06 +0000 | Christian Urban | moved all strong_exhaust code to nominal_dt_quot; tuned examples | changeset | files | 
| Thu, 23 Dec 2010 00:22:41 +0000 | Christian Urban | moved generic functions into nominal_library | changeset | files | 
| Wed, 22 Dec 2010 23:12:51 +0000 | Christian Urban | slight tuning | changeset | files | 
| Wed, 22 Dec 2010 22:30:43 +0000 | Christian Urban | slight tuning | changeset | files | 
| Wed, 22 Dec 2010 21:13:44 +0000 | Christian Urban | tuned examples | changeset | files | 
| Wed, 22 Dec 2010 21:13:32 +0000 | Christian Urban | added fold_right which produces the correct term for left-infix operators | changeset | files | 
| Wed, 22 Dec 2010 12:47:09 +0000 | Christian Urban | updated to Isabelle 22 December | changeset | files | 
| Wed, 22 Dec 2010 12:17:49 +0000 | Christian Urban | a bit tuning | changeset | files | 
| Wed, 22 Dec 2010 10:32:01 +0000 | Christian Urban | corrected premises of strong exhausts theorems | changeset | files | 
| Wed, 22 Dec 2010 09:13:25 +0000 | Christian Urban | properly exported strong exhaust theorem; cleaned up some examples | changeset | files | 
| 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 | changeset | files | 
| Sun, 19 Dec 2010 07:50:37 +0000 | Christian Urban | one interesting case done | changeset | files | 
| Sun, 19 Dec 2010 07:43:32 +0000 | Christian Urban | a stronger statement for at_set_avoiding | changeset | files | 
| Fri, 17 Dec 2010 01:01:44 +0000 | Christian Urban | tuned | changeset | files | 
| Fri, 17 Dec 2010 00:39:27 +0000 | Christian Urban | tuned | changeset | files | 
| Thu, 16 Dec 2010 08:42:48 +0000 | Christian Urban | simple cases for strong inducts done; infrastructure for the difficult ones is there | changeset | files | 
| Thu, 16 Dec 2010 02:25:35 +0000 | Christian Urban | added theorem-rewriter conversion | changeset | files | 
| 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) | changeset | files | 
| Sun, 12 Dec 2010 22:09:11 +0000 | Christian Urban | created strong_exhausts terms | changeset | files | 
| 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 | changeset | files | 
| Fri, 10 Dec 2010 19:01:44 +0000 | Christian Urban | updated | changeset | files | 
| Thu, 09 Dec 2010 18:12:42 +0000 | Christian Urban | a bit more tuning of the paper | changeset | files | 
| Thu, 09 Dec 2010 17:10:08 +0000 | Christian Urban | brought the paper to 20 pages plus one page appendix | changeset | files | 
| Wed, 08 Dec 2010 17:07:08 +0000 | Christian Urban | first tests about exhaust | changeset | files | 
| Wed, 08 Dec 2010 13:16:25 +0000 | Christian Urban | moved some code into the nominal_library | changeset | files | 
| Wed, 08 Dec 2010 13:05:04 +0000 | Christian Urban | moved definition of raw bn-functions into nominal_dt_rawfuns | changeset | files | 
| Wed, 08 Dec 2010 12:37:25 +0000 | Christian Urban | kept the nested structure of constructors (belonging to one datatype) | changeset | files | 
| Tue, 07 Dec 2010 19:16:09 +0000 | Christian Urban | moved general theorems into the libraries | changeset | files | 
| Tue, 07 Dec 2010 14:27:39 +0000 | Christian Urban | automated permute_bn theorems | changeset | files | 
| Tue, 07 Dec 2010 14:27:21 +0000 | Christian Urban | updated to changes in Isabelle | changeset | files | 
| Mon, 06 Dec 2010 17:11:54 +0000 | Christian Urban | deleted nominal_dt_supp.ML | changeset | files | 
| Mon, 06 Dec 2010 17:11:34 +0000 | Christian Urban | moved code from nominal_dt_supp to nominal_dt_quot | changeset | files | 
| Mon, 06 Dec 2010 16:35:42 +0000 | Christian Urban | automated alpha_perm_bn theorems | changeset | files | 
| 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 | changeset | files | 
| Fri, 03 Dec 2010 13:51:07 +0000 | Christian Urban | updated to Isabelle 2nd December | changeset | files | 
| Mon, 29 Nov 2010 08:01:09 +0000 | Christian Urban | isarfied some of the high-level proofs | changeset | files | 
| Mon, 29 Nov 2010 05:17:41 +0000 | Christian Urban | added abs_rename_res lemma | changeset | files | 
| Mon, 29 Nov 2010 05:10:02 +0000 | Christian Urban | completed proofs in Foo2 | changeset | files | 
| Sun, 28 Nov 2010 16:37:34 +0000 | Christian Urban | completed the strong exhausts rules for Foo2 using general lemmas | changeset | files | 
| Sat, 27 Nov 2010 23:00:16 +0000 | Christian Urban | tuned proof to reduce number of warnings | changeset | files | 
| Sat, 27 Nov 2010 22:55:29 +0000 | Christian Urban | disabled the Foo examples, because of heavy work | changeset | files | 
| Fri, 26 Nov 2010 22:43:26 +0000 | Christian Urban | slightly simplified the Foo2 tests and hint at a general lemma | changeset | files | 
| Fri, 26 Nov 2010 19:03:23 +0000 | Christian Urban | completely different method fro deriving the exhaust lemma | changeset | files | 
| Fri, 26 Nov 2010 10:53:55 +0000 | Christian Urban | merged | changeset | files | 
| Thu, 25 Nov 2010 01:18:24 +0000 | Christian Urban | merged | changeset | files | 
| Wed, 24 Nov 2010 02:36:21 +0000 | Christian Urban | added example from the F-ing paper by Rossberg, Russo and Dreyer | changeset | files | 
| Wed, 24 Nov 2010 01:08:48 +0000 | Christian Urban | implemented concrete suggestion of 3rd reviewer | changeset | files | 
| Fri, 26 Nov 2010 12:17:24 +0900 | Cezary Kaliszyk | missing freshness assumptions | changeset | files | 
| Thu, 25 Nov 2010 15:06:45 +0900 | Cezary Kaliszyk | foo2 strong induction | changeset | files | 
| Wed, 24 Nov 2010 17:44:50 +0900 | Cezary Kaliszyk | foo2 full exhausts | changeset | files | 
| Wed, 24 Nov 2010 16:59:26 +0900 | Cezary Kaliszyk | Foo2 strong_exhaust for first variable. | changeset | files | 
| Mon, 22 Nov 2010 16:16:25 +0900 | Cezary Kaliszyk | single rename in let2 | changeset | files | 
| Mon, 22 Nov 2010 16:14:47 +0900 | Cezary Kaliszyk | current isabelle | changeset | files | 
| Sun, 21 Nov 2010 02:17:19 +0000 | Christian Urban | added example Foo2.thy | changeset | files | 
| Mon, 15 Nov 2010 20:54:01 +0000 | Christian Urban | tuned example | changeset | files | 
| Mon, 15 Nov 2010 09:52:29 +0000 | Christian Urban | proved that bn functions return a finite set | changeset | files | 
| Mon, 15 Nov 2010 08:17:11 +0000 | Christian Urban | added a test for the various shallow binders | changeset | files | 
| Mon, 15 Nov 2010 01:10:02 +0000 | Christian Urban | fixed bug in fv function where a shallow binder binds lists of names | changeset | files | 
| Sun, 14 Nov 2010 16:34:47 +0000 | Christian Urban | merged Nominal-General directory into Nominal; renamed Abs.thy to Nominal2_Abs.thy | changeset | files | 
| Sun, 14 Nov 2010 12:09:14 +0000 | Christian Urban | deleted special Nominal2_FSet theory | changeset | files | 
| Sun, 14 Nov 2010 11:46:39 +0000 | Christian Urban | moved rest of the lemmas from Nominal2_FSet to the TypeScheme example | changeset | files | 
| Sun, 14 Nov 2010 11:05:22 +0000 | Christian Urban | moved most material fron Nominal2_FSet into the Nominal_Base theory | changeset | files | 
| Sun, 14 Nov 2010 10:02:30 +0000 | Christian Urban | tuned example | changeset | files | 
| Sun, 14 Nov 2010 01:00:56 +0000 | Christian Urban | lifted permute_bn simp rules | changeset | files | 
| Sat, 13 Nov 2010 22:23:26 +0000 | Christian Urban | lifted permute_bn constants | changeset | files | 
| Sat, 13 Nov 2010 10:25:03 +0000 | Christian Urban | respectfulness for permute_bn functions | changeset | files | 
| Fri, 12 Nov 2010 01:20:53 +0000 | Christian Urban | automated permute_bn functions (raw ones first) | changeset | files | 
| 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 | changeset | files | 
| Wed, 10 Nov 2010 13:40:46 +0000 | Christian Urban | expanded the paper by uncommenting the comments and adding the appendix | changeset | files | 
| Sun, 07 Nov 2010 11:22:31 +0000 | Christian Urban | fixed locally the problem with the function package; all tests work again | changeset | files | 
| Sat, 06 Nov 2010 06:18:41 +0000 | Christian Urban | added a test about subtyping; disabled two tests, because of problem with function package | changeset | files | 
| Fri, 05 Nov 2010 15:21:10 +0000 | Christian Urban | small typo | changeset | files | 
| Fri, 29 Oct 2010 15:37:24 +0100 | Christian Urban | squeezed qpaper to 6 pages | changeset | files | 
| Fri, 29 Oct 2010 14:25:50 +0900 | Cezary Kaliszyk | Qpaper / Move examples to commented out appendix | changeset | files | 
| Thu, 28 Oct 2010 15:16:43 +0900 | Cezary Kaliszyk | Unanonymize qpaper | changeset | files | 
| Thu, 28 Oct 2010 14:12:30 +0900 | Cezary Kaliszyk | FSet changes for Qpaper | changeset | files | 
| Thu, 28 Oct 2010 14:03:46 +0900 | Cezary Kaliszyk | Remove FSet and use the one from Isabelle | changeset | files | 
| Tue, 19 Oct 2010 15:08:24 +0100 | Christian Urban | took out comment about map-types / adapted to recent changes | changeset | files | 
| Tue, 19 Oct 2010 10:10:41 +0100 | Christian Urban | use definitions instead of functions | changeset | files | 
| Mon, 18 Oct 2010 12:15:44 +0100 | Christian Urban | tuned | changeset | files | 
| Mon, 18 Oct 2010 11:51:22 +0100 | Christian Urban | used functions instead of definitions | changeset | files | 
| Mon, 18 Oct 2010 09:42:51 +0100 | Christian Urban | added missing style file | changeset | files | 
| Mon, 18 Oct 2010 14:13:28 +0900 | Cezary Kaliszyk | Use the generalized compositional quotient theorem | changeset | files | 
| Sun, 17 Oct 2010 21:40:23 +0100 | Christian Urban | fixed typo | changeset | files | 
| Sun, 17 Oct 2010 15:53:37 +0100 | Christian Urban | all tests work again | changeset | files | 
| Sun, 17 Oct 2010 15:28:05 +0100 | Christian Urban | some tuning | changeset | files | 
| Sun, 17 Oct 2010 13:35:52 +0100 | Christian Urban | naming scheme is now *_fset (not f*_) | changeset | files | 
| Fri, 15 Oct 2010 23:45:54 +0100 | Christian Urban | more cleaning | changeset | files | 
| Fri, 15 Oct 2010 17:37:44 +0100 | Christian Urban | further tuning | changeset | files | 
| Fri, 15 Oct 2010 16:01:03 +0100 | Christian Urban | renamed fminus_raw to diff_list | changeset | files | 
| Fri, 15 Oct 2010 15:58:48 +0100 | Christian Urban | renamed fcard_raw to card_list | changeset | files | 
| Fri, 15 Oct 2010 15:56:16 +0100 | Christian Urban | slight update | changeset | files | 
| Fri, 15 Oct 2010 15:47:20 +0100 | Christian Urban | Further reorganisation and cleaning | changeset | files | 
| Fri, 15 Oct 2010 14:11:23 +0100 | Christian Urban | further cleaning | changeset | files | 
| Fri, 15 Oct 2010 13:28:39 +0100 | Christian Urban | typo | changeset | files | 
| Fri, 15 Oct 2010 16:32:34 +0900 | Cezary Kaliszyk | FSet: stronger fact in Isabelle. | changeset | files | 
| Fri, 15 Oct 2010 16:23:26 +0900 | Cezary Kaliszyk | FSet synchronizing | changeset | files | 
| Fri, 15 Oct 2010 15:52:40 +0900 | Cezary Kaliszyk | Synchronizing FSet further. | changeset | files | 
| Fri, 15 Oct 2010 15:24:19 +0900 | Cezary Kaliszyk | Partially merging changes from Isabelle | changeset | files | 
| 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 | changeset | files | 
| Thu, 14 Oct 2010 15:58:34 +0100 | Christian Urban | changed format of the pearl paper | changeset | files | 
| Thu, 14 Oct 2010 11:09:52 +0100 | Christian Urban | deleted some unused lemmas | changeset | files | 
| 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) | changeset | files | 
| Wed, 13 Oct 2010 22:55:58 +0100 | Christian Urban | more on the pearl paper | changeset | files | 
| Tue, 12 Oct 2010 13:06:18 +0100 | Christian Urban | added a section about abstractions | changeset | files | 
| Tue, 12 Oct 2010 10:07:48 +0100 | Christian Urban | tiny work on the pearl paper | changeset | files | 
| Fri, 08 Oct 2010 23:53:51 +0100 | Christian Urban | tuned | changeset | files | 
| Fri, 08 Oct 2010 23:49:18 +0100 | Christian Urban | added apendix to paper detailing one proof | changeset | files | 
| Fri, 08 Oct 2010 15:37:11 +0100 | Christian Urban | minor | changeset | files | 
| Fri, 08 Oct 2010 15:35:14 +0100 | Christian Urban | minor | changeset | files | 
| Fri, 08 Oct 2010 13:41:54 +0100 | Christian Urban | down to 20 pages | changeset | files | 
| Thu, 07 Oct 2010 14:23:32 +0900 | Cezary Kaliszyk | minor | changeset | files | 
| Wed, 06 Oct 2010 21:32:44 +0100 | Christian Urban | down to 21 pages and changed strong induction section | changeset | files | 
| Wed, 06 Oct 2010 08:13:09 +0100 | Christian Urban | tuned | changeset | files | 
| Wed, 06 Oct 2010 08:09:40 +0100 | Christian Urban | down to 22 pages | changeset | files | 
| Tue, 05 Oct 2010 21:48:31 +0100 | Christian Urban | down to 23 pages | changeset | files | 
| Tue, 05 Oct 2010 08:43:49 +0100 | Christian Urban | down to 24 pages and a bit | changeset | files | 
| Tue, 05 Oct 2010 07:30:37 +0100 | Christian Urban | llncs and more sqeezing | changeset | files | 
| Mon, 04 Oct 2010 12:39:57 +0100 | Christian Urban | first part of sqeezing everything into 20 pages (at the moment we have 26) | changeset | files | 
| Mon, 04 Oct 2010 07:25:37 +0100 | Christian Urban | changed to llncs | changeset | files | 
| Fri, 01 Oct 2010 07:11:47 -0400 | Christian Urban | merged | changeset | files | 
| Fri, 01 Oct 2010 07:09:59 -0400 | Christian Urban | minor experiments | changeset | files | 
| Thu, 30 Sep 2010 07:43:46 -0400 | Christian Urban | merged | changeset | files | 
| Wed, 29 Sep 2010 16:49:13 -0400 | Christian Urban | simplified exhaust proofs | changeset | files | 
| Fri, 01 Oct 2010 15:44:50 +0900 | Cezary Kaliszyk | Made the paper to compile with the renamings. | changeset | files | 
| Wed, 29 Sep 2010 09:51:57 -0400 | Christian Urban | merged | changeset | files | 
| Wed, 29 Sep 2010 09:47:26 -0400 | Christian Urban | worked example Foo1 with induct_schema | changeset | files | 
| Wed, 29 Sep 2010 07:39:06 -0400 | Christian Urban | merged | changeset | files | 
| Wed, 29 Sep 2010 06:45:01 -0400 | Christian Urban | use also induct_schema for the Let-example (permute_bn is used) | changeset | files | 
| Wed, 29 Sep 2010 04:42:37 -0400 | Christian Urban | test with induct_schema for simpler strong_ind proofs | changeset | files | 
| Wed, 29 Sep 2010 16:36:31 +0900 | Cezary Kaliszyk | substitution definition with 'next_name'. | changeset | files | 
| Tue, 28 Sep 2010 08:21:47 -0400 | Christian Urban | merged | changeset | files | 
| Tue, 28 Sep 2010 05:56:11 -0400 | Christian Urban | added Foo1 to explore a contrived example | changeset | files | 
| Mon, 27 Sep 2010 12:19:17 -0400 | Christian Urban | added postprocessed fresh-lemmas for constructors | changeset | files | 
| Mon, 27 Sep 2010 09:51:15 -0400 | Christian Urban | post-processed eq_iff and supp threormes according to the fv-supp equality | changeset | files | 
| Mon, 27 Sep 2010 04:56:49 -0400 | Christian Urban | more consistent naming in Abs.thy | changeset | files | 
| Mon, 27 Sep 2010 04:56:28 -0400 | Christian Urban | some experiments | changeset | files | 
| Mon, 27 Sep 2010 04:10:36 -0400 | Christian Urban | added simp rules for prod_fv and prod_alpha | changeset | files | 
| Sun, 26 Sep 2010 17:57:30 -0400 | Christian Urban | a few more words about Ott | changeset | files | 
| Sat, 25 Sep 2010 08:38:04 -0400 | Christian Urban | lifted size_thms and exported them as <name>.size | changeset | files | 
| Sat, 25 Sep 2010 08:28:45 -0400 | Christian Urban | cleaned up two examples | changeset | files | 
| Sat, 25 Sep 2010 02:53:39 +0200 | Christian Urban | added example about datatypes | changeset | files | 
| Thu, 23 Sep 2010 05:28:40 +0200 | Christian Urban | updated to Isabelle 22 Sept | changeset | files | 
| Wed, 22 Sep 2010 23:17:25 +0200 | Christian Urban | removed dead code | changeset | files | 
| Wed, 22 Sep 2010 18:13:26 +0200 | Christian Urban | fixed | changeset | files | 
| 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 | changeset | files | 
| Mon, 20 Sep 2010 21:52:45 +0800 | Christian Urban | introduced a general procedure for structural inductions; simplified reflexivity proof | changeset | files | 
| Sat, 18 Sep 2010 06:09:43 +0800 | Christian Urban | updated to Isabelle Sept 16 | changeset | files | 
| Sat, 18 Sep 2010 05:13:42 +0800 | Christian Urban | updated to Isabelle Sept 13 | changeset | files | 
| Sun, 12 Sep 2010 22:46:40 +0800 | Christian Urban | tuned code | changeset | files | 
| Sat, 11 Sep 2010 05:56:49 +0800 | Christian Urban | tuned (to conform with indentation policy of Markus) | changeset | files | 
| 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) | changeset | files | 
| Sun, 05 Sep 2010 07:00:19 +0800 | Christian Urban | generated inducts rule by Project_Rule.projections | changeset | files | 
| Sun, 05 Sep 2010 06:42:53 +0800 | Christian Urban | added the definition supp_rel (support w.r.t. a relation) | changeset | files | 
| Sat, 04 Sep 2010 14:26:09 +0800 | Christian Urban | merged | changeset | files | 
| Sat, 04 Sep 2010 07:39:38 +0800 | Christian Urban | got rid of Nominal2_Supp (is now in Nomina2_Base) | changeset | files | 
| Sat, 04 Sep 2010 07:28:35 +0800 | Christian Urban | moved everything out of Nominal_Supp | changeset | files | 
| Sat, 04 Sep 2010 06:48:14 +0800 | Christian Urban | renamed alpha_gen -> alpha_set and Abs -> Abs_set etc | changeset | files | 
| Sat, 04 Sep 2010 06:23:31 +0800 | Christian Urban | moved a proof to Abs | changeset | files | 
| Sat, 04 Sep 2010 06:10:04 +0800 | Christian Urban | got rid of Nominal_Atoms (folded into Nominal2_Base) | changeset | files | 
| Sat, 04 Sep 2010 05:43:03 +0800 | Christian Urban | cleaned a bit various thy-files in Nominal-General | changeset | files | 
| Fri, 03 Sep 2010 22:35:35 +0800 | Christian Urban | adapted paper to changes | changeset | files | 
| Fri, 03 Sep 2010 22:22:43 +0800 | Christian Urban | made the fv-definition aggree more with alpha (needed in the support proofs) | changeset | files | 
| Fri, 03 Sep 2010 20:53:09 +0800 | Christian Urban | removed lemma finite_set (already in simpset) | changeset | files | 
| Fri, 03 Sep 2010 20:48:45 +0800 | Christian Urban | added supp_set lemma | changeset | files | 
| Thu, 02 Sep 2010 18:10:06 +0800 | Christian Urban | some experiments with support | changeset | files | 
| Thu, 02 Sep 2010 01:16:26 +0800 | Christian Urban | added eqvt-attribute for permute_abs lemmas | changeset | files | 
| Tue, 31 Aug 2010 21:03:08 +0800 | Christian Urban | slides of my talk | changeset | files | 
| Mon, 30 Aug 2010 15:59:50 +0900 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 30 Aug 2010 15:59:16 +0900 | Cezary Kaliszyk | update qpaper to new isabelle | changeset | files | 
| Mon, 30 Aug 2010 15:55:08 +0900 | Cezary Kaliszyk | No need to unfold mem_def with rsp/prs (requires new isabelle). | changeset | files | 
| Mon, 30 Aug 2010 11:02:13 +0900 | Cezary Kaliszyk | Anonymize, change Quotient to Quot and fix indentation | changeset | files | 
| Sun, 29 Aug 2010 13:36:03 +0800 | Christian Urban | renamed NewParser to Nominal2 | changeset | files | 
| Sun, 29 Aug 2010 12:17:25 +0800 | Christian Urban | tuned | changeset | files | 
| Sun, 29 Aug 2010 12:14:40 +0800 | Christian Urban | updated todos | changeset | files | 
| Sun, 29 Aug 2010 01:45:07 +0800 | Christian Urban | added fs-instance proofs | changeset | files | 
| Sun, 29 Aug 2010 01:17:36 +0800 | Christian Urban | added proofs for fsupp properties | changeset | files | 
| Sun, 29 Aug 2010 00:36:47 +0800 | Christian Urban | fiexed problem with constructors that have no arguments | changeset | files | 
| Sun, 29 Aug 2010 00:09:45 +0800 | Christian Urban | proved supports lemmas | changeset | files | 
| Sat, 28 Aug 2010 18:15:23 +0800 | Christian Urban | slight cleaning | changeset | files | 
| Sat, 28 Aug 2010 13:41:31 +0800 | Christian Urban | updated to new Isabelle | changeset | files | 
| Fri, 27 Aug 2010 23:26:00 +0800 | Christian Urban | cut out most of the lifting section and cleaned up everything | changeset | files | 
| Fri, 27 Aug 2010 19:06:30 +0800 | Christian Urban | made all typographic changes | changeset | files | 
| Fri, 27 Aug 2010 16:00:19 +0800 | Christian Urban | first pass on section 1 | changeset | files | 
| Fri, 27 Aug 2010 13:57:00 +0800 | Christian Urban | make copies of the "old" files | changeset | files | 
| Fri, 27 Aug 2010 02:25:40 +0000 | Cezary Kaliszyk | Ball Bex can be lifted after unfolding. | changeset | 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) | changeset | files | 
| Fri, 27 Aug 2010 02:08:36 +0800 | Christian Urban | merged | changeset | files | 
| Fri, 27 Aug 2010 02:03:52 +0800 | Christian Urban | corrected bug with fv-function generation (that was the problem with recursive binders) | changeset | files | 
| Thu, 26 Aug 2010 14:55:15 +0900 | Cezary Kaliszyk | minor | changeset | files | 
| Thu, 26 Aug 2010 02:08:00 +0800 | Christian Urban | cleaned up (almost completely) the examples | changeset | files | 
| Wed, 25 Aug 2010 23:16:42 +0800 | Christian Urban | cleaning of unused files and code | changeset | files | 
| Wed, 25 Aug 2010 22:55:42 +0800 | Christian Urban | automatic lifting | changeset | files | 
| Wed, 25 Aug 2010 20:19:10 +0800 | Christian Urban | everything now lifts as expected | changeset | files | 
| Wed, 25 Aug 2010 11:58:37 +0800 | Christian Urban | now every lemma lifts (even with type variables) | changeset | files | 
| Wed, 25 Aug 2010 09:02:06 +0800 | Christian Urban | can now deal with type variables in nominal datatype definitions | changeset | files | 
| Sun, 22 Aug 2010 14:02:49 +0800 | Christian Urban | updated to new Isabelle | changeset | files | 
| Sun, 22 Aug 2010 12:36:53 +0800 | Christian Urban | merged | changeset | files | 
| Sun, 22 Aug 2010 11:00:53 +0800 | Christian Urban | updated to new Isabelle | changeset | files | 
| Sat, 21 Aug 2010 20:07:52 +0800 | Christian Urban | not needed anymore | changeset | files | 
| Sat, 21 Aug 2010 20:07:36 +0800 | Christian Urban | moved lifting code from Lift.thy to nominal_dt_quot.ML | changeset | files | 
| Sat, 21 Aug 2010 17:55:42 +0800 | Christian Urban | nominal_datatypes with type variables do not work | changeset | files | 
| 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 | changeset | files | 
| Fri, 20 Aug 2010 16:55:58 +0900 | Cezary Kaliszyk | Clarifications to FIXMEs. | changeset | files | 
| Fri, 20 Aug 2010 16:50:46 +0900 | Cezary Kaliszyk | Finished adding remarks from the reviewers. | changeset | files | 
| Fri, 20 Aug 2010 16:39:39 +0900 | Cezary Kaliszyk | few remaining remarks as fixme's. | changeset | files | 
| Thu, 19 Aug 2010 18:24:36 +0800 | Christian Urban | used @{const_name} hopefully everywhere | changeset | files | 
| Thu, 19 Aug 2010 16:08:10 +0900 | Cezary Kaliszyk | Intuition behind REL | changeset | files | 
| Thu, 19 Aug 2010 16:05:31 +0900 | Cezary Kaliszyk | add missing mathpartir | changeset | files | 
| Thu, 19 Aug 2010 15:52:36 +0900 | Cezary Kaliszyk | Add 2 FIXMEs | changeset | files | 
| Thu, 19 Aug 2010 15:46:28 +0900 | Cezary Kaliszyk | The type does determine respectfulness, the constant without an instantiated type does not. | changeset | files | 
| Thu, 19 Aug 2010 15:02:11 +0900 | Cezary Kaliszyk | Add the SAC stylesheet and updated root file. | changeset | files | 
| Thu, 19 Aug 2010 14:28:54 +0900 | Cezary Kaliszyk | TODO | changeset | files | 
| Thu, 19 Aug 2010 13:58:47 +0900 | Cezary Kaliszyk | further comments from the referees | changeset | files | 
| Thu, 19 Aug 2010 13:00:49 +0900 | Cezary Kaliszyk | fixes for referees | changeset | files | 
| Wed, 18 Aug 2010 00:23:42 +0800 | Christian Urban | put everything in a "timeit" | changeset | files | 
| Wed, 18 Aug 2010 00:19:15 +0800 | Christian Urban | improved runtime slightly, by constructing an explicit size measure for the function definitions | changeset | files | 
| Tue, 17 Aug 2010 18:17:53 +0800 | Christian Urban | more tuning of the code | changeset | files | 
| Tue, 17 Aug 2010 18:00:55 +0800 | Christian Urban | deleted unused code | changeset | files | 
| Tue, 17 Aug 2010 17:52:25 +0800 | Christian Urban | improved code | changeset | files | 
| Tue, 17 Aug 2010 07:11:45 +0800 | Christian Urban | can also lift the various eqvt lemmas for bn, fv, fv_bn and size | changeset | files | 
| Tue, 17 Aug 2010 06:50:49 +0800 | Christian Urban | also able to lift the bn_defs | changeset | files | 
| Tue, 17 Aug 2010 06:39:27 +0800 | Christian Urban | added rsp-lemmas for alpha_bns | changeset | files | 
| Mon, 16 Aug 2010 19:57:41 +0800 | Christian Urban | cezary made the eq_iff lemmas to lift (still needs some infrastructure in quotient) | changeset | files | 
| Mon, 16 Aug 2010 17:59:09 +0800 | Christian Urban | pinpointed the problem | changeset | files | 
| Mon, 16 Aug 2010 17:39:16 +0800 | Christian Urban | modified the code for class instantiations (with help from Florian) | changeset | files | 
| Sun, 15 Aug 2010 14:00:28 +0800 | Christian Urban | defined qperms and qsizes | changeset | files | 
| Sun, 15 Aug 2010 11:03:13 +0800 | Christian Urban | simplified code | changeset | files | 
| Sat, 14 Aug 2010 23:33:23 +0800 | Christian Urban | improved code | changeset | files | 
| Sat, 14 Aug 2010 16:54:41 +0800 | Christian Urban | more experiments with lifting | changeset | files | 
| Thu, 12 Aug 2010 21:29:35 +0800 | Christian Urban | updated to Isabelle 12th Aug | changeset | files | 
| Wed, 11 Aug 2010 19:53:57 +0800 | Christian Urban | rsp for constructors | changeset | files | 
| Wed, 11 Aug 2010 16:23:50 +0800 | Christian Urban | updated to Isabelle 11 Aug | changeset | files | 
| Wed, 11 Aug 2010 16:21:24 +0800 | Christian Urban | added a function that transforms the helper-rsp lemmas into real rsp lemmas | changeset | files | 
| Sun, 08 Aug 2010 10:12:38 +0800 | Christian Urban | proved rsp-helper lemmas of size functions | changeset | files | 
| Sat, 31 Jul 2010 02:10:42 +0100 | Christian Urban | tuning | changeset | files | 
| Sat, 31 Jul 2010 02:05:25 +0100 | Christian Urban | further simplification with alpha_prove | changeset | files | 
| Sat, 31 Jul 2010 01:24:39 +0100 | Christian Urban | introduced a general alpha_prove method | changeset | files | 
| Fri, 30 Jul 2010 00:40:32 +0100 | Christian Urban | equivariance for size | changeset | files | 
| Thu, 29 Jul 2010 10:16:33 +0100 | Christian Urban | helper lemmas for rsp-lemmas | changeset | files | 
| Tue, 27 Jul 2010 23:34:30 +0200 | Christian Urban | tests | changeset | files | 
| Tue, 27 Jul 2010 14:37:59 +0200 | Christian Urban | cleaned up a bit Abs.thy | changeset | files | 
| Tue, 27 Jul 2010 09:09:02 +0200 | Christian Urban | fixed order of fold_union to make alpha and fv agree | changeset | files | 
| Mon, 26 Jul 2010 09:19:28 +0200 | Christian Urban | small cleaning | changeset | files | 
| Sun, 25 Jul 2010 22:42:21 +0200 | Christian Urban | added paper by james; some minor cleaning | changeset | files | 
| Fri, 23 Jul 2010 16:42:47 +0200 | Christian Urban | samll changes | changeset | files | 
| Fri, 23 Jul 2010 16:42:00 +0200 | Christian Urban | made compatible | changeset | files | 
| Fri, 23 Jul 2010 16:41:36 +0200 | Christian Urban | added | changeset | files | 
| Thu, 22 Jul 2010 08:30:50 +0200 | Christian Urban | updated to new Isabelle; made FSet more "quiet" | changeset | files | 
| Tue, 20 Jul 2010 06:14:16 +0100 | Christian Urban | merged | changeset | files | 
| Mon, 19 Jul 2010 08:55:49 +0100 | Christian Urban | minor | changeset | files | 
| Mon, 19 Jul 2010 16:59:43 +0100 | Christian Urban | minor polishing | changeset | files | 
| Mon, 19 Jul 2010 14:20:23 +0100 | Christian Urban | quote for a new paper | changeset | files | 
| Mon, 19 Jul 2010 08:34:38 +0100 | Christian Urban | corrected lambda-preservation theorem | changeset | files | 
| Mon, 19 Jul 2010 07:49:10 +0100 | Christian Urban | minor | changeset | files | 
| Sun, 18 Jul 2010 19:07:05 +0100 | Christian Urban | minor things on the paper | changeset | files | 
| Sun, 18 Jul 2010 17:03:05 +0100 | Christian Urban | merged | changeset | files | 
| Sun, 18 Jul 2010 17:02:33 +0100 | Christian Urban | minor things | changeset | files | 
| Sun, 18 Jul 2010 16:06:34 +0100 | Christian Urban | some test with quotient | changeset | files | 
| Sat, 17 Jul 2010 15:44:24 +0100 | Christian Urban | some minor changes | changeset | files | 
| Sat, 17 Jul 2010 12:01:04 +0100 | Christian Urban | changes suggested by Peter Homeier | changeset | files | 
| Sat, 17 Jul 2010 10:25:29 +0100 | Christian Urban | tests | changeset | files | 
| Fri, 16 Jul 2010 05:09:45 +0100 | Christian Urban | submitted version | changeset | files | 
| Fri, 16 Jul 2010 04:58:46 +0100 | Christian Urban | more paper | changeset | files | 
| Fri, 16 Jul 2010 03:22:24 +0100 | Christian Urban | more on the paper | changeset | files | 
| Fri, 16 Jul 2010 02:38:19 +0100 | Christian Urban | more on the paper | changeset | files | 
| Thu, 15 Jul 2010 09:40:05 +0100 | Christian Urban | a bit more to the paper | changeset | files | 
| Wed, 14 Jul 2010 21:30:52 +0100 | Christian Urban | more on the paper | changeset | files | 
| Tue, 13 Jul 2010 23:39:39 +0100 | Christian Urban | more on slides | changeset | files | 
| Tue, 13 Jul 2010 14:37:28 +0100 | Christian Urban | slides | changeset | files | 
| Mon, 12 Jul 2010 21:48:39 +0100 | Christian Urban | more on slides | changeset | files | 
| Sun, 11 Jul 2010 21:18:02 +0100 | Christian Urban | slides | changeset | files | 
| Sun, 11 Jul 2010 00:58:54 +0100 | Christian Urban | slides | changeset | files | 
| Sat, 10 Jul 2010 23:36:45 +0100 | Christian Urban | more on slides | changeset | files | 
| Sat, 10 Jul 2010 15:50:33 +0100 | Christian Urban | more on slides | changeset | files | 
| Sat, 10 Jul 2010 11:27:04 +0100 | Christian Urban | added material for slides | changeset | files | 
| Fri, 09 Jul 2010 23:04:51 +0100 | Christian Urban | fixed | changeset | files | 
| Fri, 09 Jul 2010 18:50:02 +0100 | Christian Urban | before examples | changeset | files | 
| Fri, 09 Jul 2010 10:00:37 +0100 | Christian Urban | finished alpha-section | changeset | files | 
| Wed, 07 Jul 2010 13:13:18 +0100 | Christian Urban | more on the paper | changeset | files | 
| Wed, 07 Jul 2010 09:34:00 +0100 | Christian Urban | more on the paper | changeset | files | 
| Fri, 02 Jul 2010 15:34:46 +0100 | Christian Urban | more on the paper | changeset | files | 
| Fri, 02 Jul 2010 01:54:19 +0100 | Christian Urban | finished fv-section | changeset | files | 
| Thu, 01 Jul 2010 14:18:36 +0100 | Christian Urban | more on the paper | changeset | files | 
| Thu, 01 Jul 2010 01:53:00 +0100 | Christian Urban | spell check | changeset | files | 
| Wed, 30 Jun 2010 16:56:37 +0100 | Christian Urban | more work on the paper | changeset | files | 
| Tue, 29 Jun 2010 18:00:59 +0100 | Christian Urban | removed an "eqvt"-warning | changeset | files | 
| Mon, 28 Jun 2010 16:22:28 +0100 | Christian Urban | more quotient-definitions | changeset | files | 
| Mon, 28 Jun 2010 15:23:56 +0100 | Christian Urban | slight cleaning | changeset | files | 
| Sun, 27 Jun 2010 21:41:21 +0100 | Christian Urban | fixed according to changes in quotient | changeset | files | 
| Thu, 24 Jun 2010 21:35:11 +0100 | Christian Urban | added definition of the quotient types | changeset | files | 
| Thu, 24 Jun 2010 19:32:33 +0100 | Christian Urban | fixed according to changes in quotient | changeset | files | 
| Thu, 24 Jun 2010 00:41:41 +0100 | Christian Urban | added comment about partial equivalence relations | changeset | files | 
| Thu, 24 Jun 2010 00:27:37 +0100 | Christian Urban | even further polishing of the qpaper | changeset | files | 
| Wed, 23 Jun 2010 22:41:16 +0100 | Christian Urban | polished paper again (and took out some claims about Homeier's package) | changeset | files | 
| Wed, 23 Jun 2010 15:59:43 +0100 | Christian Urban | some slight polishing on the paper | changeset | files | 
| Wed, 23 Jun 2010 15:40:00 +0100 | Christian Urban | merged cezary's changes | changeset | files | 
| Wed, 23 Jun 2010 15:21:04 +0100 | Christian Urban | whitespace | changeset | files | 
| Wed, 23 Jun 2010 09:01:45 +0200 | Cezary Kaliszyk | Un-do the second change to SingleLet. | changeset | files | 
| Wed, 23 Jun 2010 08:49:33 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 23 Jun 2010 08:48:38 +0200 | Cezary Kaliszyk | Changes for PER and list_all2 committed to Isabelle | changeset | files | 
| Fri, 18 Jun 2010 15:22:58 +0200 | Cezary Kaliszyk | changes for partial-equivalence quotient package | changeset | files | 
| Wed, 23 Jun 2010 06:54:48 +0100 | Christian Urban | deleted compose-lemmas in Abs (not needed anymore) | changeset | files | 
| Wed, 23 Jun 2010 06:45:03 +0100 | Christian Urban | deleted equivp_hack | changeset | files | 
| Tue, 22 Jun 2010 18:07:53 +0100 | Christian Urban | proved eqvip theorems for alphas | changeset | files | 
| Tue, 22 Jun 2010 13:31:42 +0100 | Christian Urban | cleaned up the FSet (noise was introduced by error) | changeset | files | 
| Tue, 22 Jun 2010 13:05:00 +0100 | Christian Urban | prove that alpha implies alpha_bn (needed for rsp proofs) | changeset | files | 
| Mon, 21 Jun 2010 15:41:59 +0100 | Christian Urban | further post-submission tuning | changeset | files | 
| Mon, 21 Jun 2010 06:47:40 +0100 | Christian Urban | merged with main line | changeset | files | 
| Mon, 21 Jun 2010 06:46:28 +0100 | Christian Urban | merged | changeset | files | 
| Fri, 11 Jun 2010 03:02:42 +0200 | Christian Urban | also symmetry | changeset | files | 
| Thu, 10 Jun 2010 14:53:45 +0200 | Christian Urban | merged | changeset | files | 
| Thu, 10 Jun 2010 14:53:28 +0200 | Christian Urban | premerge | changeset | files | 
| Wed, 09 Jun 2010 15:14:16 +0200 | Christian Urban | transitivity proofs done | changeset | files | 
| Mon, 07 Jun 2010 11:46:26 +0200 | Christian Urban | merged | changeset | files | 
| Mon, 07 Jun 2010 11:43:01 +0200 | Christian Urban | work on transitivity proof | changeset | files | 
| Thu, 03 Jun 2010 15:02:52 +0200 | Christian Urban | added uminus_eqvt | changeset | files | 
| Thu, 03 Jun 2010 11:48:44 +0200 | Christian Urban | fixed problem with eqvt proofs | changeset | files | 
| Wed, 02 Jun 2010 11:37:51 +0200 | Christian Urban | fixed problem with bn_info | changeset | files | 
| Tue, 01 Jun 2010 15:46:07 +0200 | Christian Urban | merged | changeset | files | 
| Tue, 01 Jun 2010 15:21:01 +0200 | Christian Urban | equivariance done | changeset | files | 
| Tue, 01 Jun 2010 15:01:05 +0200 | Christian Urban | smaller code for raw-eqvt proofs | changeset | files | 
| Mon, 31 May 2010 19:57:29 +0200 | Christian Urban | all raw definitions are defined using function | changeset | files | 
| Thu, 27 May 2010 18:40:10 +0200 | Christian Urban | merged | changeset | files | 
| Thu, 27 May 2010 18:37:52 +0200 | Christian Urban | intermediate state | changeset | files | 
| Wed, 26 May 2010 15:37:56 +0200 | Christian Urban | merged | changeset | files | 
| Wed, 26 May 2010 15:34:54 +0200 | Christian Urban | added FSet to the correct paper | changeset | files | 
| Tue, 25 May 2010 00:24:41 +0100 | Christian Urban | added slides | changeset | files | 
| Mon, 24 May 2010 21:11:33 +0100 | Christian Urban | tuned | changeset | files | 
| Mon, 24 May 2010 20:50:15 +0100 | Christian Urban | tuned | changeset | files | 
| Mon, 24 May 2010 20:02:37 +0100 | Christian Urban | alpha works now | changeset | files | 
| Sun, 23 May 2010 02:15:24 +0100 | Christian Urban | started to work on alpha | changeset | files | 
| Sat, 22 May 2010 13:51:47 +0100 | Christian Urban | properly exported bn_descr | changeset | files | 
| Fri, 21 May 2010 11:40:18 +0100 | Christian Urban | hving a working fv-definition without the export | changeset | files | 
| Fri, 21 May 2010 05:58:23 +0100 | Christian Urban | tuned | changeset | files | 
| Fri, 21 May 2010 00:44:39 +0100 | Christian Urban | proper parser for "exclude:" | changeset | files | 
| Thu, 20 May 2010 21:47:12 +0100 | Christian Urban | tuned | changeset | files | 
| Thu, 20 May 2010 21:35:00 +0100 | Christian Urban | moved some mk_union and mk_diff into the library | changeset | files | 
| 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 | changeset | files | 
| Mon, 21 Jun 2010 02:04:39 +0100 | Christian Urban | some post-submission polishing | changeset | files | 
| Mon, 21 Jun 2010 00:45:27 +0100 | Christian Urban | added a few points that need to be looked at the next version of the qpaper | changeset | files | 
| Mon, 21 Jun 2010 00:36:17 +0100 | Christian Urban | eliminated a quot_thm flag | changeset | files | 
| Sun, 20 Jun 2010 02:37:58 +0100 | Christian Urban | fixed example | changeset | files | 
| Sun, 20 Jun 2010 02:37:44 +0100 | Christian Urban | small addition to the acknowledgement | changeset | files | 
| Thu, 17 Jun 2010 09:25:44 +0200 | Cezary Kaliszyk | qpaper / address FIXMEs. | changeset | files | 
| Thu, 17 Jun 2010 07:37:26 +0200 | Cezary Kaliszyk | forgot to save | changeset | files | 
| Thu, 17 Jun 2010 07:34:29 +0200 | Cezary Kaliszyk | Fix regularization. Two "FIXME" left in introduction. Minor spellings. | changeset | files | 
| Thu, 17 Jun 2010 00:27:57 +0100 | Christian Urban | polished everything and submitted | changeset | files | 
| Wed, 16 Jun 2010 22:29:42 +0100 | Christian Urban | conclusion done | changeset | files | 
| Wed, 16 Jun 2010 14:26:23 +0200 | Cezary Kaliszyk | Answer questions in comments | changeset | files | 
| Wed, 16 Jun 2010 03:47:38 +0100 | Christian Urban | tuned | changeset | files | 
| Wed, 16 Jun 2010 03:44:10 +0100 | Christian Urban | finished section 4, but put some things I do not understand on comment | changeset | files | 
| Wed, 16 Jun 2010 02:55:52 +0100 | Christian Urban | 4 almost finished | changeset | files | 
| Tue, 15 Jun 2010 22:25:03 +0200 | Christian Urban | cleaned up definitions | changeset | files | 
| Tue, 15 Jun 2010 12:00:03 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 15 Jun 2010 11:59:16 +0200 | Cezary Kaliszyk | qpaper/Rewrite section5 | changeset | files | 
| Tue, 15 Jun 2010 09:44:16 +0200 | Christian Urban | merged | changeset | files | 
| Tue, 15 Jun 2010 08:56:13 +0200 | Christian Urban | tuned everytinh up to section 4 | changeset | files | 
| Tue, 15 Jun 2010 10:08:12 +0200 | Cezary Kaliszyk | Definition of Respects. | changeset | files | 
| Tue, 15 Jun 2010 09:22:38 +0200 | Cezary Kaliszyk | conclusion | changeset | files | 
| Tue, 15 Jun 2010 09:12:54 +0200 | Cezary Kaliszyk | Qpaper / Clarify the typing system and composition of quotients issue. | changeset | files | 
| Tue, 15 Jun 2010 07:58:33 +0200 | Cezary Kaliszyk | Remove only reference to 'equivp'. | changeset | files | 
| Tue, 15 Jun 2010 07:54:30 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 15 Jun 2010 07:52:42 +0200 | Cezary Kaliszyk | qpaper/ackno | changeset | files | 
| Tue, 15 Jun 2010 06:50:33 +0200 | Christian Urban | tuned | changeset | files | 
| Tue, 15 Jun 2010 06:35:57 +0200 | Cezary Kaliszyk | qpaper | changeset | files | 
| Tue, 15 Jun 2010 05:43:21 +0200 | Cezary Kaliszyk | qpaper / hol4 | changeset | files | 
| Tue, 15 Jun 2010 05:32:50 +0200 | Cezary Kaliszyk | qpaper/related work | changeset | files | 
| Tue, 15 Jun 2010 02:03:18 +0200 | Christian Urban | finished preliminary section | changeset | files | 
| Mon, 14 Jun 2010 19:03:34 +0200 | Christian Urban | typo | changeset | files | 
| Mon, 14 Jun 2010 19:02:25 +0200 | Christian Urban | some slight tuning of the preliminary section | changeset | files | 
| Mon, 14 Jun 2010 16:45:29 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 14 Jun 2010 16:44:53 +0200 | Cezary Kaliszyk | qpaper | changeset | files | 
| Mon, 14 Jun 2010 14:28:32 +0200 | Christian Urban | merged | changeset | files | 
| Mon, 14 Jun 2010 14:28:12 +0200 | Christian Urban | tuned | changeset | files | 
| Mon, 14 Jun 2010 15:16:42 +0200 | Cezary Kaliszyk | Qpaper / beginnig of sec5 | changeset | files | 
| Mon, 14 Jun 2010 14:45:40 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 14 Jun 2010 14:44:18 +0200 | Cezary Kaliszyk | qpaper/unfold the ball_reg_right statement | changeset | files | 
| Mon, 14 Jun 2010 12:30:08 +0200 | Christian Urban | merged | changeset | files | 
| Mon, 14 Jun 2010 11:51:34 +0200 | Christian Urban | some tuning and start work on section 4 | changeset | files | 
| Mon, 14 Jun 2010 13:24:22 +0200 | Cezary Kaliszyk | qpaper | changeset | files | 
| Mon, 14 Jun 2010 12:07:55 +0200 | Cezary Kaliszyk | qpaper / INJ | changeset | files | 
| Mon, 14 Jun 2010 11:42:07 +0200 | Cezary Kaliszyk | qpaper / REG | changeset | files | 
| Mon, 14 Jun 2010 10:14:39 +0200 | Cezary Kaliszyk | qpaper / minor | changeset | files | 
| Mon, 14 Jun 2010 09:28:52 +0200 | Cezary Kaliszyk | qpaper/various | changeset | files | 
| Mon, 14 Jun 2010 09:16:22 +0200 | Cezary Kaliszyk | qpaper | changeset | files | 
| Mon, 14 Jun 2010 08:25:03 +0200 | Cezary Kaliszyk | qpaper/more on example | changeset | files | 
| Mon, 14 Jun 2010 07:55:02 +0200 | Cezary Kaliszyk | qpaper/examples | changeset | files | 
| Mon, 14 Jun 2010 04:38:25 +0200 | Christian Urban | completed proof and started section about respectfulness and preservation | changeset | files | 
| Sun, 13 Jun 2010 20:54:50 +0200 | Christian Urban | more on the qpaper | changeset | files | 
| Sun, 13 Jun 2010 17:41:07 +0200 | Christian Urban | tuned | changeset | files | 
| Sun, 13 Jun 2010 17:40:32 +0200 | Christian Urban | more on the constant lifting section | changeset | files | 
| Sun, 13 Jun 2010 17:01:15 +0200 | Christian Urban | something about the quotient ype definitions | changeset | files | 
| Sun, 13 Jun 2010 14:39:55 +0200 | Christian Urban | added some examples | changeset | files | 
| Sun, 13 Jun 2010 13:42:37 +0200 | Christian Urban | improved definition of ABS and REP | changeset | files | 
| Sun, 13 Jun 2010 07:14:53 +0200 | Cezary Kaliszyk | qpaper. | changeset | files | 
| Sun, 13 Jun 2010 06:50:34 +0200 | Cezary Kaliszyk | some spelling | changeset | files | 
| Sun, 13 Jun 2010 06:45:20 +0200 | Cezary Kaliszyk | minor | changeset | files | 
| Sun, 13 Jun 2010 06:34:22 +0200 | Cezary Kaliszyk | qpaper / tuning in preservation and general display | changeset | files | 
| Sun, 13 Jun 2010 04:06:06 +0200 | Christian Urban | polishing of ABS/REP | changeset | files | 
| Sat, 12 Jun 2010 11:32:36 +0200 | Christian Urban | some slight tuning of the intro | changeset | files | 
| Sat, 12 Jun 2010 06:35:27 +0200 | Cezary Kaliszyk | Fix integer relation. | changeset | files | 
| Sat, 12 Jun 2010 02:36:49 +0200 | Christian Urban | completed the intro (except minor things) | changeset | files | 
| Fri, 11 Jun 2010 21:58:25 +0200 | Christian Urban | more intro | changeset | files | 
| Fri, 11 Jun 2010 17:52:06 +0200 | Christian Urban | more on the qpaper | changeset | files | 
| Fri, 11 Jun 2010 16:36:02 +0200 | Christian Urban | even more on the qpaper (intro almost done) | changeset | files | 
| Fri, 11 Jun 2010 14:04:58 +0200 | Christian Urban | more to the introduction of the qpaper | changeset | files | 
| Thu, 10 Jun 2010 13:37:32 +0200 | Christian Urban | adapted to the official sigplan style file (this gives us more space) | changeset | files | 
| Thu, 10 Jun 2010 13:28:38 +0200 | Christian Urban | added to the popl-paper a pointer to work by Altenkirch | changeset | files | 
| Thu, 10 Jun 2010 10:53:51 +0200 | Christian Urban | more on the qpaper | changeset | files | 
| Mon, 07 Jun 2010 16:17:35 +0200 | Christian Urban | new title for POPL paper | changeset | files | 
| Mon, 07 Jun 2010 15:57:03 +0200 | Christian Urban | more work on intro and abstract (done for today) | changeset | files | 
| Mon, 07 Jun 2010 15:13:39 +0200 | Christian Urban | a bit more in the introduction and abstract | changeset | files | 
| Mon, 07 Jun 2010 11:33:00 +0200 | Christian Urban | improved abstract, some tuning | changeset | files | 
| Sun, 06 Jun 2010 13:16:27 +0200 | Cezary Kaliszyk | Qpaper / minor on cleaning | changeset | files | 
| Sat, 05 Jun 2010 14:37:05 +0200 | Cezary Kaliszyk | qpaper / injection proof. | changeset | files | 
| Sat, 05 Jun 2010 10:03:42 +0200 | Cezary Kaliszyk | qpaper / example interaction | changeset | files | 
| Sat, 05 Jun 2010 08:02:39 +0200 | Cezary Kaliszyk | Qpaper/regularization proof. | changeset | files | 
| Sat, 05 Jun 2010 07:26:22 +0200 | Cezary Kaliszyk | qpaper | changeset | files | 
| Wed, 02 Jun 2010 14:24:16 +0200 | Cezary Kaliszyk | Qpaper/more. | changeset | files | 
| Wed, 02 Jun 2010 13:58:37 +0200 | Cezary Kaliszyk | Qpaper/Minor | changeset | files | 
| Tue, 01 Jun 2010 15:58:59 +0200 | Christian Urban | added larry's quote | changeset | files | 
| Tue, 01 Jun 2010 15:48:25 +0200 | Christian Urban | added larry's paper | changeset | files | 
| Tue, 01 Jun 2010 15:45:43 +0200 | Christian Urban | tuned | changeset | files | 
| Sat, 29 May 2010 00:16:39 +0200 | Christian Urban | first version of the abstract | changeset | files | 
| Thu, 27 May 2010 18:30:42 +0200 | Christian Urban | merged | changeset | files | 
| Thu, 27 May 2010 18:30:26 +0200 | Christian Urban | fixed bug where perm_simp 'forgets' how to prove equivariance for the empty set | changeset | files | 
| Thu, 27 May 2010 16:53:12 +0200 | Cezary Kaliszyk | qpaper / lemmas used in proofs | changeset | files | 
| Thu, 27 May 2010 16:33:10 +0200 | Cezary Kaliszyk | qpaper / injection statement | changeset | files | 
| Thu, 27 May 2010 16:06:43 +0200 | Cezary Kaliszyk | qpaper / regularize | changeset | files | 
| Thu, 27 May 2010 14:30:07 +0200 | Cezary Kaliszyk | qpaper / a bit about prs | changeset | files | 
| Thu, 27 May 2010 11:21:37 +0200 | Cezary Kaliszyk | Functionalized the ABS/REP definition. | changeset | files | 
| Wed, 26 May 2010 17:55:42 +0200 | Cezary Kaliszyk | qpaper / lifting introduction | changeset | files | 
| Wed, 26 May 2010 17:20:59 +0200 | Cezary Kaliszyk | merged | changeset | files | 
| Wed, 26 May 2010 17:19:16 +0200 | Christian Urban | fixed compile error | changeset | files | 
| Wed, 26 May 2010 17:10:05 +0200 | Cezary Kaliszyk | qpaper / composition of quotients. | changeset | files | 
| Wed, 26 May 2010 16:56:38 +0200 | Cezary Kaliszyk | qpaper | changeset | files | 
| Wed, 26 May 2010 16:28:35 +0200 | Cezary Kaliszyk | qpaper.. | changeset | files | 
| Wed, 26 May 2010 16:17:49 +0200 | Cezary Kaliszyk | qpaper. | changeset | files | 
| Wed, 26 May 2010 16:09:09 +0200 | Cezary Kaliszyk | Name some respectfullness | changeset | files | 
| Wed, 26 May 2010 15:35:34 +0200 | Christian Urban | added FSet to the correct paper | changeset | files | 
| Wed, 26 May 2010 15:26:22 +0200 | Christian Urban | merged | changeset | files | 
| Wed, 26 May 2010 15:26:00 +0200 | Christian Urban | added FSet | changeset | files | 
| Wed, 26 May 2010 15:24:33 +0200 | Cezary Kaliszyk | qpaper | changeset | files | 
| Wed, 26 May 2010 12:11:58 +0200 | Cezary Kaliszyk | qpaper | changeset | files | 
| Tue, 25 May 2010 18:38:52 +0200 | Cezary Kaliszyk | Substitution Lemma for TypeSchemes. | changeset | files | 
| Tue, 25 May 2010 17:29:05 +0200 | Cezary Kaliszyk | Simplified the proof | changeset | files | 
| Tue, 25 May 2010 17:09:29 +0200 | Cezary Kaliszyk | A lemma about substitution in TypeSchemes. | changeset | files | 
| Tue, 25 May 2010 17:01:37 +0200 | Cezary Kaliszyk | reversing the direction of fresh_star | changeset | files | 
| Tue, 25 May 2010 10:43:19 +0200 | Cezary Kaliszyk | overlapping deep binders proof | changeset | files | 
| Tue, 25 May 2010 07:59:16 +0200 | Christian Urban | edits from the reviewers | changeset | files | 
| Mon, 24 May 2010 22:47:06 +0100 | Christian Urban | tuned paper | changeset | files | 
| Sun, 23 May 2010 16:45:00 +0100 | Christian Urban | changed qpaper to lncs-style | changeset | files | 
| Fri, 21 May 2010 17:17:51 +0200 | Cezary Kaliszyk | Match_Lam defined on Quotient Level. | changeset | files | 
| Fri, 21 May 2010 11:55:22 +0200 | Cezary Kaliszyk | More on Function-defined subst. | changeset | files | 
| Fri, 21 May 2010 11:46:47 +0200 | Cezary Kaliszyk | Isabelle renamings | changeset | files | 
| Fri, 21 May 2010 10:47:45 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Fri, 21 May 2010 10:43:14 +0200 | Cezary Kaliszyk | Renamings. | changeset | files | 
| Fri, 21 May 2010 10:42:53 +0200 | Cezary Kaliszyk | Renamings | changeset | files | 
| Fri, 21 May 2010 10:47:07 +0200 | Cezary Kaliszyk | merge (non-trival) | changeset | files | 
| Fri, 21 May 2010 10:45:29 +0200 | Cezary Kaliszyk | Previously uncommited direct subst definition changes. | changeset | files | 
| Fri, 21 May 2010 10:44:07 +0200 | Cezary Kaliszyk | Function experiments | changeset | files | 
| Wed, 19 May 2010 12:44:03 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 19 May 2010 12:43:38 +0100 | Christian Urban | added comments about pottiers work | changeset | files | 
| Wed, 19 May 2010 12:29:08 +0200 | Cezary Kaliszyk | more subst experiments | changeset | files | 
| Wed, 19 May 2010 11:29:42 +0200 | Cezary Kaliszyk | More subst experminets | changeset | files | 
| Tue, 18 May 2010 17:56:41 +0200 | Cezary Kaliszyk | more on subst | changeset | files | 
| Tue, 18 May 2010 17:17:54 +0200 | Cezary Kaliszyk | Single variable substitution | changeset | files | 
| Tue, 18 May 2010 17:06:21 +0200 | Cezary Kaliszyk | subst fix | changeset | files | 
| Tue, 18 May 2010 15:58:52 +0200 | Cezary Kaliszyk | subst experiments | changeset | files | 
| Tue, 18 May 2010 14:40:05 +0100 | Christian Urban | soem minor tuning | changeset | files | 
| Tue, 18 May 2010 11:47:29 +0200 | Cezary Kaliszyk | Fix broken add | changeset | files | 
| Tue, 18 May 2010 11:46:58 +0200 | Cezary Kaliszyk | add missing .bib | changeset | files | 
| Tue, 18 May 2010 11:46:19 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 18 May 2010 11:45:49 +0200 | Cezary Kaliszyk | starting bibliography | changeset | files | 
| Mon, 17 May 2010 20:23:40 +0100 | Christian Urban | merged | changeset | files | 
| Mon, 17 May 2010 18:13:39 +0100 | Christian Urban | updated to new Isabelle (More_Conv -> Conv) | changeset | files | 
| Mon, 17 May 2010 17:54:07 +0100 | Christian Urban | made this example to work again | changeset | files | 
| Mon, 17 May 2010 17:34:02 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 17 May 2010 17:31:18 +0200 | Cezary Kaliszyk | alpha_alphabn for bindings in a type under bn. | changeset | files | 
| Mon, 17 May 2010 16:25:45 +0100 | Christian Urban | minor tuning | changeset | files | 
| Mon, 17 May 2010 16:29:33 +0200 | Cezary Kaliszyk | Ex4 does work, and I don't see the difference between the alphas. | changeset | files | 
| Mon, 17 May 2010 12:46:51 +0100 | Christian Urban | slight tuning | changeset | files | 
| 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 | changeset | files | 
| 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 | changeset | files | 
| Sun, 16 May 2010 11:00:44 +0100 | Christian Urban | tuned paper | changeset | files | 
| Sat, 15 May 2010 22:06:06 +0100 | Christian Urban | tuned paper | changeset | files | 
| Fri, 14 May 2010 21:18:34 +0100 | Christian Urban | tuned a bit the paper | changeset | files | 
| Fri, 14 May 2010 18:12:07 +0100 | Christian Urban | started a new file for the parser to make some experiments | changeset | files | 
| Fri, 14 May 2010 17:58:26 +0100 | Christian Urban | moved old parser and fv into attic | changeset | files | 
| Fri, 14 May 2010 17:40:43 +0100 | Christian Urban | polished example | changeset | files | 
| Fri, 14 May 2010 15:21:05 +0100 | Christian Urban | merged | changeset | files | 
| Fri, 14 May 2010 15:02:25 +0100 | Christian Urban | tuned a bit the paper | changeset | files | 
| Fri, 14 May 2010 15:37:23 +0200 | Cezary Kaliszyk | Proper fv/alpha for multiple compound binders | changeset | files | 
| Fri, 14 May 2010 10:28:42 +0200 | Cezary Kaliszyk | SingleLetFoo with everything. | changeset | files | 
| Fri, 14 May 2010 10:21:14 +0200 | Cezary Kaliszyk | Fv for multiple binding functions | changeset | files | 
| Thu, 13 May 2010 19:06:54 +0100 | Christian Urban | added a more instructive example - has some problems with fv though | changeset | files | 
| Thu, 13 May 2010 18:19:48 +0100 | Christian Urban | added flip_eqvt and swap_eqvt to the equivariance lists | changeset | files | 
| Thu, 13 May 2010 17:41:28 +0100 | Christian Urban | tuned the paper | changeset | files | 
| Thu, 13 May 2010 16:09:34 +0100 | Christian Urban | properly declared outer keyword | changeset | files | 
| Thu, 13 May 2010 15:58:36 +0100 | Christian Urban | added an example which goes outside our current speciifcation | changeset | files | 
| 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 | changeset | files | 
| Thu, 13 May 2010 15:12:34 +0100 | Christian Urban | tuned eqvt-proofs about prod_rel and prod_fv | changeset | files | 
| Thu, 13 May 2010 15:12:05 +0100 | Christian Urban | removed internal functions from the signature (they are not needed anymore) | changeset | files | 
| Thu, 13 May 2010 10:34:59 +0100 | Christian Urban | added term4 back to the examples | changeset | files | 
| Thu, 13 May 2010 07:41:18 +0200 | Cezary Kaliszyk | Make Term4 use 'equivariance'. | changeset | files | 
| Wed, 12 May 2010 16:59:53 +0100 | Christian Urban | fixed the examples for the new eqvt-procedure....temporarily disabled Manual/Term4.thy | changeset | files | 
| Wed, 12 May 2010 16:33:50 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 12 May 2010 16:33:25 +0100 | Christian Urban | moved the data-transformation into the parser | changeset | files | 
| Wed, 12 May 2010 16:26:06 +0100 | Christian Urban | added a test whether some of the constants already equivariant (then the procedure has to fail). | changeset | files | 
| Wed, 12 May 2010 16:57:01 +0200 | Cezary Kaliszyk | include set_simps and append_simps in fv_rsp | changeset | files | 
| Wed, 12 May 2010 16:39:10 +0200 | Cezary Kaliszyk | Move alpha_eqvt to unused. | changeset | files | 
| Wed, 12 May 2010 16:32:44 +0200 | Cezary Kaliszyk | Use equivariance instead of alpha_eqvt | changeset | files | 
| Wed, 12 May 2010 16:18:04 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 12 May 2010 16:11:23 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 12 May 2010 16:11:03 +0200 | Cezary Kaliszyk | fvbv_rsp include prod_rel.simps | changeset | files | 
| Wed, 12 May 2010 15:17:35 +0100 | Christian Urban | better ML-interface (returning only a list of theorems and a context) | changeset | files | 
| Wed, 12 May 2010 16:09:38 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 12 May 2010 16:08:32 +0200 | Cezary Kaliszyk | Use raw_induct instead of induct | changeset | files | 
| Wed, 12 May 2010 14:47:52 +0100 | Christian Urban | ingnored parameters in equivariance; added a proper interface to be called from ML | changeset | files | 
| Wed, 12 May 2010 13:43:48 +0100 | Christian Urban | properly exported defined bn-functions | changeset | files | 
| Tue, 11 May 2010 18:20:25 +0200 | Cezary Kaliszyk | Include raw permutation definitions in eqvt | changeset | files | 
| Tue, 11 May 2010 17:16:57 +0200 | Cezary Kaliszyk | Declare alpha_gen_eqvt as eqvt and change the proofs that used 'eqvts[symmetric]' | changeset | files | 
| Tue, 11 May 2010 14:58:46 +0100 | Christian Urban | a bit for the introduction of the q-paper | changeset | files | 
| Tue, 11 May 2010 12:18:26 +0100 | Christian Urban | added some of the quotient literature; a bit more to the qpaper | changeset | files | 
| Mon, 10 May 2010 18:09:00 +0100 | Christian Urban | fixed a problem with non-existant alphas2 | changeset | files | 
| Mon, 10 May 2010 17:57:22 +0100 | Christian Urban | added comment about bind_set | changeset | files | 
| Mon, 10 May 2010 17:55:54 +0100 | Christian Urban | fixing bind_set problem | changeset | files | 
| Mon, 10 May 2010 18:32:50 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 10 May 2010 18:32:15 +0200 | Cezary Kaliszyk | Term8 comment | changeset | files | 
| Mon, 10 May 2010 18:30:27 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 10 May 2010 18:29:45 +0200 | Cezary Kaliszyk | Restore set bindings in CoreHaskell | changeset | files | 
| Mon, 10 May 2010 15:54:16 +0200 | Cezary Kaliszyk | Recursive examples with relation composition | changeset | files | 
| Mon, 10 May 2010 15:45:04 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 10 May 2010 15:44:49 +0200 | Cezary Kaliszyk | prod_rel and prod_fv eqvt and mono | changeset | files | 
| Mon, 10 May 2010 15:14:02 +0200 | Cezary Kaliszyk | ExLetRec | changeset | files | 
| Mon, 10 May 2010 15:11:19 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 10 May 2010 15:11:05 +0200 | Cezary Kaliszyk | Parser changes for compound relations | changeset | files | 
| Mon, 10 May 2010 15:09:53 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 10 May 2010 15:09:32 +0200 | Cezary Kaliszyk | Use mk_compound_fv' and mk_compound_rel' | changeset | files | 
| Mon, 10 May 2010 12:05:13 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 10 May 2010 12:04:40 +0200 | Cezary Kaliszyk | Membership in a pair of lists. | changeset | files | 
| Mon, 10 May 2010 10:22:57 +0200 | Cezary Kaliszyk | Synchronize FSet with repository | changeset | files | 
| Sun, 09 May 2010 12:38:59 +0100 | Christian Urban | tuned file names for examples | changeset | files | 
| Sun, 09 May 2010 12:26:10 +0100 | Christian Urban | cleaned up a bit the examples; added equivariance to all examples | changeset | files | 
| Sun, 09 May 2010 11:43:24 +0100 | Christian Urban | fixed the problem with alpha containing splits | changeset | files | 
| Sun, 09 May 2010 11:37:19 +0100 | Christian Urban | added eqvt-lemma for split; changed semantics of perm_simp: excluded stands for constants about which no complaint is written out...eqvt_apply is now always applied | changeset | files | 
| Fri, 07 May 2010 12:28:11 +0200 | Cezary Kaliszyk | Manually added some newer keywords from the distribution | changeset | files | 
| Fri, 07 May 2010 12:10:04 +0200 | Cezary Kaliszyk | Regularize experiments | changeset | files | 
| Thu, 06 May 2010 14:21:10 +0200 | Cezary Kaliszyk | alpha_eqvt_tac with prod_rel and prod_fv simps | changeset | files | 
| Thu, 06 May 2010 14:14:30 +0200 | Cezary Kaliszyk | mem => member | changeset | files | 
| Thu, 06 May 2010 14:13:45 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Thu, 06 May 2010 14:13:35 +0200 | Cezary Kaliszyk | Fixes for new Isabelle | changeset | files | 
| Thu, 06 May 2010 14:13:05 +0200 | Cezary Kaliszyk | compound versions with prod_rel and prod_fun, not made default yet. | changeset | files | 
| Thu, 06 May 2010 14:10:56 +0200 | Cezary Kaliszyk | prod_rel and prod_fv simps | changeset | files | 
| Thu, 06 May 2010 14:10:26 +0200 | Cezary Kaliszyk | mem => member | changeset | files | 
| Thu, 06 May 2010 14:09:56 +0200 | Cezary Kaliszyk | prod_rel.simps and Fixed for new isabelle | changeset | files | 
| Thu, 06 May 2010 14:09:21 +0200 | Cezary Kaliszyk | Fixes for new isabelle | changeset | files | 
| Thu, 06 May 2010 13:25:37 +0200 | Cezary Kaliszyk | prod_fv and its respectfullness and preservation. | changeset | files | 
| Thu, 06 May 2010 10:43:41 +0200 | Cezary Kaliszyk | Experiments with equivariance. | changeset | files | 
| Wed, 05 May 2010 20:39:56 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 05 May 2010 20:39:21 +0100 | Christian Urban | a bit mor on the pearl journal paper | changeset | files | 
| Wed, 05 May 2010 10:24:54 +0100 | Christian Urban | solved the problem with equivariance by first eta-normalising the goal | changeset | files | 
| Wed, 05 May 2010 09:23:10 +0200 | Cezary Kaliszyk | Some cleaning in Term4 | changeset | files | 
| Tue, 04 May 2010 17:25:58 +0200 | Cezary Kaliszyk | "isabelle make" compiles all examples with newparser/newfv/newalpha only. | changeset | files | 
| Tue, 04 May 2010 17:15:21 +0200 | Cezary Kaliszyk | Move Term4 to NewParser | changeset | files | 
| Tue, 04 May 2010 16:59:31 +0200 | Cezary Kaliszyk | Fix Term4 for permutation signature change | changeset | files | 
| Tue, 04 May 2010 16:44:12 +0200 | Cezary Kaliszyk | Move LF to NewParser. Just works. | changeset | files | 
| Tue, 04 May 2010 16:42:36 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 04 May 2010 16:42:28 +0200 | Cezary Kaliszyk | ExLetMult | changeset | files | 
| Tue, 04 May 2010 16:39:12 +0200 | Cezary Kaliszyk | Ex1Rec. | changeset | files | 
| Tue, 04 May 2010 16:33:38 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 04 May 2010 16:33:30 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 04 May 2010 16:29:11 +0200 | Cezary Kaliszyk | ExPS3 in NewParser | changeset | files | 
| Tue, 04 May 2010 16:22:21 +0200 | Cezary Kaliszyk | Move ExPS8 to new parser. | changeset | files | 
| Tue, 04 May 2010 16:30:31 +0200 | Cezary Kaliszyk | Fix for new isabelle | changeset | files | 
| Tue, 04 May 2010 16:18:07 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 04 May 2010 16:17:46 +0200 | Cezary Kaliszyk | Minor | changeset | files | 
| Tue, 04 May 2010 14:38:07 +0100 | Christian Urban | increased step counter so that all steps go through | changeset | files | 
| Tue, 04 May 2010 14:33:50 +0100 | Christian Urban | fixed my error with define_raw_fv | changeset | files | 
| 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 | changeset | files | 
| Tue, 04 May 2010 14:21:18 +0200 | Cezary Kaliszyk | Separate Term8, as it may work soon. | changeset | files | 
| Tue, 04 May 2010 14:13:18 +0200 | Cezary Kaliszyk | moved CoreHaskell to NewParser. | changeset | files | 
| Tue, 04 May 2010 13:52:40 +0200 | Cezary Kaliszyk | ExPS7 in NewParser | changeset | files | 
| Tue, 04 May 2010 12:34:33 +0200 | Cezary Kaliszyk | Move ExLeroy to New Parser | changeset | files | 
| Tue, 04 May 2010 11:22:22 +0200 | Cezary Kaliszyk | Move 2 more to NewParser | changeset | files | 
| Tue, 04 May 2010 11:12:09 +0200 | Cezary Kaliszyk | Move TypeSchemes to NewParser | changeset | files | 
| Tue, 04 May 2010 11:08:30 +0200 | Cezary Kaliszyk | Move ExLet to NewParser. | changeset | files | 
| Tue, 04 May 2010 07:22:33 +0100 | Christian Urban | tuned | changeset | files | 
| Tue, 04 May 2010 06:24:54 +0100 | Christian Urban | roll back of the last commit (there was a difference) | changeset | files | 
| Tue, 04 May 2010 06:05:13 +0100 | Christian Urban | tuned | changeset | files | 
| 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 | changeset | files | 
| Tue, 04 May 2010 05:36:55 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 04 May 2010 05:36:43 +0100 | Christian Urban | some preliminary changes to the pearl-jv paper | changeset | files | 
| Mon, 03 May 2010 08:52:15 +0100 | Christian Urban | some preliminary notes of the abstract (qpaper); still need to see the motivating example | changeset | files | 
| Mon, 03 May 2010 15:47:30 +0200 | Cezary Kaliszyk | Added cheats to classical | changeset | files | 
| Mon, 03 May 2010 15:38:20 +0200 | Cezary Kaliszyk | Ex2 moved to new parser. | changeset | files | 
| Mon, 03 May 2010 15:37:21 +0200 | Cezary Kaliszyk | alpha_eqvt_tac fixed to work when the existential is not at the top level. | changeset | files | 
| Mon, 03 May 2010 15:36:47 +0200 | Cezary Kaliszyk | SingleLet and Ex3 work with NewParser. | changeset | files | 
| Mon, 03 May 2010 15:13:15 +0200 | Cezary Kaliszyk | Comment | changeset | files | 
| Mon, 03 May 2010 14:31:11 +0200 | Cezary Kaliszyk | Another example where only alpha_eqvt fails. | changeset | files | 
| Mon, 03 May 2010 14:30:37 +0200 | Cezary Kaliszyk | Register only non-looping rules in eq_iff | changeset | files | 
| Mon, 03 May 2010 14:03:30 +0200 | Cezary Kaliszyk | Equivariance fails for single let? | changeset | files | 
| Mon, 03 May 2010 13:42:44 +0200 | Cezary Kaliszyk | NewParser | changeset | files | 
| Mon, 03 May 2010 12:24:27 +0200 | Cezary Kaliszyk | Introduce eq_iff_simp to match the one from Parser. | changeset | files | 
| Mon, 03 May 2010 11:43:27 +0200 | Cezary Kaliszyk | remove tracing | changeset | files | 
| Mon, 03 May 2010 11:43:08 +0200 | Cezary Kaliszyk | Cheat support equations in new parser | changeset | files | 
| Mon, 03 May 2010 11:37:44 +0200 | Cezary Kaliszyk | Remove dependency on NewFv | changeset | files | 
| Mon, 03 May 2010 11:35:38 +0200 | Cezary Kaliszyk | Fix Parser | changeset | files | 
| Mon, 03 May 2010 10:15:23 +0200 | Cezary Kaliszyk | Add explicit cheats in NewParser and comment out the examples for outside use. | changeset | files | 
| Mon, 03 May 2010 09:57:05 +0200 | Cezary Kaliszyk | Fix Datatype_Aux calls in NewParser. | changeset | files | 
| Mon, 03 May 2010 09:55:43 +0200 | Cezary Kaliszyk | Move old fv_alpha_export to Fv. | changeset | files | 
| Mon, 03 May 2010 00:01:12 +0100 | Christian Urban | moved old parser and old fv back into their original places; isabelle make works again | changeset | files | 
| Mon, 03 May 2010 00:00:33 +0100 | Christian Urban | slight tuning | changeset | files | 
| Sun, 02 May 2010 21:15:52 +0100 | Christian Urban | simplified the supp-of-finite-sets proof | changeset | files | 
| Sun, 02 May 2010 16:02:27 +0100 | Christian Urban | tried to add some comments in the huge(!) nominal2_cmd function | changeset | files | 
| Sun, 02 May 2010 16:01:45 +0100 | Christian Urban | replaced make_pair with library function HOLogic.mk_prod | changeset | files | 
| Sun, 02 May 2010 16:00:52 +0100 | Christian Urban | removed duplicate eqvt attribute | changeset | files | 
| 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) | changeset | files | 
| Sat, 01 May 2010 09:15:46 +0100 | Christian Urban | merged | changeset | files | 
| Sat, 01 May 2010 09:14:25 +0100 | Christian Urban | tuned | changeset | files | 
| Fri, 30 Apr 2010 16:31:43 +0100 | Christian Urban | replaced hide by the new hide_const | changeset | files | 
| Fri, 30 Apr 2010 15:36:02 +0100 | Christian Urban | generalised the fs-instance lemma (not just fsets of atoms are finitely supported, but also fsets of finitely supported elements) | changeset | files | 
| Fri, 30 Apr 2010 15:34:26 +0100 | Christian Urban | added lemmas establishing the support of finite sets of finitely supported elements | changeset | files | 
| Fri, 30 Apr 2010 14:21:18 +0100 | Christian Urban | added eqvt-lemmas for Bex, Ball and Union | changeset | files | 
| 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. | changeset | files | 
| Fri, 30 Apr 2010 14:48:13 +0200 | Cezary Kaliszyk | Merged nominal_datatype into NewParser until eqvts | changeset | files | 
| Fri, 30 Apr 2010 13:57:59 +0200 | Cezary Kaliszyk | more parser/new parser synchronization. | changeset | files | 
| Fri, 30 Apr 2010 10:48:48 +0200 | Cezary Kaliszyk | Simplify old parser for integration | changeset | files | 
| Fri, 30 Apr 2010 10:32:34 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Fri, 30 Apr 2010 10:31:32 +0200 | Cezary Kaliszyk | Change signature of fv and alpha generation. | changeset | files | 
| Fri, 30 Apr 2010 10:09:45 +0100 | Christian Urban | reorganised eqvt-file (now uses perm_simp already) | changeset | files | 
| Fri, 30 Apr 2010 10:04:24 +0200 | Cezary Kaliszyk | qpaper | changeset | files | 
| Thu, 29 Apr 2010 17:52:33 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Thu, 29 Apr 2010 17:52:19 +0200 | Cezary Kaliszyk | New Alpha. | changeset | files | 
| Thu, 29 Apr 2010 17:16:35 +0200 | Cezary Kaliszyk | Minimal cleaning in LamEx | changeset | files | 
| Thu, 29 Apr 2010 17:03:59 +0200 | Cezary Kaliszyk | Remove things moved to the isabelle distribution | changeset | files | 
| Thu, 29 Apr 2010 16:59:33 +0200 | Cezary Kaliszyk | Unify and give only one name to 'setify', 'listify' and 'set' | changeset | files | 
| Thu, 29 Apr 2010 16:18:38 +0200 | Cezary Kaliszyk | Fixing the definitions in the Parser. | changeset | files | 
| Thu, 29 Apr 2010 16:16:45 +0200 | Cezary Kaliszyk | Some of the exceptions that the parser should check in TODO. | changeset | files | 
| Thu, 29 Apr 2010 16:15:49 +0200 | Cezary Kaliszyk | Extracting the fv body function and exporting the terms. | changeset | files | 
| Thu, 29 Apr 2010 13:19:12 +0200 | Cezary Kaliszyk | Fix for recursive binders. | changeset | files | 
| Thu, 29 Apr 2010 12:11:44 +0200 | Cezary Kaliszyk | revert 0c9ef14e9ba4 | changeset | files | 
| Thu, 29 Apr 2010 11:54:39 +0200 | Cezary Kaliszyk | Support in positive position and atoms in negative positions. | changeset | files | 
| Thu, 29 Apr 2010 11:00:18 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Thu, 29 Apr 2010 10:59:08 +0200 | Cezary Kaliszyk | Include support of unknown datatypes in new fv | changeset | files | 
| Thu, 29 Apr 2010 10:16:33 +0200 | Christian Urban | merged | changeset | files | 
| Thu, 29 Apr 2010 10:16:15 +0200 | Christian Urban | added basic functions for constructing supp-terms | changeset | files | 
| Thu, 29 Apr 2010 10:11:48 +0200 | Cezary Kaliszyk | quotient paper | changeset | files | 
| Thu, 29 Apr 2010 09:25:32 +0200 | Christian Urban | added missing latex-style file | changeset | files | 
| Thu, 29 Apr 2010 09:14:16 +0200 | Christian Urban | merged | changeset | files | 
| Thu, 29 Apr 2010 09:13:18 +0200 | Christian Urban | added stub for quotient paper; call with isabelle make qpaper | changeset | files | 
| Wed, 28 Apr 2010 17:05:20 +0200 | Cezary Kaliszyk | Cleaning of Int and FSet Examples | changeset | files | 
| Wed, 28 Apr 2010 08:32:33 +0200 | Christian Urban | use the more general type-class at_base | changeset | files | 
| Wed, 28 Apr 2010 08:24:46 +0200 | Christian Urban | deleted left-over code | changeset | files | 
| Wed, 28 Apr 2010 08:22:20 +0200 | Christian Urban | simpliied and moved the remaining lemmas about the atom-function to Nominal2_Base | changeset | files | 
| Wed, 28 Apr 2010 07:27:28 +0200 | Christian Urban | use sort at_base instead of at | changeset | files | 
| Wed, 28 Apr 2010 07:20:57 +0200 | Christian Urban | white spaces | changeset | files | 
| Wed, 28 Apr 2010 07:09:11 +0200 | Christian Urban | avoided repeated dest of dt_info | changeset | files | 
| Wed, 28 Apr 2010 06:55:07 +0200 | Christian Urban | tuned | changeset | files | 
| Wed, 28 Apr 2010 06:40:10 +0200 | Christian Urban | factured out common functionality of prefixing the dt-names with a string | changeset | files | 
| Wed, 28 Apr 2010 06:24:10 +0200 | Christian Urban | closed Datatype_Aux; replaced nth_dtyp by the function used in Perm.thy | changeset | files | 
| Tue, 27 Apr 2010 23:11:40 +0200 | Christian Urban | added some further problemetic tests | changeset | files | 
| Tue, 27 Apr 2010 22:45:50 +0200 | Christian Urban | some tuning | changeset | files | 
| Tue, 27 Apr 2010 22:21:16 +0200 | Christian Urban | moved mk_atom into the library; that meant that concrete atom classes need to be in Nominal2_Base | changeset | files | 
| Tue, 27 Apr 2010 19:51:35 +0200 | Christian Urban | merged | changeset | files | 
| Tue, 27 Apr 2010 19:01:22 +0200 | Cezary Kaliszyk | Rewrote FV code and included the function package. | changeset | files | 
| Tue, 27 Apr 2010 14:30:44 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 27 Apr 2010 14:29:59 +0200 | Cezary Kaliszyk | Function in Core Haskell | changeset | files | 
| Tue, 27 Apr 2010 13:44:27 +0200 | Christian Urban | one more pass over the paper | changeset | files | 
| Tue, 27 Apr 2010 12:23:06 +0200 | Christian Urban | more polishing on the paper | changeset | files | 
| Mon, 26 Apr 2010 20:19:42 +0200 | Christian Urban | merged | changeset | files | 
| Mon, 26 Apr 2010 20:17:41 +0200 | Christian Urban | some changes to the paper | changeset | files | 
| Mon, 26 Apr 2010 13:08:14 +0200 | Christian Urban | rewrote eqvts_raw to be a symtab, that can be looked up | changeset | files | 
| Mon, 26 Apr 2010 10:01:13 +0200 | Cezary Kaliszyk | merge ??? | changeset | files | 
| Wed, 21 Apr 2010 12:25:52 +0200 | Cezary Kaliszyk | infix for In | changeset | files | 
| Mon, 26 Apr 2010 08:19:11 +0200 | Christian Urban | eliminated command so that all compiles | changeset | files | 
| Mon, 26 Apr 2010 08:08:20 +0200 | Christian Urban | changed theorem_i to theorem....requires new Isabelle | changeset | files | 
| Sun, 25 Apr 2010 09:26:36 +0200 | Christian Urban | tuned | changeset | files | 
| Sun, 25 Apr 2010 09:13:16 +0200 | Christian Urban | tuned and cleaned | changeset | files | 
| Sun, 25 Apr 2010 08:18:06 +0200 | Christian Urban | tuned and made to compile | changeset | files | 
| Sun, 25 Apr 2010 08:06:43 +0200 | Christian Urban | added definition of raw-permutations to the new-parser | changeset | files | 
| Sun, 25 Apr 2010 07:54:28 +0200 | Christian Urban | tuned | changeset | files | 
| Sun, 25 Apr 2010 01:31:22 +0200 | Christian Urban | slight tuning | changeset | files | 
| Sat, 24 Apr 2010 10:00:33 +0200 | Christian Urban | added a comment about a function where I am not sure who wrote it. | changeset | files | 
| Sat, 24 Apr 2010 09:49:23 +0200 | Christian Urban | merged | changeset | files | 
| Fri, 23 Apr 2010 11:12:38 +0200 | Cezary Kaliszyk | Minor | changeset | files | 
| Fri, 23 Apr 2010 10:21:34 +0200 | Cezary Kaliszyk | Minor cleaning of IntEx | changeset | files | 
| Fri, 23 Apr 2010 09:54:42 +0200 | Cezary Kaliszyk | Further cleaning of proofs in FSet | changeset | files | 
| Thu, 22 Apr 2010 17:27:24 +0200 | Cezary Kaliszyk | Update term8 | changeset | files | 
| Thu, 22 Apr 2010 12:42:15 +0200 | Cezary Kaliszyk | Converted 'thm' to a lemma. | changeset | files | 
| Thu, 22 Apr 2010 12:33:51 +0200 | Cezary Kaliszyk | Moved working Fset3 properties to FSet. | changeset | files | 
| Thu, 22 Apr 2010 06:44:24 +0200 | Christian Urban | tuned parser | changeset | files | 
| Thu, 22 Apr 2010 05:16:23 +0200 | Christian Urban | moved lemmas from FSet.thy to do with atom to Nominal2_Base, and to do with 'a::at set to Nominal2_Atoms; moved Nominal2_Eqvt.thy one up to be loaded before Nominal2_Atoms | changeset | files | 
| Wed, 21 Apr 2010 21:52:30 +0200 | Christian Urban | tuned proofs | changeset | files | 
| Wed, 21 Apr 2010 21:31:07 +0200 | Christian Urban | merged | changeset | files | 
| Wed, 21 Apr 2010 21:29:09 +0200 | Christian Urban | moved some lemmas into the right places | changeset | files | 
| Wed, 21 Apr 2010 20:01:18 +0200 | Cezary Kaliszyk | minor | changeset | files | 
| Wed, 21 Apr 2010 19:11:51 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 21 Apr 2010 19:10:55 +0200 | Cezary Kaliszyk | append_rsp2 + isarification | changeset | files | 
| Wed, 21 Apr 2010 17:42:57 +0200 | Christian Urban | some small changes | changeset | files | 
| Wed, 21 Apr 2010 16:25:24 +0200 | Christian Urban | merged | changeset | files | 
| Wed, 21 Apr 2010 16:25:00 +0200 | Christian Urban | deleted the incomplete proof about pairs of abstractions | changeset | files | 
| Wed, 21 Apr 2010 16:24:18 +0200 | Christian Urban | added a variant of the induction principle for permutations | changeset | files | 
| Wed, 21 Apr 2010 13:39:34 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 21 Apr 2010 13:38:37 +0200 | Cezary Kaliszyk | More about concat | changeset | files | 
| Wed, 21 Apr 2010 12:38:20 +0200 | Christian Urban | merged | changeset | files | 
| Wed, 21 Apr 2010 12:37:44 +0200 | Christian Urban | incomplete tests | changeset | files | 
| Wed, 21 Apr 2010 12:37:19 +0200 | Christian Urban | added an improved version of the induction principle for permutations | changeset | files | 
| Wed, 21 Apr 2010 10:34:10 +0200 | Cezary Kaliszyk | Working lifting of concat with inline proofs of second level preservation. | changeset | files | 
| Wed, 21 Apr 2010 10:24:39 +0200 | Cezary Kaliszyk | FSet3 cleaning part2 | changeset | files | 
| Wed, 21 Apr 2010 10:20:48 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 21 Apr 2010 10:13:17 +0200 | Cezary Kaliszyk | Remove the part already in FSet and leave the experiments | changeset | files | 
| Wed, 21 Apr 2010 10:09:07 +0200 | Christian Urban | merged | changeset | files | 
| Wed, 21 Apr 2010 10:08:47 +0200 | Christian Urban | removed a sorry | changeset | files | 
| Tue, 20 Apr 2010 18:24:50 +0200 | Christian Urban | renamed Ex1.thy to SingleLet.thy | changeset | files | 
| Tue, 20 Apr 2010 11:29:00 +0200 | Christian Urban | tuning of the code | changeset | files | 
| Wed, 21 Apr 2010 09:48:35 +0200 | Cezary Kaliszyk | Reorder FSet | changeset | files | 
| Wed, 21 Apr 2010 09:13:55 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 21 Apr 2010 09:13:32 +0200 | Cezary Kaliszyk | lattice properties. | changeset | files | 
| Tue, 20 Apr 2010 17:25:31 +0200 | Cezary Kaliszyk | All lifted in Term4. Requires new isabelle. | changeset | files | 
| Tue, 20 Apr 2010 15:59:57 +0200 | Cezary Kaliszyk | fsets are distributive lattices. | changeset | files | 
| Tue, 20 Apr 2010 10:23:39 +0200 | Cezary Kaliszyk | Fix of comment | changeset | files | 
| Tue, 20 Apr 2010 09:13:52 +0200 | Christian Urban | reordered code | changeset | files | 
| Tue, 20 Apr 2010 09:02:22 +0200 | Christian Urban | renamed "_empty" and "_append" to "_zero" and "_plus" | changeset | files | 
| Tue, 20 Apr 2010 08:57:13 +0200 | Christian Urban | removed dead code (nominal cannot deal with argument types of constructors that are functions) | changeset | files | 
| Tue, 20 Apr 2010 08:45:53 +0200 | Christian Urban | added comment about abstraction in raw permuations | changeset | files | 
| Tue, 20 Apr 2010 07:44:47 +0200 | Christian Urban | optimised the code of define_raw_perm | changeset | files | 
| Mon, 19 Apr 2010 17:26:07 +0200 | Christian Urban | deleting function perm_arg in favour of the library function mk_perm | changeset | files | 
| Mon, 19 Apr 2010 16:55:57 +0200 | Christian Urban | merged | changeset | files | 
| Mon, 19 Apr 2010 16:55:36 +0200 | Christian Urban | tuned; fleshed out some library functions about permutations; closed Datatype_Aux structure (increases readability) | changeset | files | 
| Mon, 19 Apr 2010 16:19:17 +0200 | Cezary Kaliszyk | FSet is a semi-lattice | changeset | files | 
| Mon, 19 Apr 2010 15:54:55 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 19 Apr 2010 15:54:38 +0200 | Cezary Kaliszyk | Putting FSet in bot typeclass. | changeset | files | 
| Mon, 19 Apr 2010 15:33:19 +0200 | Cezary Kaliszyk | reorder | changeset | files | 
| Mon, 19 Apr 2010 15:37:54 +0200 | Christian Urban | merged | changeset | files | 
| Mon, 19 Apr 2010 15:37:33 +0200 | Christian Urban | small updates to the paper; remaining points in PAPER-TODO | changeset | files | 
| Mon, 19 Apr 2010 15:28:57 +0200 | Cezary Kaliszyk | sub_list definition and respects | changeset | files | 
| Mon, 19 Apr 2010 15:08:29 +0200 | Cezary Kaliszyk | Alternate list_eq and equivalence | changeset | files | 
| Mon, 19 Apr 2010 14:08:01 +0200 | Cezary Kaliszyk | Some new lemmas | changeset | files | 
| Mon, 19 Apr 2010 13:58:10 +0200 | Cezary Kaliszyk | More cleaning | changeset | files | 
| Mon, 19 Apr 2010 12:28:48 +0200 | Cezary Kaliszyk | remove more metis | changeset | files | 
| Mon, 19 Apr 2010 12:20:18 +0200 | Cezary Kaliszyk | more metis cleaning | changeset | files | 
| Mon, 19 Apr 2010 11:55:12 +0200 | Cezary Kaliszyk | Getting rid of 'metis'. | changeset | files | 
| Mon, 19 Apr 2010 11:38:43 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 19 Apr 2010 11:32:33 +0200 | Cezary Kaliszyk | Remove 'defer'. | changeset | files | 
| Mon, 19 Apr 2010 09:27:53 +0200 | Christian Urban | merged | changeset | files | 
| Mon, 19 Apr 2010 09:25:31 +0200 | Christian Urban | tuned proofs | changeset | files | 
| Mon, 19 Apr 2010 11:04:31 +0200 | Cezary Kaliszyk | 2 more lifted lemmas needed for second representation | changeset | files | 
| Mon, 19 Apr 2010 10:35:08 +0200 | Cezary Kaliszyk | Accept non-equality eqvt rules in support proofs. | changeset | files | 
| Mon, 19 Apr 2010 10:00:52 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 19 Apr 2010 09:59:32 +0200 | Cezary Kaliszyk | Locations of files in Parser | changeset | files | 
| Mon, 19 Apr 2010 09:25:55 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 19 Apr 2010 09:25:43 +0200 | Cezary Kaliszyk | minor FSet3 edits. | changeset | files | 
| Sun, 18 Apr 2010 18:01:22 +0200 | Christian Urban | tuned | changeset | files | 
| Sun, 18 Apr 2010 17:58:45 +0200 | Christian Urban | moved some general function into nominal_library.ML | changeset | files | 
| Sun, 18 Apr 2010 17:57:27 +0200 | Christian Urban | tuned; transformation functions now take a context, a thm and return a thm | changeset | files | 
| Sun, 18 Apr 2010 17:56:05 +0200 | Christian Urban | tuned | changeset | files | 
| Sun, 18 Apr 2010 10:58:29 +0200 | Christian Urban | equivariance for alpha_raw in CoreHaskell is automatically derived | changeset | files | 
| Sun, 18 Apr 2010 09:26:38 +0200 | Christian Urban | preliminary parser for perm_simp metod | changeset | files | 
| Fri, 16 Apr 2010 16:29:11 +0200 | Christian Urban | automatic proofs for equivariance of alphas | changeset | files | 
| Fri, 16 Apr 2010 11:09:32 +0200 | Cezary Kaliszyk | Finished proof in Lambda.thy | changeset | files | 
| Fri, 16 Apr 2010 10:47:13 +0200 | Christian Urban | merged | changeset | files | 
| Fri, 16 Apr 2010 10:46:50 +0200 | Christian Urban | attempt to manual prove eqvt for alpha | changeset | files | 
| Fri, 16 Apr 2010 10:41:40 +0200 | Cezary Kaliszyk | Lifting in Term4. | changeset | files | 
| Fri, 16 Apr 2010 10:18:16 +0200 | Christian Urban | some tuning of eqvt-infrastructure | changeset | files | 
| Thu, 15 Apr 2010 21:56:03 +0200 | Christian Urban | some tuning of proofs | changeset | files | 
| Thu, 15 Apr 2010 16:01:28 +0200 | Christian Urban | typo | changeset | files | 
| Thu, 15 Apr 2010 15:56:38 +0200 | Christian Urban | merged | changeset | files | 
| Thu, 15 Apr 2010 15:56:21 +0200 | Christian Urban | half of the pair-abs-equivalence | changeset | files | 
| Thu, 15 Apr 2010 15:31:36 +0200 | Cezary Kaliszyk | More on Manual/Trm4 | changeset | files | 
| Thu, 15 Apr 2010 14:08:08 +0200 | Cezary Kaliszyk | alpha4_equivp and constant lifting. | changeset | files | 
| Thu, 15 Apr 2010 13:55:44 +0200 | Cezary Kaliszyk | alpha4_eqvt and alpha4_reflp | changeset | files | 
| Thu, 15 Apr 2010 12:27:36 +0200 | Cezary Kaliszyk | fv_eqvt in term4 | changeset | files | 
| Thu, 15 Apr 2010 12:15:38 +0200 | Cezary Kaliszyk | Updating in Term4. | changeset | files | 
| Thu, 15 Apr 2010 12:08:46 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Thu, 15 Apr 2010 11:42:28 +0200 | Cezary Kaliszyk | Prove insert_rsp2 | changeset | files | 
| Thu, 15 Apr 2010 12:07:54 +0200 | Christian Urban | merged | changeset | files | 
| Thu, 15 Apr 2010 12:07:34 +0200 | Christian Urban | changed header | changeset | files | 
| Thu, 15 Apr 2010 11:05:54 +0200 | Cezary Kaliszyk | Minor paper fixes. | changeset | files | 
| Wed, 14 Apr 2010 22:41:22 +0200 | Christian Urban | temporary fix for CoreHaskell | changeset | files | 
| 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 | changeset | files | 
| Wed, 14 Apr 2010 20:21:11 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 14 Apr 2010 20:20:54 +0200 | Cezary Kaliszyk | Fix the 'subscript' error. | changeset | files | 
| Wed, 14 Apr 2010 18:47:20 +0200 | Christian Urban | merged | changeset | files | 
| Wed, 14 Apr 2010 18:46:59 +0200 | Christian Urban | thmdecls can deal with lemmas like alpha_gen which contain pairs or tuples | changeset | files | 
| Wed, 14 Apr 2010 16:11:04 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 14 Apr 2010 16:10:44 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 14 Apr 2010 11:08:33 +0200 | Cezary Kaliszyk | Separate alpha_definition. | changeset | files | 
| Wed, 14 Apr 2010 11:07:42 +0200 | Cezary Kaliszyk | Fix spelling in theory header | changeset | files | 
| Wed, 14 Apr 2010 10:50:11 +0200 | Cezary Kaliszyk | Separate define_fv. | changeset | files | 
| Wed, 14 Apr 2010 16:05:58 +0200 | Christian Urban | tuned and removed dead code | changeset | files | 
| Wed, 14 Apr 2010 15:02:07 +0200 | Christian Urban | moved a couple of more functions to the library | changeset | files | 
| Wed, 14 Apr 2010 14:41:54 +0200 | Christian Urban | added a library for basic nominal functions; separated nominal_eqvt file | changeset | files | 
| Wed, 14 Apr 2010 13:21:38 +0200 | Christian Urban | merged | changeset | files | 
| Wed, 14 Apr 2010 13:21:11 +0200 | Christian Urban | first working version of the automatic equivariance procedure | changeset | files | 
| Wed, 14 Apr 2010 10:39:03 +0200 | Cezary Kaliszyk | Initial cleaning/reorganization in Fv. | changeset | files | 
| Wed, 14 Apr 2010 10:29:56 +0200 | Christian Urban | merged | changeset | files | 
| Wed, 14 Apr 2010 10:29:34 +0200 | Christian Urban | preliminary tests | changeset | files | 
| Wed, 14 Apr 2010 10:28:17 +0200 | Christian Urban | deleted test | changeset | files | 
| Wed, 14 Apr 2010 08:42:38 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 14 Apr 2010 08:36:54 +0200 | Cezary Kaliszyk | merge part: delete_rsp | changeset | files | 
| Wed, 14 Apr 2010 08:35:31 +0200 | Cezary Kaliszyk | merge part1: none_memb_nil | changeset | files | 
| Wed, 14 Apr 2010 08:16:54 +0200 | Christian Urban | added header and more tuning | changeset | files | 
| Wed, 14 Apr 2010 07:57:55 +0200 | Christian Urban | more tuning | changeset | files | 
| Wed, 14 Apr 2010 07:34:03 +0200 | Christian Urban | tuned | changeset | files | 
| Tue, 13 Apr 2010 15:59:53 +0200 | Cezary Kaliszyk | Working FSet with additional lemmas. | changeset | files | 
| Tue, 13 Apr 2010 15:00:49 +0200 | Cezary Kaliszyk | Much more in FSet (currently non-working) | changeset | files | 
| Tue, 13 Apr 2010 07:40:54 +0200 | Christian Urban | made everything to compile | changeset | files | 
| Tue, 13 Apr 2010 00:53:48 +0200 | Christian Urban | merged | changeset | files | 
| Tue, 13 Apr 2010 00:53:32 +0200 | Christian Urban | some small tunings (incompleted work in Lambda.thy) | changeset | files | 
| Tue, 13 Apr 2010 00:47:57 +0200 | Christian Urban | moved equivariance of map into Nominal2_Eqvt file | changeset | files | 
| Mon, 12 Apr 2010 17:44:26 +0200 | Christian Urban | early ott paper | changeset | files | 
| Mon, 12 Apr 2010 17:05:19 +0200 | Cezary Kaliszyk | Porting lemmas from Quotient package FSet to new FSet. | changeset | files | 
| Mon, 12 Apr 2010 14:31:23 +0200 | Christian Urban | added alpha-caml paper | changeset | files | 
| Mon, 12 Apr 2010 13:34:54 +0200 | Christian Urban | implemented in thmdecls the case where eqvt-lemmas are of the form _ ==> _ | changeset | files | 
| 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 _ ==> _ | changeset | files | 
| Sun, 11 Apr 2010 22:47:45 +0200 | Christian Urban | folded changes from the conference version | changeset | files | 
| Sun, 11 Apr 2010 22:01:56 +0200 | Christian Urban | added TODO item about parser creating syntax for the wrong type | changeset | files | 
| Sun, 11 Apr 2010 18:18:22 +0200 | Christian Urban | corrected imports header | changeset | files | 
| Sun, 11 Apr 2010 18:11:23 +0200 | Christian Urban | tuned | changeset | files | 
| Sun, 11 Apr 2010 18:11:13 +0200 | Christian Urban | a few tests | changeset | files | 
| Sun, 11 Apr 2010 18:10:08 +0200 | Christian Urban | added eqvt rules that are more standard | changeset | files | 
| Sun, 11 Apr 2010 18:08:57 +0200 | Christian Urban | used warning instead of tracing (does not seem to produce stable output) | changeset | files | 
| Sun, 11 Apr 2010 18:06:45 +0200 | Christian Urban | added small ittems about equivaraince of alpha_gens and name of lam.perm | changeset | files | 
| Sun, 11 Apr 2010 10:36:09 +0200 | Christian Urban | added more robust tracing infrastructure; a strict version of the eqvt_tac raises an error if not all permutations cannot be analysed | changeset | files | 
| 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 | changeset | files | 
| Fri, 09 Apr 2010 09:02:54 -0700 | Brian Huffman | rewrite paragraph introducing equivariance, add citation to Pitts03 | changeset | files | 
| Fri, 09 Apr 2010 08:16:08 -0700 | Brian Huffman | edit 'contributions' section so we do not just quote directly from the reviewer | changeset | files | 
| 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 | changeset | files | 
| Thu, 08 Apr 2010 14:18:38 +0200 | Christian Urban | clarified comment about distinct lists in th efuture work section | changeset | files | 
| Thu, 08 Apr 2010 13:04:49 +0200 | Christian Urban | tuned type-schemes example | changeset | files | 
| Thu, 08 Apr 2010 11:52:05 +0200 | Christian Urban | updated (comment about weirdo example) | changeset | files | 
| Thu, 08 Apr 2010 11:50:30 +0200 | Christian Urban | check whether the "weirdo" example from the binding bestiary works with shallow binders | changeset | files | 
| Thu, 08 Apr 2010 11:40:13 +0200 | Christian Urban | properly separated the example from my PhD and gave the correct alpha-equivalence relation (according to the paper) | changeset | files | 
| Thu, 08 Apr 2010 10:25:38 +0200 | Christian Urban | merged | changeset | files | 
| Thu, 08 Apr 2010 10:25:13 +0200 | Christian Urban | some further changes | changeset | files | 
| Thu, 08 Apr 2010 00:49:08 -0700 | Brian Huffman | merged | changeset | files | 
| Thu, 08 Apr 2010 00:47:13 -0700 | Brian Huffman | change some wording in conclusion | changeset | files | 
| Thu, 08 Apr 2010 00:25:08 -0700 | Brian Huffman | remove extra word | changeset | files | 
| Thu, 08 Apr 2010 09:13:36 +0200 | Christian Urban | merged | changeset | files | 
| Thu, 08 Apr 2010 09:12:13 +0200 | Christian Urban | added new paper directory for further work | changeset | files | 
| Thu, 08 Apr 2010 00:09:53 -0700 | Brian Huffman | use qualified name as string in concrete atom example | changeset | files | 
| Thu, 08 Apr 2010 00:01:45 -0700 | Brian Huffman | merged | changeset | files | 
| Thu, 08 Apr 2010 00:00:21 -0700 | Brian Huffman | simplify instance proof | changeset | files | 
| Wed, 07 Apr 2010 23:39:08 -0700 | Brian Huffman | polish explanation of additive group syntax | changeset | files | 
| Thu, 08 Apr 2010 08:40:49 +0200 | Christian Urban | final version of the pearl paper | changeset | files | 
| Wed, 07 Apr 2010 22:08:46 +0200 | Christian Urban | my final version of the paper | changeset | files | 
| Wed, 07 Apr 2010 17:37:29 +0200 | Christian Urban | added an induction principle for permutations; removed add_perm construction | changeset | files | 
| Tue, 06 Apr 2010 23:33:40 +0200 | Christian Urban | isarfied proof about existence of a permutation list | changeset | files | 
| Tue, 06 Apr 2010 14:08:06 +0200 | Christian Urban | added reference to E. Gunter's work | changeset | files | 
| Tue, 06 Apr 2010 07:36:15 +0200 | Christian Urban | typos in paper | changeset | files | 
| Sun, 04 Apr 2010 21:39:28 +0200 | Christian Urban | separated general nominal theory into separate folder | changeset | files | 
| Sat, 03 Apr 2010 22:31:11 +0200 | Christian Urban | added README and moved examples into separate directory | changeset | files | 
| Sat, 03 Apr 2010 21:53:04 +0200 | Christian Urban | merged pearl paper with this repository; started litrature subdirectory | changeset | files | 
| Fri, 02 Apr 2010 15:28:55 +0200 | Christian Urban | submitted version (just in time ;o) | changeset | files | 
| Fri, 02 Apr 2010 13:12:10 +0200 | Christian Urban | first complete version (slightly less than 3h more to go) | changeset | files | 
| Fri, 02 Apr 2010 07:59:03 +0200 | Christian Urban | tuned | changeset | files | 
| Fri, 02 Apr 2010 07:43:22 +0200 | Christian Urban | tuned strong ind section | changeset | files | 
| Fri, 02 Apr 2010 07:30:25 +0200 | Christian Urban | polished infrastruct section | changeset | files | 
| Fri, 02 Apr 2010 06:45:50 +0200 | Christian Urban | completed lifting section | changeset | files | 
| Fri, 02 Apr 2010 05:09:47 +0200 | Christian Urban | more on the lifting section | changeset | files | 
| Fri, 02 Apr 2010 03:23:25 +0200 | Christian Urban | more on the strong induction section | changeset | files | 
| Thu, 01 Apr 2010 18:45:50 +0200 | Christian Urban | completed conclusion | changeset | files | 
| Thu, 01 Apr 2010 17:56:39 +0200 | Christian Urban | merged | changeset | files | 
| Thu, 01 Apr 2010 17:56:26 +0200 | Christian Urban | merged | changeset | files | 
| Thu, 01 Apr 2010 17:55:46 +0200 | Christian Urban | updated related work section | changeset | files | 
| Thu, 01 Apr 2010 17:41:34 +0200 | Cezary Kaliszyk | fv_fv_bn | changeset | files | 
| Thu, 01 Apr 2010 17:00:52 +0200 | Cezary Kaliszyk | Update fv_bn definition for bindings allowed in types for which bn is present. | changeset | files | 
| Thu, 01 Apr 2010 16:55:34 +0200 | Cezary Kaliszyk | fv_perm_bn | changeset | files | 
| Thu, 01 Apr 2010 16:17:56 +0200 | Cezary Kaliszyk | Minor formula fixes. | changeset | files | 
| Thu, 01 Apr 2010 16:08:54 +0200 | Christian Urban | fixed alpha_bn | changeset | files | 
| Thu, 01 Apr 2010 15:41:48 +0200 | Christian Urban | current state | changeset | files | 
| Thu, 01 Apr 2010 14:53:14 +0200 | Christian Urban | merged | changeset | files | 
| Thu, 01 Apr 2010 14:49:01 +0200 | Christian Urban | added alpha_bn definition | changeset | files | 
| Thu, 01 Apr 2010 14:50:58 +0200 | Cezary Kaliszyk | hfill for right aligning single table cells. | changeset | files | 
| Thu, 01 Apr 2010 14:09:47 +0200 | Cezary Kaliszyk | Cleaning the strong induction example. | changeset | files | 
| Thu, 01 Apr 2010 12:19:26 +0200 | Cezary Kaliszyk | minor | changeset | files | 
| Thu, 01 Apr 2010 12:13:25 +0200 | Cezary Kaliszyk | Fighting with space in displaying strong induction... | changeset | files | 
| Thu, 01 Apr 2010 11:34:43 +0200 | Cezary Kaliszyk | starting strong induction | changeset | files | 
| Thu, 01 Apr 2010 10:57:49 +0200 | Cezary Kaliszyk | General paper minor fixes. | changeset | files | 
| Thu, 01 Apr 2010 09:28:03 +0200 | Cezary Kaliszyk | Forgot to save before commit. | changeset | files | 
| Thu, 01 Apr 2010 08:48:33 +0200 | Cezary Kaliszyk | Let with multiple bindings. | changeset | files | 
| Thu, 01 Apr 2010 08:06:01 +0200 | Cezary Kaliszyk | Fill the space below the figure. | changeset | files | 
| Thu, 01 Apr 2010 06:47:37 +0200 | Christian Urban | last commit for now. | changeset | files | 
| Thu, 01 Apr 2010 06:04:43 +0200 | Christian Urban | more on the conclusion | changeset | files | 
| Thu, 01 Apr 2010 05:40:12 +0200 | Christian Urban | completed related work section | changeset | files | 
| Thu, 01 Apr 2010 03:28:28 +0200 | Christian Urban | more on the paper | changeset | files | 
| Thu, 01 Apr 2010 01:05:05 +0200 | Christian Urban | added an item about alpha-equivalence (the existential should be closer to the abstraction) | changeset | files | 
| Wed, 31 Mar 2010 22:48:35 +0200 | Christian Urban | polished everything up to TODO | changeset | files | 
| Wed, 31 Mar 2010 18:47:22 +0200 | Christian Urban | merged | changeset | files | 
| Wed, 31 Mar 2010 18:47:02 +0200 | Christian Urban | added alpha-definition for ~~ty | changeset | files | 
| Wed, 31 Mar 2010 17:51:15 +0200 | Cezary Kaliszyk | permute_bn | changeset | files | 
| Wed, 31 Mar 2010 17:04:09 +0200 | Christian Urban | abbreviations for \<otimes> and \<oplus> | changeset | files | 
| Wed, 31 Mar 2010 16:27:57 +0200 | Christian Urban | merged | changeset | files | 
| Wed, 31 Mar 2010 16:27:44 +0200 | Christian Urban | a test with let having multiple bodies | changeset | files | 
| Wed, 31 Mar 2010 16:26:51 +0200 | Christian Urban | polished and removed tys from bn-functions. | changeset | files | 
| Wed, 31 Mar 2010 15:20:58 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 31 Mar 2010 12:30:17 +0200 | Cezary Kaliszyk | More on paper | changeset | files | 
| Wed, 31 Mar 2010 05:44:24 +0200 | Christian Urban | started to polish alpha-equivalence section, but needs more work | changeset | files | 
| Wed, 31 Mar 2010 02:59:18 +0200 | Christian Urban | started with a related work section | changeset | files | 
| Tue, 30 Mar 2010 22:31:15 +0200 | Christian Urban | polished and added an example for fvars | changeset | files | 
| Tue, 30 Mar 2010 21:15:13 +0200 | Christian Urban | cleaned up the section about fv's | changeset | files | 
| Tue, 30 Mar 2010 17:55:46 +0200 | Christian Urban | tuned beginning of section 4 | changeset | files | 
| Tue, 30 Mar 2010 17:52:16 +0200 | Cezary Kaliszyk | More on section 5. | changeset | files | 
| Tue, 30 Mar 2010 17:00:34 +0200 | Cezary Kaliszyk | More on section 5. | changeset | files | 
| Tue, 30 Mar 2010 16:59:23 +0200 | Christian Urban | merged | changeset | files | 
| Tue, 30 Mar 2010 16:59:00 +0200 | Christian Urban | removed "raw" distinction | changeset | files | 
| Tue, 30 Mar 2010 16:09:49 +0200 | Cezary Kaliszyk | More on Section 5 | changeset | files | 
| Tue, 30 Mar 2010 15:09:26 +0200 | Cezary Kaliszyk | Beginning of section 5. | changeset | files | 
| Tue, 30 Mar 2010 15:07:42 +0200 | Christian Urban | merged | changeset | files | 
| Tue, 30 Mar 2010 13:58:07 +0200 | Cezary Kaliszyk | Avoid mentioning other nominal datatypes as it makes things too complicated. | changeset | files | 
| Tue, 30 Mar 2010 13:37:35 +0200 | Christian Urban | merged | changeset | files | 
| Tue, 30 Mar 2010 13:36:02 +0200 | Cezary Kaliszyk | close the missing parenthesis on both sides. | changeset | files | 
| Tue, 30 Mar 2010 13:23:12 +0200 | Christian Urban | merged | changeset | files | 
| Tue, 30 Mar 2010 13:22:54 +0200 | Christian Urban | changes to section 2 | changeset | files | 
| Tue, 30 Mar 2010 12:31:28 +0200 | Cezary Kaliszyk | Clean alpha | changeset | files | 
| Tue, 30 Mar 2010 12:19:20 +0200 | Cezary Kaliszyk | clean fv_bn | changeset | files | 
| Tue, 30 Mar 2010 11:45:41 +0200 | Cezary Kaliszyk | alpha_bn | changeset | files | 
| Tue, 30 Mar 2010 11:32:12 +0200 | Cezary Kaliszyk | Change @{text} to @{term} | changeset | files | 
| Tue, 30 Mar 2010 10:36:05 +0200 | Cezary Kaliszyk | alpha | changeset | files | 
| Tue, 30 Mar 2010 09:15:40 +0200 | Cezary Kaliszyk | more | changeset | files | 
| Tue, 30 Mar 2010 09:00:52 +0200 | Cezary Kaliszyk | fv and fv_bn | changeset | files | 
| Tue, 30 Mar 2010 02:55:18 +0200 | Christian Urban | more of the paper | changeset | files | 
| Mon, 29 Mar 2010 22:26:19 +0200 | Christian Urban | merged | changeset | files | 
| Mon, 29 Mar 2010 18:12:54 +0200 | Cezary Kaliszyk | Updated strong induction to modified definitions. | changeset | files | 
| Mon, 29 Mar 2010 17:32:17 +0200 | Cezary Kaliszyk | Initial renaming | changeset | files | 
| Mon, 29 Mar 2010 17:14:02 +0200 | Christian Urban | small changes in the core-haskell spec | changeset | files | 
| Mon, 29 Mar 2010 16:56:59 +0200 | Cezary Kaliszyk | Update according to paper | changeset | files | 
| Mon, 29 Mar 2010 16:44:26 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 29 Mar 2010 16:44:05 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 29 Mar 2010 16:29:50 +0200 | Cezary Kaliszyk | Changed to Lists. | changeset | files | 
| Mon, 29 Mar 2010 16:41:21 +0200 | Christian Urban | clarified core-haskell example | changeset | files | 
| Mon, 29 Mar 2010 14:58:00 +0200 | Christian Urban | spell check | changeset | files | 
| Mon, 29 Mar 2010 12:06:22 +0200 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 29 Mar 2010 12:06:05 +0200 | Cezary Kaliszyk | Abs_gen and Abs_let simplifications. | changeset | files | 
| Mon, 29 Mar 2010 11:23:29 +0200 | Christian Urban | more on the paper | changeset | files | 
| Mon, 29 Mar 2010 01:23:24 +0200 | Christian Urban | fixed a problem due to a change in type-def (needs new Isabelle) | changeset | files | 
| Mon, 29 Mar 2010 00:30:47 +0200 | Christian Urban | merged | changeset | files | 
| Mon, 29 Mar 2010 00:30:20 +0200 | Christian Urban | more on the paper | changeset | files | 
| Sun, 28 Mar 2010 22:54:38 +0200 | Christian Urban | got rid of the aux-function on the raw level, by defining it with function on the quotient level | changeset | files | 
| Sat, 27 Mar 2010 16:20:39 +0100 | Cezary Kaliszyk | Lets finally abstract lists. | changeset | files | 
| Sat, 27 Mar 2010 16:17:45 +0100 | Cezary Kaliszyk | Core Haskell can now use proper strings. | changeset | files | 
| Sat, 27 Mar 2010 14:55:07 +0100 | Cezary Kaliszyk | Automatically lift theorems and constants only using the new quotient types. Requires new Isabelle. | changeset | files | 
| Sat, 27 Mar 2010 14:38:22 +0100 | Cezary Kaliszyk | Remove list_eq notation. | changeset | files | 
| Sat, 27 Mar 2010 13:50:59 +0100 | Cezary Kaliszyk | Get lifted types information from the quotient package. | changeset | files | 
| Sat, 27 Mar 2010 12:26:59 +0100 | Cezary Kaliszyk | Equivariance when bn functions are lists. | changeset | files | 
| Sat, 27 Mar 2010 12:20:17 +0100 | Cezary Kaliszyk | Accepts lists in FV. | changeset | files | 
| Sat, 27 Mar 2010 12:01:28 +0100 | Cezary Kaliszyk | Parsing of list-bn functions into components. | changeset | files | 
| Sat, 27 Mar 2010 09:56:35 +0100 | Cezary Kaliszyk | Automatically compute support if only one type of Abs is present in the type. | changeset | files | 
| Sat, 27 Mar 2010 09:41:00 +0100 | Cezary Kaliszyk | Manually proved TySch support; All properties of TySch now true. | changeset | files | 
| Sat, 27 Mar 2010 09:21:43 +0100 | Cezary Kaliszyk | Generalize Abs_eq_iff. | changeset | files | 
| Sat, 27 Mar 2010 09:15:09 +0100 | Cezary Kaliszyk | Minor fix. | changeset | files | 
| Sat, 27 Mar 2010 08:42:07 +0100 | Cezary Kaliszyk | New compose lemmas. Reverted alpha_gen sym/trans changes. Equivp for alpha_res should work now. | changeset | files | 
| Sat, 27 Mar 2010 08:17:43 +0100 | Cezary Kaliszyk | Initial proof modifications for alpha_res | changeset | files | 
| Sat, 27 Mar 2010 08:11:45 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Sat, 27 Mar 2010 08:11:11 +0100 | Cezary Kaliszyk | Fv/Alpha now takes into account Alpha_Type given from the parser. | changeset | files | 
| Sat, 27 Mar 2010 06:51:13 +0100 | Cezary Kaliszyk | Minor cleaning. | changeset | files | 
| Sat, 27 Mar 2010 06:44:47 +0100 | Christian Urban | merged | changeset | files | 
| Sat, 27 Mar 2010 06:44:14 +0100 | Christian Urban | more on the paper | changeset | files | 
| Sat, 27 Mar 2010 06:44:16 +0100 | Cezary Kaliszyk | Removed some warnings. | changeset | files | 
| Fri, 26 Mar 2010 22:23:22 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Fri, 26 Mar 2010 22:22:41 +0100 | Cezary Kaliszyk | Modified abs_gen_sym and abs_gen_trans so it becomes usable in the proofs. | changeset | files | 
| Fri, 26 Mar 2010 22:08:13 +0100 | Christian Urban | merged | changeset | files | 
| Fri, 26 Mar 2010 22:02:59 +0100 | Christian Urban | more on the paper | changeset | files | 
| Fri, 26 Mar 2010 18:44:47 +0100 | Christian Urban | simplification | changeset | files | 
| Fri, 26 Mar 2010 17:22:17 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Fri, 26 Mar 2010 17:22:02 +0100 | Cezary Kaliszyk | Describe 'nominal_datatype2'. | changeset | files | 
| Fri, 26 Mar 2010 17:01:22 +0100 | Cezary Kaliszyk | Fixed renamings. | changeset | files | 
| Fri, 26 Mar 2010 16:46:40 +0100 | Christian Urban | merged | changeset | files | 
| Fri, 26 Mar 2010 16:20:39 +0100 | Cezary Kaliszyk | Removed remaining cheats + some cleaning. | changeset | files | 
| Fri, 26 Mar 2010 10:55:13 +0100 | Cezary Kaliszyk | Extract PS7 and PS8 from Test. PS7 needs the same fix as Core Haskell. | changeset | files | 
| Fri, 26 Mar 2010 10:35:26 +0100 | Cezary Kaliszyk | Update cheats in TODO. | changeset | files | 
| Fri, 26 Mar 2010 10:07:26 +0100 | Cezary Kaliszyk | Removed another cheat and cleaned the code a bit. | changeset | files | 
| Fri, 26 Mar 2010 09:23:23 +0100 | Cezary Kaliszyk | Fix Manual/LamEx for experiments. | changeset | files | 
| Thu, 25 Mar 2010 20:12:57 +0100 | Cezary Kaliszyk | Proper bn_rsp, for bn functions calling each other. | changeset | files | 
| Thu, 25 Mar 2010 17:30:46 +0100 | Cezary Kaliszyk | Gathering things to prove by induction together; removed cheat_bn_eqvt. | changeset | files | 
| Thu, 25 Mar 2010 15:06:58 +0100 | Cezary Kaliszyk | Update TODO | changeset | files | 
| Thu, 25 Mar 2010 14:31:51 +0100 | Cezary Kaliszyk | Showed ACons_subst. | changeset | files | 
| Thu, 25 Mar 2010 14:24:06 +0100 | Cezary Kaliszyk | Only ACons_subst left to show. | changeset | files | 
| Thu, 25 Mar 2010 12:04:38 +0100 | Cezary Kaliszyk | Solved all boring subgoals, and looking at properly defning permute_bv | changeset | files | 
| Thu, 25 Mar 2010 11:29:54 +0100 | Cezary Kaliszyk | One more copy-and-paste in core-haskell. | changeset | files | 
| Thu, 25 Mar 2010 11:16:25 +0100 | Cezary Kaliszyk | Properly defined permute_bn. No more sorry's in Let strong induction. | changeset | files | 
| Thu, 25 Mar 2010 11:10:15 +0100 | Cezary Kaliszyk | Showed Let substitution. | changeset | files | 
| Thu, 25 Mar 2010 11:01:22 +0100 | Cezary Kaliszyk | Only let substitution is left. | changeset | files | 
| Thu, 25 Mar 2010 10:44:14 +0100 | Cezary Kaliszyk | further in the proof | changeset | files | 
| Thu, 25 Mar 2010 10:25:33 +0100 | Cezary Kaliszyk | trying to prove the string induction for let. | changeset | files | 
| Thu, 25 Mar 2010 09:08:42 +0100 | Christian Urban | added experiemental permute_bn | changeset | files | 
| Thu, 25 Mar 2010 08:05:03 +0100 | Christian Urban | first attempt of strong induction for lets with assignments | changeset | files | 
| Thu, 25 Mar 2010 07:21:41 +0100 | Christian Urban | more on the paper | changeset | files | 
| Wed, 24 Mar 2010 19:50:42 +0100 | Christian Urban | more on the paper | changeset | files | 
| Wed, 24 Mar 2010 18:02:33 +0100 | Cezary Kaliszyk | Further in the strong induction proof. | changeset | files | 
| Wed, 24 Mar 2010 16:06:31 +0100 | Cezary Kaliszyk | Solved one of the strong-induction goals. | changeset | files | 
| Wed, 24 Mar 2010 14:49:51 +0100 | Cezary Kaliszyk | avoiding for atom. | changeset | files | 
| Wed, 24 Mar 2010 13:54:20 +0100 | Cezary Kaliszyk | Started proving strong induction. | changeset | files | 
| Wed, 24 Mar 2010 12:36:58 +0100 | Cezary Kaliszyk | stating the strong induction; further. | changeset | files | 
| Wed, 24 Mar 2010 12:05:38 +0100 | Cezary Kaliszyk | Working on stating induct. | changeset | files | 
| Wed, 24 Mar 2010 12:53:39 +0100 | Christian Urban | some tuning; possible fix for strange paper generation | changeset | files | 
| Wed, 24 Mar 2010 12:34:28 +0100 | Christian Urban | more on the paper | changeset | files | 
| Wed, 24 Mar 2010 12:04:03 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 24 Mar 2010 12:03:48 +0100 | Cezary Kaliszyk | Showed support of Core Haskell | changeset | files | 
| Wed, 24 Mar 2010 11:13:39 +0100 | Cezary Kaliszyk | Support proof modification for Core Haskell. | changeset | files | 
| Wed, 24 Mar 2010 10:55:59 +0100 | Cezary Kaliszyk | Experiments with Core Haskell support. | changeset | files | 
| Wed, 24 Mar 2010 10:49:50 +0100 | Cezary Kaliszyk | Export all the cheats needed for Core Haskell. | changeset | files | 
| Wed, 24 Mar 2010 09:59:47 +0100 | Cezary Kaliszyk | Compute Fv for non-recursive bn functions calling other bn functions | changeset | files | 
| Wed, 24 Mar 2010 08:45:54 +0100 | Cezary Kaliszyk | Core Haskell experiments. | changeset | files | 
| Wed, 24 Mar 2010 07:23:53 +0100 | Christian Urban | tuned paper | changeset | files | 
| Tue, 23 Mar 2010 17:44:43 +0100 | Christian Urban | more of the paper | changeset | files | 
| Tue, 23 Mar 2010 17:22:37 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 23 Mar 2010 17:22:19 +0100 | Christian Urban | more tuning in the paper | changeset | files | 
| Tue, 23 Mar 2010 16:28:46 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 23 Mar 2010 16:28:29 +0100 | Cezary Kaliszyk | Parsing bn functions that call other bn functions and transmitting this information to fv/alpha. | changeset | files | 
| Tue, 23 Mar 2010 13:07:11 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 23 Mar 2010 13:07:02 +0100 | Christian Urban | more tuning | changeset | files | 
| Tue, 23 Mar 2010 13:03:42 +0100 | Christian Urban | tuned paper | changeset | files | 
| Tue, 23 Mar 2010 11:52:55 +0100 | Christian Urban | more on the paper | changeset | files | 
| Tue, 23 Mar 2010 11:43:09 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 23 Mar 2010 11:42:06 +0100 | Cezary Kaliszyk | Modification to Core Haskell to make it accepted with an empty binding function. | changeset | files | 
| Tue, 23 Mar 2010 10:26:46 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 23 Mar 2010 10:24:12 +0100 | Christian Urban | tuned paper | changeset | files | 
| Tue, 23 Mar 2010 09:56:29 +0100 | Cezary Kaliszyk | Initial list unfoldings in Core Haskell. | changeset | files | 
| Tue, 23 Mar 2010 09:38:03 +0100 | Cezary Kaliszyk | compiles | changeset | files | 
| Tue, 23 Mar 2010 09:34:32 +0100 | Cezary Kaliszyk | More modification needed for compilation | changeset | files | 
| Tue, 23 Mar 2010 09:21:43 +0100 | Cezary Kaliszyk | Moved let properties from Term5 to ExLetRec. | changeset | files | 
| Tue, 23 Mar 2010 09:13:17 +0100 | Cezary Kaliszyk | Move Let properties to ExLet | changeset | files | 
| Tue, 23 Mar 2010 09:06:28 +0100 | Cezary Kaliszyk | Added missing file | changeset | files | 
| Tue, 23 Mar 2010 09:05:23 +0100 | Cezary Kaliszyk | More reorganization. | changeset | files | 
| Tue, 23 Mar 2010 08:51:43 +0100 | Cezary Kaliszyk | Move Leroy out of Test, rename accordingly. | changeset | files | 
| Tue, 23 Mar 2010 08:46:44 +0100 | Cezary Kaliszyk | Term1 is identical to Example 3 | changeset | files | 
| Tue, 23 Mar 2010 08:45:08 +0100 | Cezary Kaliszyk | Move example3 out. | changeset | files | 
| Tue, 23 Mar 2010 08:42:02 +0100 | Cezary Kaliszyk | Move Ex1 and Ex2 out of Test | changeset | files | 
| Tue, 23 Mar 2010 08:33:48 +0100 | Cezary Kaliszyk | Move examples which create more permutations out | changeset | files | 
| Tue, 23 Mar 2010 08:22:48 +0100 | Cezary Kaliszyk | Move LamEx out of Test. | changeset | files | 
| Tue, 23 Mar 2010 08:20:13 +0100 | Cezary Kaliszyk | Move lambda examples to manual | changeset | files | 
| Tue, 23 Mar 2010 08:19:33 +0100 | Cezary Kaliszyk | Move manual examples to a subdirectory. | changeset | files | 
| Tue, 23 Mar 2010 08:16:39 +0100 | Cezary Kaliszyk | Removed compat tests. | changeset | files | 
| Tue, 23 Mar 2010 08:11:39 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 23 Mar 2010 08:11:11 +0100 | Cezary Kaliszyk | Move Non-respectful examples to NotRsp | changeset | files | 
| Tue, 23 Mar 2010 07:43:20 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 23 Mar 2010 07:39:10 +0100 | Christian Urban | more on the paper | changeset | files | 
| Tue, 23 Mar 2010 07:04:27 +0100 | Cezary Kaliszyk | Move the comment to appropriate place. | changeset | files | 
| Tue, 23 Mar 2010 07:04:14 +0100 | Cezary Kaliszyk | Remove compose_eqvt | changeset | files | 
| Mon, 22 Mar 2010 18:56:35 +0100 | Cezary Kaliszyk | sym proof with compose. | changeset | files | 
| Mon, 22 Mar 2010 18:38:59 +0100 | Cezary Kaliszyk | Marked the place where a compose lemma applies. | changeset | files | 
| Mon, 22 Mar 2010 18:29:57 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 22 Mar 2010 18:29:29 +0100 | Cezary Kaliszyk | equivp_cheat can be removed for all one-permutation examples. | changeset | files | 
| Mon, 22 Mar 2010 18:20:06 +0100 | Christian Urban | merged | changeset | files | 
| Mon, 22 Mar 2010 18:19:13 +0100 | Christian Urban | more on the paper | changeset | files | 
| Mon, 22 Mar 2010 16:22:28 +0100 | Christian Urban | merged | changeset | files | 
| Mon, 22 Mar 2010 16:22:07 +0100 | Christian Urban | tuned paper | changeset | files | 
| Mon, 22 Mar 2010 17:21:27 +0100 | Cezary Kaliszyk | Got rid of alpha_bn_rsp_cheat. | changeset | files | 
| Mon, 22 Mar 2010 15:27:01 +0100 | Cezary Kaliszyk | alpha_bn_rsp_pre automatized. | changeset | files | 
| Mon, 22 Mar 2010 14:07:35 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 22 Mar 2010 14:07:07 +0100 | Cezary Kaliszyk | fv_rsp proved automatically. | changeset | files | 
| Mon, 22 Mar 2010 11:55:29 +0100 | Christian Urban | more on the paper | changeset | files | 
| Mon, 22 Mar 2010 10:21:14 +0100 | Christian Urban | merged | changeset | files | 
| Mon, 22 Mar 2010 10:20:57 +0100 | Christian Urban | tuned paper | changeset | files | 
| Mon, 22 Mar 2010 09:16:25 +0100 | Christian Urban | some tuning | changeset | files | 
| Mon, 22 Mar 2010 10:15:46 +0100 | Cezary Kaliszyk | Strong induction for Type Schemes. | changeset | files | 
| Mon, 22 Mar 2010 09:02:30 +0100 | Cezary Kaliszyk | Fixed missing colon. | changeset | files | 
| Sun, 21 Mar 2010 22:27:08 +0100 | Christian Urban | tuned paper | changeset | files | 
| Sat, 20 Mar 2010 18:16:26 +0100 | Christian Urban | merged | changeset | files | 
| Sat, 20 Mar 2010 16:27:51 +0100 | Christian Urban | proved at_set_avoiding2 which is needed for strong induction principles | changeset | files | 
| Sat, 20 Mar 2010 13:50:00 +0100 | Christian Urban | moved lemmas supp_perm_eq and exists_perm to Nominal2_Supp | changeset | files | 
| Sat, 20 Mar 2010 10:12:09 +0100 | Cezary Kaliszyk | Size experiments. | changeset | files | 
| Sat, 20 Mar 2010 09:27:28 +0100 | Cezary Kaliszyk | Use 'alpha_bn_refl' to get rid of one of the sorrys. | changeset | files | 
| Sat, 20 Mar 2010 08:56:07 +0100 | Cezary Kaliszyk | Build alpha-->alphabn implications | changeset | files | 
| Sat, 20 Mar 2010 08:04:59 +0100 | Cezary Kaliszyk | Prove reflp for all relations. | changeset | files | 
| Sat, 20 Mar 2010 04:51:26 +0100 | Christian Urban | started cleaning up and introduced 3 versions of ~~gen | changeset | files | 
| Sat, 20 Mar 2010 02:46:07 +0100 | Christian Urban | moved infinite_Un into mainstream Isabelle; moved permute_boolI/E lemmas | changeset | files | 
| Fri, 19 Mar 2010 21:04:24 +0100 | Christian Urban | more work on the paper | changeset | files | 
| Fri, 19 Mar 2010 18:56:13 +0100 | Cezary Kaliszyk | Described automatically created funs. | changeset | files | 
| Fri, 19 Mar 2010 18:43:29 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Fri, 19 Mar 2010 18:42:57 +0100 | Cezary Kaliszyk | Automatically derive support for datatypes with at-most one binding per constructor. | changeset | files | 
| Fri, 19 Mar 2010 17:20:25 +0100 | Christian Urban | picture | changeset | files | 
| Fri, 19 Mar 2010 15:43:59 +0100 | Christian Urban | merged | changeset | files | 
| Fri, 19 Mar 2010 15:43:43 +0100 | Christian Urban | polished | changeset | files | 
| Fri, 19 Mar 2010 15:01:01 +0100 | Cezary Kaliszyk | Update Test to use fset. | changeset | files | 
| Fri, 19 Mar 2010 14:54:57 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Fri, 19 Mar 2010 14:54:30 +0100 | Cezary Kaliszyk | Use fs typeclass in showing finite support + some cheat cleaning. | changeset | files | 
| Fri, 19 Mar 2010 12:31:55 +0100 | Christian Urban | merged | changeset | files | 
| Fri, 19 Mar 2010 12:31:17 +0100 | Christian Urban | more one the paper | changeset | files | 
| Fri, 19 Mar 2010 12:28:35 +0100 | Cezary Kaliszyk | Keep only one copy of infinite_Un. | changeset | files | 
| Fri, 19 Mar 2010 12:24:16 +0100 | Cezary Kaliszyk | Added a missing 'import'. | changeset | files | 
| Fri, 19 Mar 2010 12:22:10 +0100 | Cezary Kaliszyk | Showed the instance: fset::(at) fs | changeset | files | 
| Fri, 19 Mar 2010 10:24:49 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Fri, 19 Mar 2010 10:24:16 +0100 | Cezary Kaliszyk | Remove atom_decl from the parser. | changeset | files | 
| Fri, 19 Mar 2010 10:23:52 +0100 | Cezary Kaliszyk | TySch strong induction looks ok. | changeset | files | 
| Fri, 19 Mar 2010 09:31:38 +0100 | Cezary Kaliszyk | Working on TySch strong induction. | changeset | files | 
| Fri, 19 Mar 2010 09:03:10 +0100 | Cezary Kaliszyk | Something is wrong with the statement of strong induction for TySch, as the All case is trivial and Fun case unprovable... | changeset | files | 
| Fri, 19 Mar 2010 09:40:57 +0100 | Christian Urban | merged | changeset | files | 
| Fri, 19 Mar 2010 09:40:34 +0100 | Christian Urban | more tuning on the paper | changeset | files | 
| Fri, 19 Mar 2010 08:31:43 +0100 | Cezary Kaliszyk | The nominal infrastructure for fset. 'fs' missing, but not needed so far. | changeset | files | 
| Fri, 19 Mar 2010 06:55:17 +0100 | Cezary Kaliszyk | A few more theorems in FSet. | changeset | files | 
| Fri, 19 Mar 2010 00:36:08 +0100 | Cezary Kaliszyk | merge 2 | changeset | files | 
| Fri, 19 Mar 2010 00:35:58 +0100 | Cezary Kaliszyk | merge 1 | changeset | files | 
| Fri, 19 Mar 2010 00:35:20 +0100 | Cezary Kaliszyk | support of fset_to_set, support of fmap_atom. | changeset | files | 
| Thu, 18 Mar 2010 23:39:48 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 18 Mar 2010 23:39:26 +0100 | Christian Urban | more tuning on the paper | changeset | files | 
| Thu, 18 Mar 2010 23:38:01 +0100 | Christian Urban | added item about size functions | changeset | files | 
| Thu, 18 Mar 2010 23:20:46 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Thu, 18 Mar 2010 23:19:55 +0100 | Cezary Kaliszyk | Reached strong_induction in fset-based TySch. Will not work until isabelle changes are pushed. | changeset | files | 
| Thu, 18 Mar 2010 22:06:28 +0100 | Christian Urban | tuned | changeset | files | 
| Thu, 18 Mar 2010 19:39:01 +0100 | Christian Urban | another little bit for the introduction | changeset | files | 
| Thu, 18 Mar 2010 19:02:33 +0100 | Cezary Kaliszyk | Leroy96 supp=fv and fixes to make it compile | changeset | files | 
| Thu, 18 Mar 2010 18:43:21 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 18 Mar 2010 18:43:03 +0100 | Christian Urban | more of the introduction | changeset | files | 
| Thu, 18 Mar 2010 18:10:49 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Thu, 18 Mar 2010 18:10:20 +0100 | Cezary Kaliszyk | Added a cleaned version of FSet. | changeset | files | 
| Thu, 18 Mar 2010 16:22:10 +0100 | Christian Urban | corrected the strong induction principle in the lambda-calculus case; gave a second (oartial) version that is more elegant | changeset | files | 
| Thu, 18 Mar 2010 15:32:49 +0100 | Cezary Kaliszyk | Continued description of alpha. | changeset | files | 
| Thu, 18 Mar 2010 15:13:20 +0100 | Cezary Kaliszyk | Rename "_property" to ".property" | changeset | files | 
| Thu, 18 Mar 2010 14:48:27 +0100 | Cezary Kaliszyk | First part of the description of alpha_ty. | changeset | files | 
| Thu, 18 Mar 2010 14:29:42 +0100 | Cezary Kaliszyk | Description of generation of alpha_bn. | changeset | files | 
| Thu, 18 Mar 2010 14:05:49 +0100 | Cezary Kaliszyk | case names also for _induct | changeset | files | 
| Thu, 18 Mar 2010 12:32:03 +0100 | Cezary Kaliszyk | Case_Names for _inducts. Does not work for _induct yet. | changeset | files | 
| Thu, 18 Mar 2010 12:09:59 +0100 | Cezary Kaliszyk | Added fv,bn,distinct,perm to the simplifier. | changeset | files | 
| Thu, 18 Mar 2010 11:37:10 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Thu, 18 Mar 2010 11:36:03 +0100 | Cezary Kaliszyk | Simplified the description. | changeset | files | 
| Thu, 18 Mar 2010 11:33:56 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 18 Mar 2010 11:33:37 +0100 | Christian Urban | slightly more in the paper | changeset | files | 
| Thu, 18 Mar 2010 11:29:12 +0100 | Cezary Kaliszyk | Update the description of the generation of fv function. | changeset | files | 
| Thu, 18 Mar 2010 11:16:53 +0100 | Cezary Kaliszyk | fv_bn may need to call other fv_bns. | changeset | files | 
| Thu, 18 Mar 2010 10:15:57 +0100 | Cezary Kaliszyk | Update TODO. | changeset | files | 
| Thu, 18 Mar 2010 10:12:41 +0100 | Cezary Kaliszyk | Which proofs need a 'sorry'. | changeset | files | 
| Thu, 18 Mar 2010 10:05:36 +0100 | Christian Urban | added TODO | changeset | files | 
| Thu, 18 Mar 2010 10:02:21 +0100 | Christian Urban | vixed variable names | changeset | files | 
| Thu, 18 Mar 2010 09:31:31 +0100 | Christian Urban | simplified strong induction proof by using flip | changeset | files | 
| Thu, 18 Mar 2010 08:32:55 +0100 | Cezary Kaliszyk | Rename bound variables + minor cleaning. | changeset | files | 
| Thu, 18 Mar 2010 08:03:42 +0100 | Cezary Kaliszyk | Move most of the exporting out of the parser. | changeset | files | 
| Thu, 18 Mar 2010 07:43:44 +0100 | Cezary Kaliszyk | Prove pseudo-inject (eq-iff) on the exported level and rename appropriately. | changeset | files | 
| Thu, 18 Mar 2010 07:35:44 +0100 | Cezary Kaliszyk | Prove eqvts on exported terms. | changeset | files | 
| Thu, 18 Mar 2010 07:26:36 +0100 | Cezary Kaliszyk | Clean 'Lift', start working only on exported things in Parser. | changeset | files | 
| Thu, 18 Mar 2010 00:17:21 +0100 | Christian Urban | slightly more of the paper | changeset | files | 
| Wed, 17 Mar 2010 20:42:42 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 17 Mar 2010 20:42:22 +0100 | Christian Urban | paper uses now a heap file - does not compile so long anymore | changeset | files | 
| Wed, 17 Mar 2010 18:53:23 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 17 Mar 2010 18:52:59 +0100 | Cezary Kaliszyk | compose_sym2 works also for term5 | changeset | files | 
| Wed, 17 Mar 2010 17:59:04 +0100 | Cezary Kaliszyk | Updated Term1, including statement of strong induction. | changeset | files | 
| Wed, 17 Mar 2010 17:40:14 +0100 | Cezary Kaliszyk | Proper compose_sym2 | changeset | files | 
| Wed, 17 Mar 2010 17:11:23 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 17 Mar 2010 17:10:19 +0100 | Christian Urban | temporarily disabled tests in Nominal/ROOT | changeset | files | 
| Wed, 17 Mar 2010 15:13:31 +0100 | Christian Urban | made paper to compile | changeset | files | 
| Wed, 17 Mar 2010 15:13:03 +0100 | Christian Urban | added partial proof for the strong induction principle | changeset | files | 
| Wed, 17 Mar 2010 17:09:01 +0100 | Cezary Kaliszyk | Trying to find a compose lemma for 2 arguments. | changeset | files | 
| Wed, 17 Mar 2010 12:23:04 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 17 Mar 2010 12:18:35 +0100 | Cezary Kaliszyk | cheat_alpha_eqvt no longer needed. Cleaned the tracing messages. | changeset | files | 
| Wed, 17 Mar 2010 11:54:22 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 17 Mar 2010 11:53:56 +0100 | Christian Urban | added proof of supp/fv for type schemes | changeset | files | 
| Wed, 17 Mar 2010 11:40:58 +0100 | Cezary Kaliszyk | Updated Type Schemes to automatic lifting. One goal is not true because of the restriction. | changeset | files | 
| Wed, 17 Mar 2010 11:20:24 +0100 | Cezary Kaliszyk | Remove Term5a, since it is now identical to Term5. | changeset | files | 
| Wed, 17 Mar 2010 11:11:42 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 17 Mar 2010 11:11:25 +0100 | Cezary Kaliszyk | Finished all proofs in Term5 and Term5n. | changeset | files | 
| Wed, 17 Mar 2010 10:34:25 +0100 | Christian Urban | added partial proof of supp for type schemes | changeset | files | 
| Wed, 17 Mar 2010 09:57:54 +0100 | Cezary Kaliszyk | Fix in alpha; support of the recursive Let works :) | changeset | files | 
| Wed, 17 Mar 2010 09:42:56 +0100 | Cezary Kaliszyk | The recursive supp just has one equation too much. | changeset | files | 
| Wed, 17 Mar 2010 09:25:01 +0100 | Cezary Kaliszyk | Fix for the change of alpha_gen. | changeset | files | 
| Wed, 17 Mar 2010 09:18:27 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 17 Mar 2010 09:17:55 +0100 | Cezary Kaliszyk | Generate compound FV and Alpha for recursive bindings. | changeset | files | 
| Wed, 17 Mar 2010 08:39:46 +0100 | Cezary Kaliszyk | Lifting theorems with compound fv and compound alpha. | changeset | files | 
| Wed, 17 Mar 2010 08:07:25 +0100 | Christian Urban | commented out examples that should not work; but for example type-scheme example should work | changeset | files | 
| Wed, 17 Mar 2010 06:49:33 +0100 | Christian Urban | added another supp-proof for the non-recursive case | changeset | files | 
| Tue, 16 Mar 2010 20:07:13 +0100 | Cezary Kaliszyk | Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not. | changeset | files | 
| Tue, 16 Mar 2010 18:19:00 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 16 Mar 2010 18:18:08 +0100 | Cezary Kaliszyk | The old recursive alpha works fine. | changeset | files | 
| Tue, 16 Mar 2010 18:13:34 +0100 | Christian Urban | added the final unfolded result | changeset | files | 
| Tue, 16 Mar 2010 18:02:08 +0100 | Christian Urban | merge and proof of support for non-recursive case | changeset | files | 
| Tue, 16 Mar 2010 17:20:46 +0100 | Cezary Kaliszyk | Added Term5 non-recursive. The bug is there only for the recursive case. | changeset | files | 
| Tue, 16 Mar 2010 17:11:32 +0100 | Cezary Kaliszyk | Alpha is wrong. | changeset | files | 
| Tue, 16 Mar 2010 16:51:06 +0100 | Cezary Kaliszyk | alpha_bn doesn't need the permutation in non-recursive case. | changeset | files | 
| Tue, 16 Mar 2010 16:17:05 +0100 | Cezary Kaliszyk | alpha5_transp and equivp | changeset | files | 
| Tue, 16 Mar 2010 15:38:14 +0100 | Cezary Kaliszyk | alpha5_symp proved. | changeset | files | 
| Tue, 16 Mar 2010 15:27:47 +0100 | Cezary Kaliszyk | FV_bn generated for recursive functions as well, and used in main fv for bindings. | changeset | files | 
| Tue, 16 Mar 2010 12:08:37 +0100 | Cezary Kaliszyk | The proof in 'Test' gets simpler. | changeset | files | 
| Tue, 16 Mar 2010 12:06:22 +0100 | Cezary Kaliszyk | Removed pi o bn = bn' assumption in alpha | changeset | files | 
| Mon, 15 Mar 2010 23:42:56 +0100 | Christian Urban | merged (confirmed to work with Isabelle from 6th March) | changeset | files | 
| Mon, 15 Mar 2010 17:52:31 +0100 | Christian Urban | another synchronisation | changeset | files | 
| Mon, 15 Mar 2010 17:51:35 +0100 | Christian Urban | proof for support when bn-function is present, but fb_function is empty | changeset | files | 
| Mon, 15 Mar 2010 17:42:17 +0100 | Cezary Kaliszyk | fv_eqvt_cheat no longer needed. | changeset | files | 
| Mon, 15 Mar 2010 14:32:05 +0100 | Cezary Kaliszyk | derive "inducts" from "induct" instead of lifting again is much faster. | changeset | files | 
| Mon, 15 Mar 2010 13:56:17 +0100 | Cezary Kaliszyk | build_eqvts works with recursive case if proper induction rule is used. | changeset | files | 
| Mon, 15 Mar 2010 11:50:12 +0100 | Cezary Kaliszyk | cheat_alpha_eqvt no longer needed; the proofs work. | changeset | files | 
| Mon, 15 Mar 2010 10:36:09 +0100 | Cezary Kaliszyk | LF works with new alpha...? | changeset | files | 
| Mon, 15 Mar 2010 10:07:15 +0100 | Cezary Kaliszyk | explicit flag "cheat_equivp" | changeset | files | 
| Mon, 15 Mar 2010 10:02:19 +0100 | Cezary Kaliszyk | Prove alpha_gen_compose_eqvt | changeset | files | 
| Mon, 15 Mar 2010 09:27:25 +0100 | Cezary Kaliszyk | Use eqvt. | changeset | files | 
| Mon, 15 Mar 2010 08:39:23 +0100 | Christian Urban | added preliminary test version....but Test works now | changeset | files | 
| Mon, 15 Mar 2010 08:28:10 +0100 | Christian Urban | added an eqvt-proof for bi | changeset | files | 
| Mon, 15 Mar 2010 06:11:35 +0100 | Christian Urban | synchronised with main hg-repository; used add_typedef_global in nominal_atoms | changeset | files | 
| Sun, 14 Mar 2010 11:36:15 +0100 | Christian Urban | localised the typedef in Attic (requires new Isabelle) | changeset | files | 
| Sat, 13 Mar 2010 13:49:15 +0100 | Christian Urban | started supp-fv proofs (is going to work) | changeset | files | 
| Fri, 12 Mar 2010 17:42:31 +0100 | Cezary Kaliszyk | Even with pattern simplified to a single clause, the supp equation doesn't seem true. | changeset | files | 
| Fri, 12 Mar 2010 12:42:35 +0100 | Cezary Kaliszyk | Still don't know how to prove supp=fv for simplest Let... | changeset | files | 
| Thu, 11 Mar 2010 20:49:31 +0100 | Cezary Kaliszyk | Do not fail if the finite support proof fails. | changeset | files | 
| Thu, 11 Mar 2010 19:43:50 +0100 | Christian Urban | generalised the supp for atoms to all concrete atoms (not just names) | changeset | files | 
| Thu, 11 Mar 2010 19:41:11 +0100 | Christian Urban | support of atoms at the end of Abs.thy | changeset | files | 
| Thu, 11 Mar 2010 19:24:07 +0100 | Cezary Kaliszyk | Trying to prove atom_image_fresh_swap | changeset | files | 
| Thu, 11 Mar 2010 17:49:07 +0100 | Cezary Kaliszyk | Finite_support proof no longer needed in LF. | changeset | files | 
| Thu, 11 Mar 2010 17:47:29 +0100 | Cezary Kaliszyk | Show that the new types are in finite support typeclass. | changeset | files | 
| Thu, 11 Mar 2010 16:50:44 +0100 | Cezary Kaliszyk | mk_supports_eq and supports_tac. | changeset | files | 
| Thu, 11 Mar 2010 16:16:15 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Thu, 11 Mar 2010 16:15:29 +0100 | Cezary Kaliszyk | Fixes for term1 for new alpha. Still not able to show support equations. | changeset | files | 
| Thu, 11 Mar 2010 16:12:15 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 11 Mar 2010 15:10:07 +0100 | Christian Urban | finally the proof that new and old alpha agree | changeset | files | 
| Thu, 11 Mar 2010 15:11:57 +0100 | Cezary Kaliszyk | Remove "_raw" from lifted theorems. | changeset | files | 
| Thu, 11 Mar 2010 14:09:54 +0100 | Cezary Kaliszyk | looking at trm5_equivp | changeset | files | 
| Thu, 11 Mar 2010 14:05:36 +0100 | Cezary Kaliszyk | The cheats described explicitely. | changeset | files | 
| Thu, 11 Mar 2010 13:44:54 +0100 | Cezary Kaliszyk | The alpha5_eqvt tactic works if I manage to build the goal. | changeset | files | 
| Thu, 11 Mar 2010 13:34:45 +0100 | Cezary Kaliszyk | With the 4 cheats, all examples fully lift. | changeset | files | 
| Thu, 11 Mar 2010 12:30:53 +0100 | Cezary Kaliszyk | Lift alpha_bn_constants. | changeset | files | 
| Thu, 11 Mar 2010 12:26:24 +0100 | Cezary Kaliszyk | Lifting constants. | changeset | files | 
| Thu, 11 Mar 2010 11:41:27 +0100 | Cezary Kaliszyk | Proper error message. | changeset | files | 
| Thu, 11 Mar 2010 11:32:37 +0100 | Cezary Kaliszyk | Lifting constants works for all examples. | changeset | files | 
| Thu, 11 Mar 2010 11:25:56 +0100 | Cezary Kaliszyk | Remove tracing from fv/alpha. | changeset | files | 
| Thu, 11 Mar 2010 11:25:18 +0100 | Cezary Kaliszyk | Equivp working only on the standard alpha-equivalences. | changeset | files | 
| Thu, 11 Mar 2010 11:20:50 +0100 | Cezary Kaliszyk | explicit cheat_fv_eqvt | changeset | files | 
| Thu, 11 Mar 2010 11:15:14 +0100 | Cezary Kaliszyk | extract build_eqvts_tac. | changeset | files | 
| Thu, 11 Mar 2010 10:39:29 +0100 | Cezary Kaliszyk | build_eqvts no longer requires permutations. | changeset | files | 
| Thu, 11 Mar 2010 10:22:24 +0100 | Cezary Kaliszyk | Add explicit alpha_eqvt_cheat. | changeset | files | 
| Thu, 11 Mar 2010 10:10:23 +0100 | Cezary Kaliszyk | Export tactic out of alpha_eqvt. | changeset | files | 
| Wed, 10 Mar 2010 16:59:08 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 10 Mar 2010 16:58:14 +0100 | Cezary Kaliszyk | More tries about the proofs in trm5 | changeset | files | 
| Wed, 10 Mar 2010 16:51:15 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 10 Mar 2010 16:50:42 +0100 | Christian Urban | almost done with showing the equivalence between old and new alpha-equivalence (one subgoal remaining) | changeset | files | 
| Wed, 10 Mar 2010 15:40:15 +0100 | Cezary Kaliszyk | alpha_equivp for trm5 | changeset | files | 
| Wed, 10 Mar 2010 15:34:13 +0100 | Cezary Kaliszyk | Undoing mistakenly committed parser experiments. | changeset | files | 
| Wed, 10 Mar 2010 15:32:51 +0100 | Cezary Kaliszyk | alpha_eqvt for recursive term1. | changeset | files | 
| Wed, 10 Mar 2010 14:47:04 +0100 | Cezary Kaliszyk | Looking at alpha_eqvt for term5, not much progress. | changeset | files | 
| Wed, 10 Mar 2010 14:24:27 +0100 | Cezary Kaliszyk | Reordered examples in Test. | changeset | files | 
| Wed, 10 Mar 2010 13:29:12 +0100 | Cezary Kaliszyk | Allows multiple bindings with same lhs. | changeset | files | 
| Wed, 10 Mar 2010 13:10:00 +0100 | Cezary Kaliszyk | Linked parser to fv and alpha. | changeset | files | 
| Wed, 10 Mar 2010 12:53:44 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 10 Mar 2010 12:53:30 +0100 | Cezary Kaliszyk | A minor fix for shallow binders. LF works again. | changeset | files | 
| Wed, 10 Mar 2010 12:48:55 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 10 Mar 2010 12:48:38 +0100 | Christian Urban | parser produces ordered bn-fun information | changeset | files | 
| Wed, 10 Mar 2010 11:39:28 +0100 | Cezary Kaliszyk | Testing equalities in trm5, all seems good. | changeset | files | 
| Wed, 10 Mar 2010 11:19:59 +0100 | Cezary Kaliszyk | Fv&Alpha seem to work. | changeset | files | 
| Wed, 10 Mar 2010 10:47:21 +0100 | Cezary Kaliszyk | include alpha in the definitions. | changeset | files | 
| Wed, 10 Mar 2010 10:11:20 +0100 | Cezary Kaliszyk | Filled the algorithm for alpha_bn_arg | changeset | files | 
| Wed, 10 Mar 2010 09:58:43 +0100 | Cezary Kaliszyk | rhs of alpha_bn, and template for the arguments. | changeset | files | 
| Wed, 10 Mar 2010 09:45:38 +0100 | Cezary Kaliszyk | alpha_bn_constr template | changeset | files | 
| Wed, 10 Mar 2010 09:36:07 +0100 | Cezary Kaliszyk | exported template for alpha_bn | changeset | files | 
| Wed, 10 Mar 2010 09:10:11 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 10 Mar 2010 09:09:52 +0100 | Cezary Kaliszyk | Use alpha_bns in normal alpha defs. | changeset | files | 
| Wed, 10 Mar 2010 08:44:19 +0100 | Cezary Kaliszyk | alpha_bn_frees | changeset | files | 
| Tue, 09 Mar 2010 22:10:10 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 09 Mar 2010 22:08:38 +0100 | Christian Urban | added bn-information, but it is not yet ordered according to the dts | changeset | files | 
| Tue, 09 Mar 2010 21:22:22 +0100 | Cezary Kaliszyk | Separate lists for separate constructors, to match bn_eqs. | changeset | files | 
| Tue, 09 Mar 2010 17:25:35 +0100 | Cezary Kaliszyk | All examples should work. | changeset | files | 
| Tue, 09 Mar 2010 17:02:29 +0100 | Cezary Kaliszyk | Fix to get old alpha. | changeset | files | 
| Tue, 09 Mar 2010 16:57:51 +0100 | Cezary Kaliszyk | Separate primrecs in Fv. | changeset | files | 
| Tue, 09 Mar 2010 16:24:39 +0100 | Cezary Kaliszyk | A version of Fv that takes into account recursive and non-recursive bindings. | changeset | files | 
| 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. | changeset | files | 
| Tue, 09 Mar 2010 11:06:57 +0100 | Cezary Kaliszyk | fv_bi and alpha_bi | changeset | files | 
| Tue, 09 Mar 2010 09:55:19 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 09 Mar 2010 09:54:58 +0100 | Christian Urban | added first test about new compat | changeset | files | 
| Tue, 09 Mar 2010 09:38:49 +0100 | Cezary Kaliszyk | fv_compat | changeset | files | 
| Tue, 09 Mar 2010 08:46:55 +0100 | Christian Urban | added another compat example | changeset | files | 
| Mon, 08 Mar 2010 20:18:27 +0100 | Christian Urban | added a test-file for compatibility | changeset | files | 
| Mon, 08 Mar 2010 16:11:42 +0100 | Christian Urban | added compat definitions to some examples | changeset | files | 
| Mon, 08 Mar 2010 15:28:25 +0100 | Cezary Kaliszyk | Proper recognition of atoms and atom sets. | changeset | files | 
| Mon, 08 Mar 2010 15:06:14 +0100 | Christian Urban | deleted comments about "weird" | changeset | files | 
| Mon, 08 Mar 2010 15:01:26 +0100 | Christian Urban | merged | changeset | files | 
| Mon, 08 Mar 2010 15:01:01 +0100 | Christian Urban | updated to new Isabelle | changeset | files | 
| Mon, 08 Mar 2010 14:31:04 +0100 | Cezary Kaliszyk | Term5 written as nominal_datatype is the recursive let. | changeset | files | 
| 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. | changeset | files | 
| Mon, 08 Mar 2010 11:12:15 +0100 | Cezary Kaliszyk | More fine-grained nominal restriction for debugging. | changeset | files | 
| Mon, 08 Mar 2010 11:10:43 +0100 | Cezary Kaliszyk | Fix permutation addition. | changeset | files | 
| Mon, 08 Mar 2010 10:33:55 +0100 | Cezary Kaliszyk | Update the comments | changeset | files | 
| Mon, 08 Mar 2010 10:08:31 +0100 | Cezary Kaliszyk | Gather bindings with same binder, and generate only one permutation for them. | changeset | files | 
| Mon, 08 Mar 2010 02:40:16 +0100 | Cezary Kaliszyk | Undo effects of simp. | changeset | files | 
| Sun, 07 Mar 2010 21:30:57 +0100 | Christian Urban | merged | changeset | files | 
| Sun, 07 Mar 2010 21:30:12 +0100 | Christian Urban | updated to renamings in Isabelle | changeset | files | 
| Thu, 04 Mar 2010 15:56:58 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 04 Mar 2010 15:31:34 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 04 Mar 2010 15:31:21 +0100 | Christian Urban | more proofs in Abs and work on Core Haskell | changeset | files | 
| Wed, 03 Mar 2010 19:10:40 +0100 | Christian Urban | added a lemma that permutations can be represented as sums of swapping | changeset | files | 
| Fri, 05 Mar 2010 18:14:04 +0100 | Cezary Kaliszyk | Still unable to show supp=fv for let with one existential. | changeset | files | 
| Fri, 05 Mar 2010 17:09:48 +0100 | Cezary Kaliszyk | Ported LF to the parser interface. | changeset | files | 
| Fri, 05 Mar 2010 14:56:19 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Fri, 05 Mar 2010 14:55:21 +0100 | Cezary Kaliszyk | Lift fv and bn eqvts; no need to lift alpha_eqvt. | changeset | files | 
| Fri, 05 Mar 2010 13:04:47 +0100 | Cezary Kaliszyk | Not much progress about the single existential let case. | changeset | files | 
| Fri, 05 Mar 2010 10:23:40 +0100 | Cezary Kaliszyk | Fixed LF for one quantifier over 2 premises. | changeset | files | 
| Fri, 05 Mar 2010 09:41:22 +0100 | Cezary Kaliszyk | Trying to fix the proofs for the single existential... So far failed. | changeset | files | 
| Thu, 04 Mar 2010 18:57:23 +0100 | Cezary Kaliszyk | Lift distinct. | changeset | files | 
| 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. | changeset | files | 
| Thu, 04 Mar 2010 15:15:44 +0100 | Cezary Kaliszyk | Lift BV,FV,Permutations and injection :). | changeset | files | 
| 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. | changeset | files | 
| Thu, 04 Mar 2010 11:16:36 +0100 | Cezary Kaliszyk | A version that just leaves the supp/\supp goal. Obviously not true. | changeset | files | 
| Thu, 04 Mar 2010 10:59:52 +0100 | Cezary Kaliszyk | Prove symp and transp of weird without the supp /\ supp = {} assumption. | changeset | files | 
| Wed, 03 Mar 2010 17:51:47 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 03 Mar 2010 17:49:34 +0100 | Cezary Kaliszyk | Experiments with proving weird transp | changeset | files | 
| Wed, 03 Mar 2010 17:47:29 +0100 | Cezary Kaliszyk | Code for solving symp goals with multiple existentials. | changeset | files | 
| Wed, 03 Mar 2010 15:28:25 +0100 | Cezary Kaliszyk | reflp for multiple quantifiers. | changeset | files | 
| Wed, 03 Mar 2010 14:46:14 +0100 | Christian Urban | fixed mess in Test.thy | changeset | files | 
| Wed, 03 Mar 2010 14:22:58 +0100 | Cezary Kaliszyk | Fix eqvt for multiple quantifiers. | changeset | files | 
| Wed, 03 Mar 2010 12:48:05 +0100 | Christian Urban | only tuned | changeset | files | 
| Wed, 03 Mar 2010 12:47:06 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 03 Mar 2010 12:45:55 +0100 | Christian Urban | start of paper - does not compile yet | changeset | files | 
| Wed, 03 Mar 2010 11:50:25 +0100 | Christian Urban | added ACM style file for ICFP | changeset | files | 
| Wed, 03 Mar 2010 11:42:15 +0100 | Cezary Kaliszyk | weird eqvt | changeset | files | 
| Wed, 03 Mar 2010 10:39:43 +0100 | Cezary Kaliszyk | Add the supp intersection conditions. | changeset | files | 
| Tue, 02 Mar 2010 21:43:27 +0100 | Cezary Kaliszyk | Comment out the part that does not work with 2 quantifiers. | changeset | files | 
| Tue, 02 Mar 2010 21:10:04 +0100 | Cezary Kaliszyk | Fixes for the fv problem and alpha problem. | changeset | files | 
| Tue, 02 Mar 2010 20:14:21 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 02 Mar 2010 20:11:56 +0100 | Christian Urban | preliinary test about alpha-weirdo | changeset | files | 
| Tue, 02 Mar 2010 18:57:26 +0100 | Christian Urban | Another problem with permutations in alpha and possibly also in fv | changeset | files | 
| 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 | changeset | files | 
| Tue, 02 Mar 2010 19:48:44 +0100 | Cezary Kaliszyk | Some tests around Term4. Not sure how to fix the generated fv function. | changeset | files | 
| Tue, 02 Mar 2010 17:48:56 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 02 Mar 2010 17:48:41 +0100 | Cezary Kaliszyk | Porting from Lift to Parser; until defining the Quotient type. | changeset | files | 
| Tue, 02 Mar 2010 17:11:58 +0100 | Cezary Kaliszyk | Add image_eqvt and atom_eqvt to eqvt bases. | changeset | files | 
| Tue, 02 Mar 2010 17:11:19 +0100 | Cezary Kaliszyk | Include the raw eqvt lemmas. | changeset | files | 
| Tue, 02 Mar 2010 16:04:48 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 02 Mar 2010 16:03:19 +0100 | Christian Urban | added some more examples from Peter Sewell's bestiary | changeset | files | 
| Tue, 02 Mar 2010 15:13:00 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 02 Mar 2010 15:12:50 +0100 | Cezary Kaliszyk | Minor | changeset | files | 
| Tue, 02 Mar 2010 15:11:41 +0100 | Cezary Kaliszyk | Working bv_eqvt | changeset | files | 
| Tue, 02 Mar 2010 15:10:47 +0100 | Cezary Kaliszyk | Moving wrappers out of Lift. | changeset | files | 
| Tue, 02 Mar 2010 15:07:27 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 02 Mar 2010 15:05:50 +0100 | Christian Urban | added distinctness of perms | changeset | files | 
| Tue, 02 Mar 2010 15:05:35 +0100 | Christian Urban | updated (added lemma about commuting permutations) | changeset | files | 
| Tue, 02 Mar 2010 14:51:40 +0100 | Cezary Kaliszyk | Change type schemes to name set. | changeset | files | 
| Tue, 02 Mar 2010 14:24:57 +0100 | Cezary Kaliszyk | More fixes for new alpha, the whole lift script should now work again. | changeset | files | 
| Tue, 02 Mar 2010 13:28:54 +0100 | Cezary Kaliszyk | Length fix for nested recursions. | changeset | files | 
| Tue, 02 Mar 2010 12:28:07 +0100 | Cezary Kaliszyk | Fix equivp. | changeset | files | 
| Tue, 02 Mar 2010 11:04:49 +0100 | Cezary Kaliszyk | Fixed eqvt code. | changeset | files | 
| Tue, 02 Mar 2010 08:58:28 +0100 | Christian Urban | most tests work - the ones that do not I commented out | changeset | files | 
| Tue, 02 Mar 2010 08:49:04 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 02 Mar 2010 08:48:35 +0100 | Cezary Kaliszyk | Add a check of fv_functions. | changeset | files | 
| Tue, 02 Mar 2010 08:43:53 +0100 | Christian Urban | some tuning | changeset | files | 
| Tue, 02 Mar 2010 08:42:10 +0100 | Cezary Kaliszyk | Link calls to Raw permutations, FV definition and alpha_definition into the parser. | changeset | files | 
| Tue, 02 Mar 2010 06:43:09 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 02 Mar 2010 06:42:43 +0100 | Christian Urban | rawified the bind specs (ready to be used now) | changeset | files | 
| Mon, 01 Mar 2010 21:50:40 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 01 Mar 2010 21:50:24 +0100 | Cezary Kaliszyk | Trying to prove equivariance. | changeset | files | 
| Mon, 01 Mar 2010 19:23:08 +0100 | Christian Urban | modified for new binding format - hope it is the intended one | changeset | files | 
| Mon, 01 Mar 2010 16:55:41 +0100 | Christian Urban | further code-refactoring in the parser | changeset | files | 
| Mon, 01 Mar 2010 16:04:03 +0100 | Cezary Kaliszyk | The new alpha-equivalence and testing in Trm2 and Trm5. | changeset | files | 
| Mon, 01 Mar 2010 14:26:14 +0100 | Christian Urban | slight simplification of the raw-decl generation | changeset | files | 
| Mon, 01 Mar 2010 11:40:48 +0100 | Cezary Kaliszyk | Example that shows that current alpha is wrong. | changeset | files | 
| Mon, 01 Mar 2010 07:46:50 +0100 | Christian Urban | added example from my phd | changeset | files | 
| Sat, 27 Feb 2010 11:54:59 +0100 | Christian Urban | streamlined parser | changeset | files | 
| 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" | changeset | files | 
| Fri, 26 Feb 2010 18:21:39 +0100 | Cezary Kaliszyk | More about the general lifting procedure. | changeset | files | 
| Fri, 26 Feb 2010 16:22:47 +0100 | Cezary Kaliszyk | Update TODO | changeset | files | 
| Fri, 26 Feb 2010 16:15:03 +0100 | Cezary Kaliszyk | Progress with general lifting procedure. | changeset | files | 
| Fri, 26 Feb 2010 15:42:00 +0100 | Cezary Kaliszyk | RSP of perms can be shown in one go. | changeset | files | 
| Fri, 26 Feb 2010 15:10:55 +0100 | Cezary Kaliszyk | Change in signature of prove_const_rsp for general lifting. | changeset | files | 
| Fri, 26 Feb 2010 13:57:43 +0100 | Cezary Kaliszyk | Permutation and FV_Alpha interface change. | changeset | files | 
| 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. | changeset | files | 
| Thu, 25 Feb 2010 15:41:23 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Thu, 25 Feb 2010 15:40:09 +0100 | Cezary Kaliszyk | Preparing the generalized lifting procedure | changeset | files | 
| Thu, 25 Feb 2010 14:20:40 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 25 Feb 2010 14:20:10 +0100 | Christian Urban | added ott-example about Leroy96 | changeset | files | 
| Thu, 25 Feb 2010 14:14:40 +0100 | Cezary Kaliszyk | Forgot to add one file. | changeset | files | 
| Thu, 25 Feb 2010 14:14:08 +0100 | Cezary Kaliszyk | Split Terms into separate files and add them to tests. | changeset | files | 
| Thu, 25 Feb 2010 12:32:15 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Thu, 25 Feb 2010 12:30:50 +0100 | Cezary Kaliszyk | Move the eqvt code out of Terms and fixed induction for single-rule examples. | changeset | files | 
| Thu, 25 Feb 2010 12:24:37 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 25 Feb 2010 11:51:34 +0100 | Christian Urban | a few simplifications | changeset | files | 
| Thu, 25 Feb 2010 11:30:00 +0100 | Christian Urban | first attempt to make sense out of the core-haskell definition | changeset | files | 
| Thu, 25 Feb 2010 12:15:11 +0100 | Cezary Kaliszyk | Code for proving eqvt, still in Terms. | changeset | files | 
| Thu, 25 Feb 2010 09:41:14 +0100 | Cezary Kaliszyk | Use eqvt infrastructure. | changeset | files | 
| Thu, 25 Feb 2010 09:22:29 +0100 | Cezary Kaliszyk | Simple function eqvt code. | changeset | files | 
| Thu, 25 Feb 2010 08:40:52 +0100 | Christian Urban | added IsaMakefile...but so far included only a test for the parser | changeset | files | 
| Thu, 25 Feb 2010 07:57:17 +0100 | Christian Urban | moved Quot package to Attic (still compiles there with "isabelle make") | changeset | files | 
| Thu, 25 Feb 2010 07:48:57 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 25 Feb 2010 07:48:33 +0100 | Christian Urban | moved Nominal to "toplevel" | changeset | files | 
| Thu, 25 Feb 2010 07:05:52 +0100 | Cezary Kaliszyk | Export perm_frees. | changeset | files | 
| Wed, 24 Feb 2010 23:25:30 +0100 | Cezary Kaliszyk | Restructuring the code in Perm | changeset | files | 
| Wed, 24 Feb 2010 18:38:49 +0100 | Cezary Kaliszyk | Simplified and finised eqvt proofs for t1 and t5 | changeset | files | 
| Wed, 24 Feb 2010 17:42:52 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 24 Feb 2010 17:42:37 +0100 | Cezary Kaliszyk | Define lifted perms. | changeset | files | 
| Wed, 24 Feb 2010 17:32:43 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 24 Feb 2010 17:32:22 +0100 | Christian Urban | parsing and definition of raw datatype and bv-function work (not very beautiful) | changeset | files | 
| Wed, 24 Feb 2010 15:39:17 +0100 | Cezary Kaliszyk | With permute_rsp we can lift the instance proofs :). | changeset | files | 
| Wed, 24 Feb 2010 15:36:07 +0100 | Cezary Kaliszyk | Note the instance proofs, since they can be easily lifted. | changeset | files | 
| Wed, 24 Feb 2010 15:13:22 +0100 | Cezary Kaliszyk | More refactoring and removed references to the global simpset in Perm. | changeset | files | 
| 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. | changeset | files | 
| Wed, 24 Feb 2010 14:37:51 +0100 | Cezary Kaliszyk | Regularize finite support proof for trm1 | changeset | files | 
| Wed, 24 Feb 2010 14:09:34 +0100 | Cezary Kaliszyk | Made the fv-supp proof much more straightforward. | changeset | files | 
| Wed, 24 Feb 2010 12:06:55 +0100 | Cezary Kaliszyk | Regularize the proofs about finite support. | changeset | files | 
| Wed, 24 Feb 2010 11:28:34 +0100 | Cezary Kaliszyk | Respects of permute and constructors. | changeset | files | 
| Wed, 24 Feb 2010 11:03:30 +0100 | Cezary Kaliszyk | Generate fv_rsp automatically. | changeset | files | 
| Wed, 24 Feb 2010 10:59:31 +0100 | Cezary Kaliszyk | Define the constants automatically. | changeset | files | 
| Wed, 24 Feb 2010 10:47:41 +0100 | Cezary Kaliszyk | Rename also the lifted types to non-capital. | changeset | files | 
| Wed, 24 Feb 2010 10:44:38 +0100 | Cezary Kaliszyk | Use the infrastructure in LF. Much shorter :). | changeset | files | 
| Wed, 24 Feb 2010 10:38:45 +0100 | Cezary Kaliszyk | Final synchronization of names. | changeset | files | 
| Wed, 24 Feb 2010 10:25:59 +0100 | Cezary Kaliszyk | LF renaming part 3 (proper names of alpha equvalences) | changeset | files | 
| Wed, 24 Feb 2010 10:08:54 +0100 | Cezary Kaliszyk | LF renaming part 2 (proper fv functions) | changeset | files | 
| Wed, 24 Feb 2010 09:58:44 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 24 Feb 2010 09:58:12 +0100 | Cezary Kaliszyk | LF renaming part1. | changeset | files | 
| Wed, 24 Feb 2010 09:56:32 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 24 Feb 2010 09:56:12 +0100 | Christian Urban | parsing of function definitions almost works now; still an error with undefined constants | changeset | files | 
| Tue, 23 Feb 2010 18:28:48 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 23 Feb 2010 18:27:32 +0100 | Cezary Kaliszyk | rsp for bv; the only issue is that it requires an appropriate induction principle. | changeset | files | 
| Tue, 23 Feb 2010 16:32:04 +0100 | Christian Urban | merged | changeset | files | 
| 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 | changeset | files | 
| Tue, 23 Feb 2010 16:12:30 +0100 | Cezary Kaliszyk | rsp infrastructure. | changeset | files | 
| Tue, 23 Feb 2010 14:20:42 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 23 Feb 2010 14:19:44 +0100 | Cezary Kaliszyk | Progress towards automatic rsp of constants and fv. | changeset | files | 
| Tue, 23 Feb 2010 13:33:01 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 23 Feb 2010 13:32:35 +0100 | Christian Urban | "raw"-ified the term-constructors and types given in the specification | changeset | files | 
| Tue, 23 Feb 2010 12:49:45 +0100 | Cezary Kaliszyk | Looking at proving the rsp rules automatically. | changeset | files | 
| Tue, 23 Feb 2010 11:56:47 +0100 | Cezary Kaliszyk | Minor beutification. | changeset | files | 
| Tue, 23 Feb 2010 11:22:06 +0100 | Cezary Kaliszyk | Define the quotient from ML | changeset | files | 
| Tue, 23 Feb 2010 10:47:14 +0100 | Cezary Kaliszyk | All works in LF but will require renaming. | changeset | files | 
| Tue, 23 Feb 2010 09:34:41 +0100 | Cezary Kaliszyk | Reordering in LF. | changeset | files | 
| Tue, 23 Feb 2010 09:31:59 +0100 | Cezary Kaliszyk | Fixes for auxiliary datatypes. | changeset | files | 
| Mon, 22 Feb 2010 18:09:44 +0100 | Cezary Kaliszyk | Fixed pseudo_injectivity for trm4 | changeset | files | 
| Mon, 22 Feb 2010 17:19:28 +0100 | Cezary Kaliszyk | Testing auto equivp code. | changeset | files | 
| Mon, 22 Feb 2010 16:44:58 +0100 | Cezary Kaliszyk | A tactic for final equivp | changeset | files | 
| Mon, 22 Feb 2010 16:16:04 +0100 | Cezary Kaliszyk | More equivp infrastructure. | changeset | files | 
| Mon, 22 Feb 2010 15:41:30 +0100 | Cezary Kaliszyk | tactify transp | changeset | files | 
| Mon, 22 Feb 2010 15:09:53 +0100 | Cezary Kaliszyk | export the reflp and symp tacs. | changeset | files | 
| Mon, 22 Feb 2010 15:03:48 +0100 | Cezary Kaliszyk | Generalize atom_trans and atom_sym. | changeset | files | 
| Mon, 22 Feb 2010 14:50:53 +0100 | Cezary Kaliszyk | Some progress about transp | changeset | files | 
| Mon, 22 Feb 2010 13:41:13 +0100 | Cezary Kaliszyk | alpha-symmetric addons. | changeset | files | 
| Mon, 22 Feb 2010 12:12:32 +0100 | Cezary Kaliszyk | alpha reflexivity | changeset | files | 
| Mon, 22 Feb 2010 10:57:39 +0100 | Cezary Kaliszyk | Renaming. | changeset | files | 
| Mon, 22 Feb 2010 10:39:05 +0100 | Cezary Kaliszyk | Added missing description. | changeset | files | 
| Mon, 22 Feb 2010 10:16:13 +0100 | Cezary Kaliszyk | Added Brian's suggestion. | changeset | files | 
| Mon, 22 Feb 2010 09:55:43 +0100 | Cezary Kaliszyk | Update TODO | changeset | files | 
| Sun, 21 Feb 2010 22:39:11 +0100 | Cezary Kaliszyk | Removed bindings 'in itself' where possible. | changeset | files | 
| Sat, 20 Feb 2010 06:31:03 +0100 | Cezary Kaliszyk | Some adaptation | changeset | files | 
| Fri, 19 Feb 2010 17:50:43 +0100 | Cezary Kaliszyk | proof cleaning and standardizing. | changeset | files | 
| Fri, 19 Feb 2010 16:45:24 +0100 | Cezary Kaliszyk | Automatic production and proving of pseudo-injectivity. | changeset | files | 
| Fri, 19 Feb 2010 12:05:58 +0100 | Cezary Kaliszyk | Experiments for the pseudo-injectivity tactic. | changeset | files | 
| Fri, 19 Feb 2010 10:26:38 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Fri, 19 Feb 2010 10:17:35 +0100 | Cezary Kaliszyk | Constructing alpha_inj goal. | changeset | files | 
| Thu, 18 Feb 2010 23:07:52 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 18 Feb 2010 23:07:28 +0100 | Christian Urban | start work with the parser | changeset | files | 
| 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. | changeset | files | 
| Thu, 18 Feb 2010 15:03:09 +0100 | Cezary Kaliszyk | First (non-working) version of alpha-equivalence | changeset | files | 
| Thu, 18 Feb 2010 13:36:38 +0100 | Cezary Kaliszyk | Description of the fv procedure. | changeset | files | 
| Thu, 18 Feb 2010 12:06:59 +0100 | Cezary Kaliszyk | Testing auto constant lifting. | changeset | files | 
| Thu, 18 Feb 2010 11:28:20 +0100 | Cezary Kaliszyk | Fix for new Isabelle (primrec) | changeset | files | 
| Thu, 18 Feb 2010 11:19:16 +0100 | Cezary Kaliszyk | Automatic lifting of constants. | changeset | files | 
| Thu, 18 Feb 2010 10:01:48 +0100 | Cezary Kaliszyk | Changed back to original version of trm5 | changeset | files | 
| Thu, 18 Feb 2010 10:00:58 +0100 | Cezary Kaliszyk | The alternate version of trm5 with additional binding. All proofs work the same. | changeset | files | 
| Thu, 18 Feb 2010 09:46:38 +0100 | Cezary Kaliszyk | Code for handling atom sets. | changeset | files | 
| Thu, 18 Feb 2010 08:43:13 +0100 | Cezary Kaliszyk | Replace Terms by Terms2. | changeset | files | 
| Thu, 18 Feb 2010 08:37:45 +0100 | Cezary Kaliszyk | Fixed proofs in Terms2 and found a mistake in Terms. | changeset | files | 
| Wed, 17 Feb 2010 17:51:35 +0100 | Cezary Kaliszyk | Terms2 with bindings for binders synchronized with bindings they are used in. | changeset | files | 
| Wed, 17 Feb 2010 17:29:26 +0100 | Cezary Kaliszyk | Cleaning of proofs in Terms. | changeset | files | 
| Wed, 17 Feb 2010 16:22:16 +0100 | Cezary Kaliszyk | Testing Fv | changeset | files | 
| Wed, 17 Feb 2010 15:52:08 +0100 | Cezary Kaliszyk | Fix the strong induction principle. | changeset | files | 
| Wed, 17 Feb 2010 15:45:03 +0100 | Cezary Kaliszyk | Reorder | changeset | files | 
| Wed, 17 Feb 2010 15:28:50 +0100 | Cezary Kaliszyk | Add bindings of recursive types by free_variables. | changeset | files | 
| Wed, 17 Feb 2010 15:20:22 +0100 | Cezary Kaliszyk | Bindings adapted to multiple defined datatypes. | changeset | files | 
| Wed, 17 Feb 2010 15:00:04 +0100 | Cezary Kaliszyk | Reorganization | changeset | files | 
| Wed, 17 Feb 2010 14:44:32 +0100 | Cezary Kaliszyk | Now should work. | changeset | files | 
| Wed, 17 Feb 2010 14:35:06 +0100 | Cezary Kaliszyk | Some optimizations and fixes. | changeset | files | 
| Wed, 17 Feb 2010 14:17:02 +0100 | Cezary Kaliszyk | Simplified format of bindings. | changeset | files | 
| Wed, 17 Feb 2010 13:56:31 +0100 | Cezary Kaliszyk | Tested the Perm code; works everywhere in Terms. | changeset | files | 
| Wed, 17 Feb 2010 13:54:35 +0100 | Cezary Kaliszyk | Wrapped the permutation code. | changeset | files | 
| Wed, 17 Feb 2010 10:20:26 +0100 | Cezary Kaliszyk | Description of intended bindings. | changeset | files | 
| Wed, 17 Feb 2010 10:12:01 +0100 | Cezary Kaliszyk | Code for generating the fv function, no bindings yet. | changeset | files | 
| Wed, 17 Feb 2010 09:27:02 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 17 Feb 2010 09:26:49 +0100 | Cezary Kaliszyk | indent | changeset | files | 
| Wed, 17 Feb 2010 09:26:38 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 17 Feb 2010 09:26:10 +0100 | Cezary Kaliszyk | Simplifying perm_eq | changeset | files | 
| Tue, 16 Feb 2010 15:13:14 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 16 Feb 2010 15:12:31 +0100 | Cezary Kaliszyk | indenting | changeset | files | 
| Tue, 16 Feb 2010 15:12:49 +0100 | Cezary Kaliszyk | Minor | changeset | files | 
| Tue, 16 Feb 2010 14:57:39 +0100 | Cezary Kaliszyk | Merge | changeset | files | 
| Tue, 16 Feb 2010 14:57:22 +0100 | Cezary Kaliszyk | Ported Stefan's permutation code, still needs some localizing. | changeset | files | 
| Mon, 15 Feb 2010 16:54:09 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 15 Feb 2010 16:53:51 +0100 | Cezary Kaliszyk | Removed varifyT. | changeset | files | 
| Mon, 15 Feb 2010 17:02:46 +0100 | Christian Urban | merged | changeset | files | 
| Mon, 15 Feb 2010 17:02:26 +0100 | Christian Urban | 2-spaces rule (where it makes sense) | changeset | files | 
| Mon, 15 Feb 2010 16:52:32 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 15 Feb 2010 16:51:30 +0100 | Cezary Kaliszyk | Fixed the definition of less and finished the missing proof. | changeset | files | 
| Mon, 15 Feb 2010 16:50:11 +0100 | Christian Urban | further tuning | changeset | files | 
| Mon, 15 Feb 2010 16:37:48 +0100 | Christian Urban | small tuning | changeset | files | 
| 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 | changeset | files | 
| Mon, 15 Feb 2010 14:58:03 +0100 | Cezary Kaliszyk | der_bname -> derived_bname | changeset | files | 
| Mon, 15 Feb 2010 14:51:17 +0100 | Cezary Kaliszyk | Names of files. | changeset | files | 
| Mon, 15 Feb 2010 14:28:03 +0100 | Cezary Kaliszyk | Finished introducing the binding. | changeset | files | 
| Mon, 15 Feb 2010 13:40:03 +0100 | Cezary Kaliszyk | Synchronize the commands. | changeset | files | 
| Mon, 15 Feb 2010 12:23:02 +0100 | Cezary Kaliszyk | Passing the binding to quotient_def | changeset | files | 
| Mon, 15 Feb 2010 12:15:14 +0100 | Cezary Kaliszyk | Added a binding to the parser. | changeset | files | 
| Mon, 15 Feb 2010 10:25:17 +0100 | Cezary Kaliszyk | Second inline | changeset | files | 
| Mon, 15 Feb 2010 10:11:26 +0100 | Cezary Kaliszyk | remove one-line wrapper. | changeset | files | 
| Fri, 12 Feb 2010 16:27:25 +0100 | Cezary Kaliszyk | Undid the read_terms change; now compiles. | changeset | files | 
| Fri, 12 Feb 2010 16:06:09 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Fri, 12 Feb 2010 16:04:10 +0100 | Cezary Kaliszyk | renamed 'as' to 'is' everywhere. | changeset | files | 
| Fri, 12 Feb 2010 15:50:43 +0100 | Cezary Kaliszyk | "is" defined as the keyword | changeset | files | 
| Fri, 12 Feb 2010 15:06:20 +0100 | Christian Urban | moved "strange" lemma to quotient_tacs; marked a number of lemmas as unused; tuned | changeset | files | 
| Fri, 12 Feb 2010 12:06:09 +0100 | Cezary Kaliszyk | The lattice instantiations are gone from Isabelle/Main, so | changeset | files | 
| Thu, 11 Feb 2010 17:58:06 +0100 | Cezary Kaliszyk | the lam/bla example. | changeset | files | 
| Thu, 11 Feb 2010 16:54:04 +0100 | Cezary Kaliszyk | Finished a working foo/bar. | changeset | files | 
| Thu, 11 Feb 2010 16:05:15 +0100 | Cezary Kaliszyk | fv_foo is not regular. | changeset | files | 
| Thu, 11 Feb 2010 15:08:45 +0100 | Cezary Kaliszyk | Testing foo/bar | changeset | files | 
| Thu, 11 Feb 2010 14:23:26 +0100 | Cezary Kaliszyk | Even when bv = fv it still doesn't lift. | changeset | files | 
| Thu, 11 Feb 2010 14:02:34 +0100 | Cezary Kaliszyk | Added the missing syntax file | changeset | files | 
| Thu, 11 Feb 2010 14:00:00 +0100 | Cezary Kaliszyk | Notation available locally | changeset | files | 
| Thu, 11 Feb 2010 10:06:02 +0100 | Cezary Kaliszyk | Main renaming + fixes for new Isabelle in IntEx2. | changeset | files | 
| Thu, 11 Feb 2010 09:23:59 +0100 | Cezary Kaliszyk | Merging QuotBase into QuotMain. | changeset | files | 
| Wed, 10 Feb 2010 21:39:40 +0100 | Christian Urban | removed dead code | changeset | files | 
| Wed, 10 Feb 2010 20:35:54 +0100 | Christian Urban | cleaned a bit | changeset | files | 
| Wed, 10 Feb 2010 17:22:18 +0100 | Cezary Kaliszyk | lowercase locale | changeset | files | 
| Wed, 10 Feb 2010 17:10:52 +0100 | Cezary Kaliszyk | hg-added the added file. | changeset | files | 
| Wed, 10 Feb 2010 17:02:29 +0100 | Cezary Kaliszyk | Changes from Makarius's code review + some noticed fixes. | changeset | files | 
| Wed, 10 Feb 2010 12:30:26 +0100 | Cezary Kaliszyk | example with a respectful bn function defined over the type itself | changeset | files | 
| Wed, 10 Feb 2010 11:53:15 +0100 | Cezary Kaliszyk | Finishe the renaming. | changeset | files | 
| Wed, 10 Feb 2010 11:39:22 +0100 | Cezary Kaliszyk | Another mistake found with OTT. | changeset | files | 
| Wed, 10 Feb 2010 11:31:53 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 10 Feb 2010 11:31:43 +0100 | Cezary Kaliszyk | Fixed rbv6, when translating to OTT. | changeset | files | 
| Wed, 10 Feb 2010 11:27:49 +0100 | Cezary Kaliszyk | Some cleaning of proofs. | changeset | files | 
| Wed, 10 Feb 2010 11:11:06 +0100 | Christian Urban | merged again | changeset | files | 
| Wed, 10 Feb 2010 11:10:44 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 10 Feb 2010 11:09:30 +0100 | Cezary Kaliszyk | more minor space and bracket modifications. | changeset | files | 
| Wed, 10 Feb 2010 10:55:14 +0100 | Cezary Kaliszyk | More changes according to the standards. | changeset | files | 
| Wed, 10 Feb 2010 10:36:47 +0100 | Cezary Kaliszyk | A concrete example, with a proof that rbv is not regular and | changeset | files | 
| Tue, 09 Feb 2010 19:08:08 +0100 | Christian Urban | proper declaration of types and terms during parsing (removes the varifyT when storing data) | changeset | files | 
| Tue, 09 Feb 2010 17:26:28 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 09 Feb 2010 17:26:08 +0100 | Christian Urban | slight correction | changeset | files | 
| Tue, 09 Feb 2010 17:26:00 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 09 Feb 2010 17:24:08 +0100 | Cezary Kaliszyk | More about trm6 | changeset | files | 
| Tue, 09 Feb 2010 17:17:06 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 09 Feb 2010 17:05:07 +0100 | Cezary Kaliszyk | the specifications of the respects. | changeset | files | 
| Tue, 09 Feb 2010 16:44:06 +0100 | Cezary Kaliszyk | trm6 with the 'Foo' constructor. | changeset | files | 
| Tue, 09 Feb 2010 16:10:08 +0100 | Cezary Kaliszyk | removing unnecessary brackets | changeset | files | 
| Tue, 09 Feb 2010 15:55:58 +0100 | Cezary Kaliszyk | More indentation cleaning. | changeset | files | 
| Tue, 09 Feb 2010 15:43:39 +0100 | Cezary Kaliszyk | 'exc' -> 'exn' and more name and space cleaning. | changeset | files | 
| Tue, 09 Feb 2010 15:36:23 +0100 | Cezary Kaliszyk | Fully qualified exception names. | changeset | files | 
| Tue, 09 Feb 2010 15:28:30 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 09 Feb 2010 15:28:15 +0100 | Cezary Kaliszyk | More indentation, names and todo cleaning in the quotient package | changeset | files | 
| Tue, 09 Feb 2010 15:20:52 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 09 Feb 2010 15:20:40 +0100 | Christian Urban | a few more attempts to show the equivalence between old and new way of defining alpha-equivalence | changeset | files | 
| Tue, 09 Feb 2010 11:40:32 +0100 | Christian Urban | minor tuning | changeset | files | 
| Tue, 09 Feb 2010 14:32:37 +0100 | Cezary Kaliszyk | Explicitly marked what is bound. | changeset | files | 
| Tue, 09 Feb 2010 12:22:00 +0100 | Cezary Kaliszyk | Cleaning and updating in Terms. | changeset | files | 
| Tue, 09 Feb 2010 11:22:34 +0100 | Cezary Kaliszyk | Looking at the trm2 example | changeset | files | 
| Tue, 09 Feb 2010 10:48:42 +0100 | Cezary Kaliszyk | Fixed pattern matching, now the test in Abs works correctly. | changeset | files | 
| Mon, 08 Feb 2010 13:50:52 +0100 | Christian Urban | added a test case | changeset | files | 
| Mon, 08 Feb 2010 13:13:20 +0100 | Christian Urban | merged | changeset | files | 
| Mon, 08 Feb 2010 13:12:55 +0100 | Christian Urban | moved some lemmas to Nominal; updated all files | changeset | files | 
| Mon, 08 Feb 2010 13:04:29 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 08 Feb 2010 13:04:13 +0100 | Cezary Kaliszyk | Comments. | changeset | files | 
| Mon, 08 Feb 2010 11:56:22 +0100 | Christian Urban | slightly tuned | changeset | files | 
| Mon, 08 Feb 2010 11:41:25 +0100 | Cezary Kaliszyk | Proper context fixes lifting inside instantiations. | changeset | files | 
| Mon, 08 Feb 2010 10:47:19 +0100 | Cezary Kaliszyk | Fixed the context import/export and simplified LFex. | changeset | files | 
| Mon, 08 Feb 2010 06:27:20 +0100 | Christian Urban | added 2 papers about core haskell | changeset | files | 
| Sun, 07 Feb 2010 10:20:29 +0100 | Christian Urban | fixed lemma name | changeset | files | 
| Sun, 07 Feb 2010 10:16:21 +0100 | Christian Urban | updated to latest Nominal2 | changeset | files | 
| Sat, 06 Feb 2010 12:58:56 +0100 | Christian Urban | minor | changeset | files | 
| Sat, 06 Feb 2010 10:04:56 +0100 | Christian Urban | some tuning | changeset | files | 
| Fri, 05 Feb 2010 15:17:21 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Fri, 05 Feb 2010 14:52:27 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Fri, 05 Feb 2010 10:32:21 +0100 | Cezary Kaliszyk | Fixes for Bex1 removal. | changeset | files | 
| Fri, 05 Feb 2010 15:09:49 +0100 | Cezary Kaliszyk | Cleaned Terms using [lifted] and found a workaround for the instantiation problem. | changeset | files | 
| Fri, 05 Feb 2010 11:37:18 +0100 | Cezary Kaliszyk | A procedure that properly instantiates the types too. | changeset | files | 
| Fri, 05 Feb 2010 11:28:49 +0100 | Cezary Kaliszyk | More code abstracted away | changeset | files | 
| Fri, 05 Feb 2010 11:19:21 +0100 | Cezary Kaliszyk | A bit more intelligent and cleaner code. | changeset | files | 
| Fri, 05 Feb 2010 11:09:43 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Fri, 05 Feb 2010 10:45:49 +0100 | Cezary Kaliszyk | A proper version of the attribute | changeset | files | 
| Fri, 05 Feb 2010 09:06:49 +0100 | Christian Urban | merged | changeset | files | 
| Fri, 05 Feb 2010 09:06:27 +0100 | Christian Urban | eqvts and eqvts_raw are separate thm-lists; otherwise permute_eqvt is problematic as it causes looks in eqvts | changeset | files | 
| Thu, 04 Feb 2010 18:09:20 +0100 | Cezary Kaliszyk | The automatic lifting translation function, still with dummy types, | changeset | files | 
| Thu, 04 Feb 2010 17:58:23 +0100 | Cezary Kaliszyk | Quotdata_dest needed for lifting theorem translation. | changeset | files | 
| Thu, 04 Feb 2010 17:39:04 +0100 | Christian Urban | fixed (permute_eqvt in eqvts makes this simpset always looping) | changeset | files | 
| Thu, 04 Feb 2010 15:19:24 +0100 | Christian Urban | rollback of the test | changeset | files | 
| Thu, 04 Feb 2010 15:16:34 +0100 | Christian Urban | linked versions - instead of copies | changeset | files | 
| Thu, 04 Feb 2010 14:55:52 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 04 Feb 2010 14:55:21 +0100 | Christian Urban | restored the old behaviour of having an eqvts list; the transformed theorems are stored in eqvts_raw | changeset | files | 
| Wed, 03 Feb 2010 18:28:50 +0100 | Cezary Kaliszyk | More let-rec experiments | changeset | files | 
| Wed, 03 Feb 2010 17:36:25 +0100 | Christian Urban | proposal for an alpha equivalence | changeset | files | 
| Wed, 03 Feb 2010 15:17:29 +0100 | Cezary Kaliszyk | Lets different. | changeset | files | 
| Wed, 03 Feb 2010 14:39:19 +0100 | Cezary Kaliszyk | Simplified the proof. | changeset | files | 
| Wed, 03 Feb 2010 14:36:48 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 03 Feb 2010 14:36:22 +0100 | Christian Urban | proved that bv for lists respects alpha for terms | changeset | files | 
| Wed, 03 Feb 2010 14:28:00 +0100 | Cezary Kaliszyk | Finished remains on the let proof. | changeset | files | 
| Wed, 03 Feb 2010 14:22:25 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 03 Feb 2010 14:19:53 +0100 | Cezary Kaliszyk | Lets are ok. | changeset | files | 
| Wed, 03 Feb 2010 14:15:07 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 03 Feb 2010 14:12:50 +0100 | Christian Urban | added type-scheme example | changeset | files | 
| Wed, 03 Feb 2010 13:00:37 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 03 Feb 2010 13:00:07 +0100 | Cezary Kaliszyk | Definitions for trm5 | changeset | files | 
| Wed, 03 Feb 2010 12:58:02 +0100 | Christian Urban | another adaptation for the eqvt-change | changeset | files | 
| Wed, 03 Feb 2010 12:45:06 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 03 Feb 2010 12:44:29 +0100 | Christian Urban | fixed proofs that broke because of eqvt | changeset | files | 
| Wed, 03 Feb 2010 12:34:53 +0100 | Cezary Kaliszyk | Minor fix. | changeset | files | 
| Wed, 03 Feb 2010 12:34:01 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 03 Feb 2010 12:29:45 +0100 | Cezary Kaliszyk | alpha5 pseudo-injective | changeset | files | 
| Wed, 03 Feb 2010 12:31:58 +0100 | Christian Urban | fixed proofs in Abs.thy | changeset | files | 
| Wed, 03 Feb 2010 12:13:22 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 03 Feb 2010 12:06:10 +0100 | Christian Urban | added a first eqvt_tac which pushes permutations inside terms | changeset | files | 
| Wed, 03 Feb 2010 12:11:23 +0100 | Cezary Kaliszyk | The alpha-equivalence relation for let-rec. Not sure if correct... | changeset | files | 
| Wed, 03 Feb 2010 11:47:37 +0100 | Cezary Kaliszyk | Starting with a let-rec example. | changeset | files | 
| Wed, 03 Feb 2010 11:21:34 +0100 | Cezary Kaliszyk | Minor | changeset | files | 
| Wed, 03 Feb 2010 10:50:24 +0100 | Cezary Kaliszyk | Some cleaning and eqvt proof | changeset | files | 
| Wed, 03 Feb 2010 09:25:21 +0100 | Cezary Kaliszyk | The trm1_support lemma explicitly and stated a strong induction principle. | changeset | files | 
| Wed, 03 Feb 2010 08:32:24 +0100 | Cezary Kaliszyk | More ingredients in Terms. | changeset | files | 
| Tue, 02 Feb 2010 17:10:42 +0100 | Cezary Kaliszyk | Finished the supp_fv proof; first proof that analyses the structure of 'Let' :) | changeset | files | 
| Tue, 02 Feb 2010 16:51:00 +0100 | Cezary Kaliszyk | More in Terms | changeset | files | 
| Tue, 02 Feb 2010 14:55:07 +0100 | Cezary Kaliszyk | First experiments in Terms. | changeset | files | 
| Tue, 02 Feb 2010 13:10:46 +0100 | Cezary Kaliszyk | LF ported to alpha_gen, equivp solved and one of the missing proofs in support<-> fv solved. Still some supp properties left. | changeset | files | 
| Tue, 02 Feb 2010 12:48:12 +0100 | Cezary Kaliszyk | Disambiguating the syntax. | changeset | files | 
| Tue, 02 Feb 2010 12:36:01 +0100 | Cezary Kaliszyk | Minor uncommited changes from LamEx2. | changeset | files | 
| Tue, 02 Feb 2010 11:56:37 +0100 | Cezary Kaliszyk | Some equivariance machinery that comes useful in LF. | changeset | files | 
| Tue, 02 Feb 2010 11:23:17 +0100 | Cezary Kaliszyk | Generalized the eqvt proof for single binders. | changeset | files | 
| Tue, 02 Feb 2010 10:43:48 +0100 | Cezary Kaliszyk | With induct instead of induct_tac, just one induction is sufficient. | changeset | files | 
| Tue, 02 Feb 2010 10:20:54 +0100 | Cezary Kaliszyk | General alpha_gen_trans for one-variable abstraction. | changeset | files | 
| Tue, 02 Feb 2010 09:51:39 +0100 | Cezary Kaliszyk | With unfolding Rep/Abs_eqvt no longer needed. | changeset | files | 
| Tue, 02 Feb 2010 08:16:34 +0100 | Cezary Kaliszyk | Lam2 finished apart from Rep_eqvt. | changeset | files | 
| Mon, 01 Feb 2010 20:02:44 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 01 Feb 2010 16:05:59 +0100 | Cezary Kaliszyk | All should be ok now. | changeset | files | 
| Mon, 01 Feb 2010 18:57:39 +0100 | Christian Urban | repaired according to changes in Abs.thy | changeset | files | 
| Mon, 01 Feb 2010 18:57:20 +0100 | Christian Urban | added a single-binder alpha equivalence; showed one half of the equivalence proof between general and single binder case | changeset | files | 
| Mon, 01 Feb 2010 16:46:07 +0100 | Christian Urban | cleaned | changeset | files | 
| Mon, 01 Feb 2010 16:23:47 +0100 | Christian Urban | updated from huffman | changeset | files | 
| Mon, 01 Feb 2010 16:13:24 +0100 | Christian Urban | updated from nominal-huffman | changeset | files | 
| Mon, 01 Feb 2010 15:57:37 +0100 | Cezary Kaliszyk | Fixed wrong rename. | changeset | files | 
| Mon, 01 Feb 2010 15:46:25 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 01 Feb 2010 15:45:40 +0100 | Cezary Kaliszyk | Lambda based on alpha_gen, under construction. | changeset | files | 
| Mon, 01 Feb 2010 15:32:20 +0100 | Christian Urban | updated from huffman - repo | changeset | files | 
| Mon, 01 Feb 2010 13:00:01 +0100 | Christian Urban | renamed Abst/abst to Abs/abs | changeset | files | 
| Mon, 01 Feb 2010 12:48:18 +0100 | Christian Urban | got rid of RAbst type - is now just pairs | changeset | files | 
| Mon, 01 Feb 2010 12:06:46 +0100 | Cezary Kaliszyk | Monotonicity of ~~gen, needed for using it in inductive definitions. | changeset | files | 
| Mon, 01 Feb 2010 11:39:59 +0100 | Cezary Kaliszyk | The current state of fv vs supp proofs in LF. | changeset | files | 
| Mon, 01 Feb 2010 11:16:31 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 01 Feb 2010 11:16:13 +0100 | Cezary Kaliszyk | More proofs in the LF example. | changeset | files | 
| Mon, 01 Feb 2010 11:00:51 +0100 | Christian Urban | merged | changeset | files | 
| Mon, 01 Feb 2010 10:00:03 +0100 | Christian Urban | slight tuning | changeset | files | 
| Mon, 01 Feb 2010 09:47:46 +0100 | Christian Urban | renamed function according to the name of the constant | changeset | files | 
| Mon, 01 Feb 2010 09:04:22 +0100 | Christian Urban | fixed problem with Bex1_rel renaming | changeset | files | 
| Mon, 01 Feb 2010 09:56:32 +0100 | Cezary Kaliszyk | Ported LF to the generic lambda and solved the simpler _supp cases. | changeset | files | 
| Sat, 30 Jan 2010 12:12:52 +0100 | Christian Urban | merged | changeset | files | 
| Sat, 30 Jan 2010 11:44:25 +0100 | Christian Urban | introduced a generic alpha (but not sure whether it is helpful) | changeset | files | 
| Fri, 29 Jan 2010 19:42:07 +0100 | Cezary Kaliszyk | More in the LF example in the new nominal way, all is clear until support. | changeset | files | 
| Fri, 29 Jan 2010 13:47:05 +0100 | Cezary Kaliszyk | Fixed the induction problem + some more proofs. | changeset | files | 
| Fri, 29 Jan 2010 12:16:08 +0100 | Cezary Kaliszyk | equivariance of rfv and alpha. | changeset | files | 
| Fri, 29 Jan 2010 10:13:07 +0100 | Cezary Kaliszyk | Added the experiments with fun and function. | changeset | files | 
| Fri, 29 Jan 2010 07:09:52 +0100 | Christian Urban | now also final step is proved - the supp of lambdas is now completely characterised | changeset | files | 
| Fri, 29 Jan 2010 00:22:00 +0100 | Christian Urban | the supp of a lambda can now be characterised, *provided* the notion of free variables coincides with support on lambda terms | changeset | files | 
| Thu, 28 Jan 2010 23:47:02 +0100 | Christian Urban | improved the proof slightly by defining alpha as a function and completely characterised the equality between two abstractions | changeset | files | 
| Thu, 28 Jan 2010 23:36:58 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 28 Jan 2010 23:36:38 +0100 | Christian Urban | general abstraction operator and complete characterisation of its support and freshness | changeset | files | 
| Thu, 28 Jan 2010 19:23:55 +0100 | Cezary Kaliszyk | Ported existing part of LF to new permutations and alphas. | changeset | files | 
| Thu, 28 Jan 2010 15:47:35 +0100 | Christian Urban | attempt of a general abstraction operator | changeset | files | 
| Thu, 28 Jan 2010 14:20:26 +0100 | Christian Urban | attempt to prove equivalence between alpha definitions | changeset | files | 
| Thu, 28 Jan 2010 12:28:50 +0100 | Cezary Kaliszyk | End of renaming. | changeset | files | 
| Thu, 28 Jan 2010 12:25:38 +0100 | Cezary Kaliszyk | Minor when looking at lam.distinct and lam.inject | changeset | files | 
| Thu, 28 Jan 2010 12:24:49 +0100 | Cezary Kaliszyk | Renamed Bexeq to Bex1_rel | changeset | files | 
| Thu, 28 Jan 2010 10:52:10 +0100 | Cezary Kaliszyk | Substracting bounds from free variables. | changeset | files | 
| Thu, 28 Jan 2010 10:26:36 +0100 | Cezary Kaliszyk | Improper interface for datatype and function packages and proper interface lateron. | changeset | files | 
| Thu, 28 Jan 2010 09:28:20 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 28 Jan 2010 09:28:06 +0100 | Christian Urban | minor | changeset | files | 
| Thu, 28 Jan 2010 01:24:09 +0100 | Christian Urban | test about supp/freshness for lam (old proofs work in principle - for single binders) | changeset | files | 
| Thu, 28 Jan 2010 08:13:39 +0100 | Cezary Kaliszyk | Recommited the changes for nitpick | changeset | files | 
| Wed, 27 Jan 2010 18:26:01 +0100 | Cezary Kaliszyk | Correct types which fixes the printing. | changeset | files | 
| Wed, 27 Jan 2010 18:06:14 +0100 | Cezary Kaliszyk | fv for subterms | changeset | files | 
| Wed, 27 Jan 2010 17:39:13 +0100 | Cezary Kaliszyk | Fix the problem with later examples. Maybe need to go back to textual specifications. | changeset | files | 
| Wed, 27 Jan 2010 17:18:30 +0100 | Cezary Kaliszyk | Some processing of variables in constructors to get free variables. | changeset | files | 
| Wed, 27 Jan 2010 16:40:16 +0100 | Cezary Kaliszyk | Parsing of the input as terms and types, and passing them as such to the function package. | changeset | files | 
| Wed, 27 Jan 2010 16:07:49 +0100 | Cezary Kaliszyk | Undid the parsing, as it is not possible with thy->lthy interaction. | changeset | files | 
| Wed, 27 Jan 2010 14:57:11 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 27 Jan 2010 14:56:58 +0100 | Cezary Kaliszyk | Some cleaning of thy vs lthy vs context. | changeset | files | 
| Wed, 27 Jan 2010 14:06:34 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 27 Jan 2010 14:06:17 +0100 | Christian Urban | tuned comment | changeset | files | 
| Wed, 27 Jan 2010 14:05:42 +0100 | Christian Urban | completely ported | changeset | files | 
| Wed, 27 Jan 2010 13:44:05 +0100 | Cezary Kaliszyk | Another string in the specification. | changeset | files | 
| Wed, 27 Jan 2010 13:32:28 +0100 | Cezary Kaliszyk | Variable takes a 'name'. | changeset | files | 
| Wed, 27 Jan 2010 12:21:40 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 27 Jan 2010 12:19:58 +0100 | Cezary Kaliszyk | When commenting discovered a missing case of Babs->Abs regularization. | changeset | files | 
| Wed, 27 Jan 2010 12:19:21 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 27 Jan 2010 12:19:00 +0100 | Christian Urban | mostly ported Terms.thy to new Nominal | changeset | files | 
| Wed, 27 Jan 2010 12:06:43 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 27 Jan 2010 12:06:24 +0100 | Cezary Kaliszyk | Commenting regularize | changeset | files | 
| Wed, 27 Jan 2010 11:48:04 +0100 | Christian Urban | very rough example file for how nominal2 specification can be parsed | changeset | files | 
| Wed, 27 Jan 2010 11:31:16 +0100 | Christian Urban | reordered cases in regularize (will be merged into two cases) | changeset | files | 
| Wed, 27 Jan 2010 08:41:42 +0100 | Christian Urban | use of equiv_relation_chk in quotient_term | changeset | files | 
| Wed, 27 Jan 2010 08:20:31 +0100 | Christian Urban | some slight tuning | changeset | files | 
| Wed, 27 Jan 2010 07:49:43 +0100 | Christian Urban | added Terms to Nominal - Instantiation of two types does not work (ask Florian) | changeset | files | 
| Wed, 27 Jan 2010 07:45:01 +0100 | Christian Urban | added another example with indirect recursion over lists | changeset | files | 
| Tue, 26 Jan 2010 20:12:41 +0100 | Christian Urban | just moved obsolete material into Attic | changeset | files | 
| Tue, 26 Jan 2010 20:07:50 +0100 | Christian Urban | added an LamEx example together with the new nominal infrastructure | changeset | files | 
| Tue, 26 Jan 2010 16:30:51 +0100 | Cezary Kaliszyk | Bex1_Bexeq_regular. | changeset | files | 
| Tue, 26 Jan 2010 15:59:04 +0100 | Cezary Kaliszyk | Hom Theorem with exists unique | changeset | files | 
| Tue, 26 Jan 2010 14:48:25 +0100 | Cezary Kaliszyk | 2 cases for regularize with split, lemmas with split now lift. | changeset | files | 
| Tue, 26 Jan 2010 14:08:47 +0100 | Cezary Kaliszyk | Simpler statement that has the problem. | changeset | files | 
| Tue, 26 Jan 2010 13:58:28 +0100 | Cezary Kaliszyk | Found a term that does not regularize. | changeset | files | 
| Tue, 26 Jan 2010 13:53:56 +0100 | Cezary Kaliszyk | A triple is still ok. | changeset | files | 
| Tue, 26 Jan 2010 13:38:42 +0100 | Cezary Kaliszyk | Combined the simpsets in clean_tac and updated the comment. Now cleaning of splits does work. | changeset | files | 
| Tue, 26 Jan 2010 12:24:23 +0100 | Cezary Kaliszyk | Changed the lambda_prs_simple_conv to use id_apply, now last eq_reflection can be removed from id_simps. | changeset | files | 
| Tue, 26 Jan 2010 12:06:47 +0100 | Cezary Kaliszyk | Sigma cleaning works with split_prs (still manual proof). | changeset | files | 
| Tue, 26 Jan 2010 11:13:08 +0100 | Christian Urban | tuned | changeset | files | 
| Tue, 26 Jan 2010 10:53:44 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 26 Jan 2010 01:42:46 +0100 | Christian Urban | cleaning of QuotProd; a little cleaning of QuotList | changeset | files | 
| Tue, 26 Jan 2010 01:00:35 +0100 | Christian Urban | added prs and rsp lemmas for Inl and Inr | changeset | files | 
| Tue, 26 Jan 2010 00:47:40 +0100 | Christian Urban | used split_option_all lemma | changeset | files | 
| Tue, 26 Jan 2010 00:18:48 +0100 | Christian Urban | used the internal Option.map instead of custom option_map | changeset | files | 
| Tue, 26 Jan 2010 09:54:43 +0100 | Cezary Kaliszyk | Generalized split_prs and split_rsp | changeset | files | 
| Tue, 26 Jan 2010 09:28:32 +0100 | Cezary Kaliszyk | All eq_reflections apart from the one of 'id_apply' can be removed. | changeset | files | 
| Tue, 26 Jan 2010 08:55:55 +0100 | Cezary Kaliszyk | continued | changeset | files | 
| Tue, 26 Jan 2010 08:09:22 +0100 | Cezary Kaliszyk | More eqreflection/equiv cleaning. | changeset | files | 
| Tue, 26 Jan 2010 07:42:52 +0100 | Cezary Kaliszyk | more eq_reflection & other cleaning. | changeset | files | 
| Tue, 26 Jan 2010 07:14:10 +0100 | Cezary Kaliszyk | Removing more eq_reflections. | changeset | files | 
| Mon, 25 Jan 2010 20:47:20 +0100 | Christian Urban | ids *cannot* be object equalities | changeset | files | 
| Mon, 25 Jan 2010 20:35:42 +0100 | Christian Urban | re-inserted lemma in QuotList | changeset | files | 
| Mon, 25 Jan 2010 19:52:53 +0100 | Christian Urban | added prs and rsp lemmas for Some and None | changeset | files | 
| Mon, 25 Jan 2010 19:14:46 +0100 | Christian Urban | tuned proofs (mainly in QuotProd) | changeset | files | 
| Mon, 25 Jan 2010 18:52:22 +0100 | Christian Urban | properly commented out the "unused lemmas section" and moved actually used lemmas elsewhere; added two minor items to the TODO list | changeset | files | 
| Mon, 25 Jan 2010 18:13:44 +0100 | Christian Urban | renamed QuotScript to QuotBase | changeset | files | 
| Mon, 25 Jan 2010 17:53:08 +0100 | Christian Urban | cleaned some theorems | changeset | files | 
| Sun, 24 Jan 2010 23:41:27 +0100 | Christian Urban | test with splits | changeset | files | 
| Sat, 23 Jan 2010 17:25:18 +0100 | Cezary Kaliszyk | The alpha equivalence relations for structures in 'Terms' | changeset | files | 
| Sat, 23 Jan 2010 15:41:54 +0100 | Cezary Kaliszyk | More experiments with defining the homomorphism directly, lifting of 'distinct' and of 'exhaust'. | changeset | files | 
| Sat, 23 Jan 2010 07:22:27 +0100 | Cezary Kaliszyk | Trying to define hom for the lifted type directly. | changeset | files | 
| Fri, 22 Jan 2010 17:44:46 +0100 | Cezary Kaliszyk | Proper alpha equivalence for Sigma calculus. | changeset | files | 
| Thu, 21 Jan 2010 19:52:46 +0100 | Cezary Kaliszyk | Changed fun_map and rel_map to definitions. | changeset | files | 
| Thu, 21 Jan 2010 12:50:43 +0100 | Cezary Kaliszyk | Lifted Peter's Sigma lemma with Ex1. | changeset | files | 
| Thu, 21 Jan 2010 12:03:47 +0100 | Cezary Kaliszyk | Automatic injection of Bexeq | changeset | files | 
| Thu, 21 Jan 2010 11:11:22 +0100 | Cezary Kaliszyk | Automatic cleaning of Bexeq<->Ex1 theorems. | changeset | files | 
| Thu, 21 Jan 2010 10:55:09 +0100 | Cezary Kaliszyk | Using Bexeq_rsp, and manually lifted lemma with Ex1. | changeset | files | 
| Thu, 21 Jan 2010 09:55:05 +0100 | Cezary Kaliszyk | Bexeq definition, Ex1_prs lemma, Bex1_rsp lemma, compiles. | changeset | files | 
| Thu, 21 Jan 2010 09:02:04 +0100 | Cezary Kaliszyk | The missing rule. | changeset | files | 
| Thu, 21 Jan 2010 07:38:34 +0100 | Cezary Kaliszyk | Ex1 -> Bex1 Regularization, Preparing Exeq. | changeset | files | 
| Wed, 20 Jan 2010 16:50:31 +0100 | Cezary Kaliszyk | Added the Sigma Calculus example | changeset | files | 
| Wed, 20 Jan 2010 16:44:31 +0100 | Cezary Kaliszyk | Better error messages for non matching quantifiers. | changeset | files | 
| Wed, 20 Jan 2010 12:33:19 +0100 | Cezary Kaliszyk | Statement of term1_hom_rsp | changeset | files | 
| Wed, 20 Jan 2010 12:20:18 +0100 | Christian Urban | proved that the function is a function | changeset | files | 
| Wed, 20 Jan 2010 11:30:32 +0100 | Cezary Kaliszyk | term1_hom as a function | changeset | files | 
| Tue, 19 Jan 2010 18:17:42 +0100 | Cezary Kaliszyk | A version of hom with quantifiers. | changeset | files | 
| Sun, 17 Jan 2010 02:24:15 +0100 | Christian Urban | added permutation functions for the raw calculi | changeset | files | 
| Sat, 16 Jan 2010 04:23:27 +0100 | Christian Urban | fixed broken (partial) proof | changeset | files | 
| Sat, 16 Jan 2010 03:56:00 +0100 | Christian Urban | used "new" alpha-equivalence relation (according to new scheme); proved equivalence theorems and so on | changeset | files | 
| Sat, 16 Jan 2010 02:09:38 +0100 | Christian Urban | liftin and lifing_tac can now lift several "and"-separated goals at once; the raw-theorems have to be given in the order of goals | changeset | files | 
| Fri, 15 Jan 2010 17:09:36 +0100 | Christian Urban | added a partial proof under which conditions rlam_rec Respects alpha...I guess something like this is true; this means the Hom lemmas need to have preconditions | changeset | files | 
| Fri, 15 Jan 2010 16:13:49 +0100 | Christian Urban | tried to witness the hom-lemma with the recursion combinator from rlam....does not work yet completely | changeset | files | 
| Fri, 15 Jan 2010 15:56:25 +0100 | Christian Urban | merged | changeset | files | 
| Fri, 15 Jan 2010 15:56:06 +0100 | Christian Urban | added free_variable function (do not know about the algorithm yet) | changeset | files | 
| Fri, 15 Jan 2010 15:51:25 +0100 | Cezary Kaliszyk | hom lifted to hom', so it is true. Infrastructure for partially regularized quantifiers. Nicer errors for regularize. | changeset | files | 
| Fri, 15 Jan 2010 12:17:30 +0100 | Christian Urban | slight tuning of relation_error | changeset | files | 
| Fri, 15 Jan 2010 11:04:21 +0100 | Cezary Kaliszyk | Appropriate respects and a statement of the lifted hom lemma | changeset | files | 
| Fri, 15 Jan 2010 10:48:49 +0100 | Christian Urban | recursion-hom for lambda | changeset | files | 
| Fri, 15 Jan 2010 10:36:48 +0100 | Cezary Kaliszyk | Incorrect version of the homomorphism lemma | changeset | files | 
| Thu, 14 Jan 2010 23:51:17 +0100 | Christian Urban | trivial | changeset | files | 
| Thu, 14 Jan 2010 23:48:31 +0100 | Christian Urban | tuned quotient_typ.ML | changeset | files | 
| Thu, 14 Jan 2010 23:17:21 +0100 | Christian Urban | tuned quotient_def.ML and cleaned somewhat LamEx.thy | changeset | files | 
| Thu, 14 Jan 2010 19:03:08 +0100 | Christian Urban | a few more lemmas...except supp of lambda-abstractions | changeset | files | 
| Thu, 14 Jan 2010 18:41:50 +0100 | Christian Urban | removed one sorry | changeset | files | 
| Thu, 14 Jan 2010 18:35:38 +0100 | Christian Urban | nearly all of the proof | changeset | files | 
| Thu, 14 Jan 2010 17:57:20 +0100 | Christian Urban | right generalisation | changeset | files | 
| Thu, 14 Jan 2010 17:53:23 +0100 | Cezary Kaliszyk | First subgoal. | changeset | files | 
| Thu, 14 Jan 2010 17:13:11 +0100 | Christian Urban | setup for strong induction | changeset | files | 
| Thu, 14 Jan 2010 16:41:17 +0100 | Cezary Kaliszyk | exported absrep_const for nitpick. | changeset | files | 
| Thu, 14 Jan 2010 15:36:29 +0100 | Cezary Kaliszyk | minor | changeset | files | 
| Thu, 14 Jan 2010 15:25:24 +0100 | Cezary Kaliszyk | Simplified matches_typ. | changeset | files | 
| Thu, 14 Jan 2010 12:23:59 +0100 | Christian Urban | added bound-variable functions to terms | changeset | files | 
| Thu, 14 Jan 2010 12:17:39 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 14 Jan 2010 12:14:35 +0100 | Christian Urban | added 3 calculi with interesting binding structure | changeset | files | 
| Thu, 14 Jan 2010 10:51:03 +0100 | Cezary Kaliszyk | produce defs with lthy, like prs and ids | changeset | files | 
| Thu, 14 Jan 2010 10:47:19 +0100 | Cezary Kaliszyk | Remove SOLVED from quotient_tac. Move atomize_eqv to 'Unused'. | changeset | files | 
| Thu, 14 Jan 2010 10:06:29 +0100 | Cezary Kaliszyk | Finished organising an efficient datastructure for qconst_info. | changeset | files | 
| Thu, 14 Jan 2010 08:02:20 +0100 | Cezary Kaliszyk | Undid changes from symtab to termtab, since we need to lookup specialized types. | changeset | files | 
| Wed, 13 Jan 2010 16:46:25 +0100 | Cezary Kaliszyk | Moved the matches_typ function outside a?d simplified it. | changeset | files | 
| Wed, 13 Jan 2010 16:39:20 +0100 | Christian Urban | one more item in the list of Markus | changeset | files | 
| Wed, 13 Jan 2010 16:23:32 +0100 | Cezary Kaliszyk | Put relation_error as a separate function. | changeset | files | 
| Wed, 13 Jan 2010 16:14:02 +0100 | Cezary Kaliszyk | Better error message for definition failure. | changeset | files | 
| Wed, 13 Jan 2010 15:17:52 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 13 Jan 2010 15:17:36 +0100 | Cezary Kaliszyk | Stored Termtab for constant information. | changeset | files | 
| Wed, 13 Jan 2010 13:40:47 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 13 Jan 2010 13:40:23 +0100 | Christian Urban | deleted SOLVED' | changeset | files | 
| Wed, 13 Jan 2010 13:12:04 +0100 | Cezary Kaliszyk | Removed the 'oops' in IntEx. | changeset | files | 
| Wed, 13 Jan 2010 09:41:57 +0100 | Christian Urban | tuned | changeset | files | 
| Wed, 13 Jan 2010 09:30:59 +0100 | Christian Urban | added SOLVED' which is now part of Isabelle....must be removed eventually | changeset | files | 
| Wed, 13 Jan 2010 09:19:20 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 13 Jan 2010 00:46:31 +0100 | Christian Urban | tuned | changeset | files | 
| Wed, 13 Jan 2010 00:45:28 +0100 | Christian Urban | absrep_fun and equiv_relation do not produce anymore spurious maps; two problems arose in IntEx, which are marked with "INJECTION PROBLEM" | changeset | files | 
| Tue, 12 Jan 2010 17:46:35 +0100 | Cezary Kaliszyk | More indenting, bracket removing and comment restructuring. | changeset | files | 
| Tue, 12 Jan 2010 16:44:33 +0100 | Cezary Kaliszyk | Finished replacing OO by OOO | changeset | files | 
| Tue, 12 Jan 2010 16:28:53 +0100 | Cezary Kaliszyk | Change OO to OOO in FSet3. | changeset | files | 
| Tue, 12 Jan 2010 16:21:42 +0100 | Cezary Kaliszyk | minor comment editing | changeset | files | 
| Tue, 12 Jan 2010 16:12:54 +0100 | Cezary Kaliszyk | modifying comments/indentation in quotient_term.ml | changeset | files | 
| Tue, 12 Jan 2010 16:03:51 +0100 | Cezary Kaliszyk | Cleaning comments, indentation etc in quotient_tacs. | changeset | files | 
| Tue, 12 Jan 2010 15:48:46 +0100 | Cezary Kaliszyk | No more exception handling in rep_abs_rsp_tac | changeset | files | 
| Tue, 12 Jan 2010 12:14:33 +0100 | Cezary Kaliszyk | handle all is no longer necessary in lambda_prs. | changeset | files | 
| Tue, 12 Jan 2010 12:04:47 +0100 | Cezary Kaliszyk | removed 3 hacks. | changeset | files | 
| Tue, 12 Jan 2010 11:25:38 +0100 | Cezary Kaliszyk | Updated some comments. | changeset | files | 
| Tue, 12 Jan 2010 10:59:51 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 12 Jan 2010 10:59:38 +0100 | Cezary Kaliszyk | Removed exception handling from equals_rsp_tac. | changeset | files | 
| Mon, 11 Jan 2010 22:36:21 +0100 | Christian Urban | added an abbreviation for OOO | changeset | files | 
| Mon, 11 Jan 2010 20:04:19 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 11 Jan 2010 20:03:43 +0100 | Cezary Kaliszyk | Undid the non-working part. | changeset | files | 
| Mon, 11 Jan 2010 16:33:00 +0100 | Christian Urban | started to adhere to Wenzel-Standard | changeset | files | 
| Mon, 11 Jan 2010 15:58:38 +0100 | Cezary Kaliszyk | Changing exceptions to 'try', part 1. | changeset | files | 
| Mon, 11 Jan 2010 15:13:09 +0100 | Cezary Kaliszyk | removed quotdata_lookup_type | changeset | files | 
| Mon, 11 Jan 2010 11:51:19 +0100 | Cezary Kaliszyk | Fix for testing matching constants in regularize. | changeset | files | 
| Mon, 11 Jan 2010 01:03:34 +0100 | Christian Urban | tuned previous commit further | changeset | files | 
| Mon, 11 Jan 2010 00:31:29 +0100 | Christian Urban | the chk-functions in quotient_term also simplify the result according to the id_simps; had to remove id_def from this theorem list though; this caused in FSet3 that relied on this rule; the problem is marked with "ID PROBLEM" | changeset | files | 
| Sat, 09 Jan 2010 09:38:34 +0100 | Christian Urban | introduced separate match function | changeset | files | 
| Sat, 09 Jan 2010 08:52:06 +0100 | Christian Urban | removed obsolete equiv_relation and rnamed new_equiv_relation | changeset | files | 
| Fri, 08 Jan 2010 19:46:22 +0100 | Cezary Kaliszyk | New_relations, all works again including concat examples. | changeset | files | 
| Fri, 08 Jan 2010 15:02:12 +0100 | Cezary Kaliszyk | map and rel simps for all quotients; needed when changing the relations to aggregate ones. | changeset | files | 
| Fri, 08 Jan 2010 14:43:30 +0100 | Cezary Kaliszyk | id_simps needs to be taken out not used directly, otherwise the new lemmas are not there. | changeset | files | 
| Fri, 08 Jan 2010 11:20:12 +0100 | Cezary Kaliszyk | Experimients with fconcat_insert | changeset | files | 
| Fri, 08 Jan 2010 10:44:30 +0100 | Cezary Kaliszyk | Modifications for new_equiv_rel, part2 | changeset | files | 
| Fri, 08 Jan 2010 10:39:08 +0100 | Cezary Kaliszyk | Modifictaions for new_relation. | changeset | files | 
| Fri, 08 Jan 2010 10:08:01 +0100 | Cezary Kaliszyk | Proved concat_empty. | changeset | files | 
| Thu, 07 Jan 2010 16:51:38 +0100 | Cezary Kaliszyk | Replacing equivp by reflp in the assumptions leads to non-provable subgoals in the gen_pre lemmas. | changeset | files | 
| Thu, 07 Jan 2010 16:06:13 +0100 | Cezary Kaliszyk | some cleaning. | changeset | files | 
| Thu, 07 Jan 2010 15:50:22 +0100 | Cezary Kaliszyk | First generalization. | changeset | files | 
| Thu, 07 Jan 2010 14:14:17 +0100 | Cezary Kaliszyk | The working proof of the special case. | changeset | files | 
| Thu, 07 Jan 2010 10:55:20 +0100 | Cezary Kaliszyk | Reduced the proof to two simple but not obvious to prove facts. | changeset | files | 
| Thu, 07 Jan 2010 10:13:15 +0100 | Cezary Kaliszyk | More cleaning and commenting AbsRepTest. Now tests work; just slow. | changeset | files | 
| Thu, 07 Jan 2010 09:55:42 +0100 | Cezary Kaliszyk | cleaning in AbsRepTest. | changeset | files | 
| Wed, 06 Jan 2010 16:24:21 +0100 | Cezary Kaliszyk | Further in the proof | changeset | files | 
| Wed, 06 Jan 2010 09:19:23 +0100 | Cezary Kaliszyk | Tried to prove the lemma manually; only left with quotient proofs. | changeset | files | 
| Wed, 06 Jan 2010 08:24:37 +0100 | Cezary Kaliszyk | Sledgehammer bug. | changeset | files | 
| Tue, 05 Jan 2010 18:10:20 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 05 Jan 2010 18:09:03 +0100 | Cezary Kaliszyk | Trying the proof | changeset | files | 
| Tue, 05 Jan 2010 17:12:35 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 05 Jan 2010 17:06:51 +0100 | Cezary Kaliszyk | Struggling with composition | changeset | files | 
| Tue, 05 Jan 2010 15:25:31 +0100 | Cezary Kaliszyk | Trying to state composition quotient. | changeset | files | 
| Tue, 05 Jan 2010 14:23:45 +0100 | Christian Urban | proper handling of error messages (code copy - maybe this can be avoided) | changeset | files | 
| Tue, 05 Jan 2010 14:09:04 +0100 | Christian Urban | added a new version of equiv_relation (is not yet used anywhere except in AbsRepTest) | changeset | files | 
| Tue, 05 Jan 2010 10:41:20 +0100 | Cezary Kaliszyk | Readded 'regularize_to_injection' which I believe will be needed. | changeset | files | 
| Sat, 02 Jan 2010 23:15:15 +0100 | Christian Urban | added a warning to the quotient_type definition, if a map function is missing | changeset | files | 
| Fri, 01 Jan 2010 23:59:32 +0100 | Christian Urban | tuned | changeset | files | 
| Fri, 01 Jan 2010 11:30:00 +0100 | Christian Urban | a slight change to abs/rep generation | changeset | files | 
| Fri, 01 Jan 2010 04:39:43 +0100 | Christian Urban | tuned | changeset | files | 
| Fri, 01 Jan 2010 01:10:38 +0100 | Christian Urban | fixed comment errors | changeset | files | 
| Fri, 01 Jan 2010 01:08:19 +0100 | Christian Urban | some slight tuning | changeset | files | 
| Thu, 31 Dec 2009 23:53:10 +0100 | Christian Urban | renamed transfer to transform (Markus) | changeset | files | 
| Wed, 30 Dec 2009 12:10:57 +0000 | cu | some small changes | changeset | files | 
| Sun, 27 Dec 2009 23:33:10 +0100 | Christian Urban | added a functor that allows checking what is added to the theorem lists | changeset | files | 
| Sat, 26 Dec 2009 23:20:46 +0100 | Christian Urban | corrected wrong [quot_respect] attribute; tuned | changeset | files | 
| Sat, 26 Dec 2009 21:36:20 +0100 | Christian Urban | renamed mk_resp_arg to equiv_relation and exported it in the signature; added tests in AbsRepFun.thy | changeset | files | 
| Sat, 26 Dec 2009 20:45:37 +0100 | Christian Urban | added an item about when the same quotient constant is defined twice (throws a bind exception in quoteint_def.ML) | changeset | files | 
| Sat, 26 Dec 2009 20:24:53 +0100 | Christian Urban | as expected problems occure when lifting concat lemmas | changeset | files | 
| Sat, 26 Dec 2009 09:03:35 +0100 | Christian Urban | tuned | changeset | files | 
| Sat, 26 Dec 2009 08:06:45 +0100 | Christian Urban | commeted the absrep function | changeset | files | 
| Sat, 26 Dec 2009 07:15:30 +0100 | Christian Urban | generalised absrep function; needs consolidation | changeset | files | 
| Fri, 25 Dec 2009 00:58:06 +0100 | Christian Urban | tuned | changeset | files | 
| Fri, 25 Dec 2009 00:17:55 +0100 | Christian Urban | added sanity checks for quotient_type | changeset | files | 
| Thu, 24 Dec 2009 22:28:19 +0100 | Christian Urban | made the quotient_type definition more like typedef; now type variables need to be explicitly given | changeset | files | 
| Thu, 24 Dec 2009 00:58:50 +0100 | Christian Urban | used Local_Theory.declaration for storing quotdata | changeset | files | 
| Wed, 23 Dec 2009 23:53:03 +0100 | Christian Urban | tuning | changeset | files | 
| Wed, 23 Dec 2009 23:22:02 +0100 | Christian Urban | renamed some fields in the info records | changeset | files | 
| Wed, 23 Dec 2009 22:42:30 +0100 | Christian Urban | modified mk_resp_arg so that the user can give terms as equivalence relations, not just constants | changeset | files | 
| Wed, 23 Dec 2009 21:30:23 +0100 | Christian Urban | cleaed a bit function mk_typedef_main | changeset | files | 
| Wed, 23 Dec 2009 13:45:42 +0100 | Christian Urban | renamed QUOT_TYPE to Quot_Type | changeset | files | 
| Wed, 23 Dec 2009 13:23:33 +0100 | Christian Urban | explicit handling of mem_def, avoiding the use of the simplifier; this fixes some quotient_type definitions | changeset | files | 
| Wed, 23 Dec 2009 10:31:54 +0100 | Christian Urban | corrected map declarations for Sum and Prod; moved absrep_fun examples in separate file | changeset | files | 
| Tue, 22 Dec 2009 22:10:48 +0100 | Christian Urban | added "Highest Priority" category; and tuned slightly code | changeset | files | 
| Tue, 22 Dec 2009 21:44:50 +0100 | Christian Urban | added a print_maps command; updated the keyword file accordingly | changeset | files | 
| Tue, 22 Dec 2009 21:31:44 +0100 | Christian Urban | renamed get_fun to absrep_fun; introduced explicit checked versions of the term functions | changeset | files | 
| Tue, 22 Dec 2009 21:16:11 +0100 | Christian Urban | tuned | changeset | files | 
| Tue, 22 Dec 2009 21:06:46 +0100 | Christian Urban | moved get_fun into quotient_term; this simplifies the overall including structure of the package | changeset | files | 
| Tue, 22 Dec 2009 20:51:37 +0100 | Christian Urban | tuned comments; renamed QUOT_TRUE to Quot_True; atomize_eqv seems to not be neccessary (has it been added to Isabelle)...it is now comented out and everything still works | changeset | files | 
| Tue, 22 Dec 2009 07:42:16 +0100 | Christian Urban | on the hunt for what condition raises which exception in the CLEVER CODE of calculate_inst | changeset | files | 
| Tue, 22 Dec 2009 07:28:09 +0100 | Christian Urban | simplified calculate_instance; worked around some clever code; clever code is unfortunately still there...needs to be removed | changeset | files | 
| Mon, 21 Dec 2009 23:13:40 +0100 | Christian Urban | used eq_reflection not with OF, but directly in @{thm ...} | changeset | files | 
| Mon, 21 Dec 2009 23:01:58 +0100 | Christian Urban | cleaned a bit calculate_inst a bit; eta-contraction seems to be not necessary? (all examples go through) | changeset | files | 
| Mon, 21 Dec 2009 22:36:31 +0100 | Christian Urban | get_fun needed change to cope with "('a fset) fset" types...this needs composition (op o); now id_simps contains also id_o and o_id, and map_id is also added in QuotList.thy; regularize and cleaning needed to be hacked (indicated by "HACK")...THIS NEEDS ATTENTION!!!; except two lemmas in IntEx, all examples go through; added considerable material to FSet3; tuned FIXME-TODO | changeset | files | 
| Sun, 20 Dec 2009 00:53:35 +0100 | Christian Urban | on suggestion of Tobias renamed "quotient_def" to "quotient_definition"; needs new keyword file | changeset | files | 
| Sun, 20 Dec 2009 00:26:53 +0100 | Christian Urban | renamed "quotient" command to "quotient_type"; needs new keyword file to be installed | changeset | files | 
| Sun, 20 Dec 2009 00:15:40 +0100 | Christian Urban | this file is now obsolete; replaced by isar-keywords-quot.el | changeset | files | 
| Sun, 20 Dec 2009 00:14:46 +0100 | Christian Urban | with "isabelle make keywords" you can create automatically a "quot" keywordfile, provided all Logics are in place | changeset | files | 
| Sat, 19 Dec 2009 22:42:31 +0100 | Christian Urban | added a very old paper about Quotients in Isabelle (related work) | changeset | files | 
| Sat, 19 Dec 2009 22:21:51 +0100 | Christian Urban | avoided global "open"s - replaced by local "open"s | changeset | files | 
| Sat, 19 Dec 2009 22:09:57 +0100 | Christian Urban | small tuning | changeset | files | 
| Sat, 19 Dec 2009 22:04:34 +0100 | Christian Urban | various tunings; map_lookup now raises an exception; addition to FIXME-TODO | changeset | files | 
| Thu, 17 Dec 2009 17:59:12 +0100 | Christian Urban | minor cleaning | changeset | files | 
| Thu, 17 Dec 2009 14:58:33 +0100 | Christian Urban | moved the QuotMain code into two ML-files | changeset | files | 
| Wed, 16 Dec 2009 14:28:48 +0100 | Christian Urban | complete fix for IsaMakefile | changeset | files | 
| Wed, 16 Dec 2009 14:26:14 +0100 | Christian Urban | first fix | changeset | files | 
| Wed, 16 Dec 2009 14:09:03 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 16 Dec 2009 14:08:42 +0100 | Christian Urban | added a paper for possible notes | changeset | files | 
| Wed, 16 Dec 2009 12:15:41 +0100 | Cezary Kaliszyk | Removed lambdas on the right hand side. This fixes all 'PROBLEM' comments. | changeset | files | 
| Tue, 15 Dec 2009 16:40:00 +0100 | Cezary Kaliszyk | lambda_prs & solve_quotient_assum cleaned. | changeset | files | 
| Tue, 15 Dec 2009 15:38:17 +0100 | Christian Urban | some commenting | changeset | files | 
| Mon, 14 Dec 2009 14:24:08 +0100 | Cezary Kaliszyk | Fixed previous commit. | changeset | files | 
| Mon, 14 Dec 2009 13:59:08 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 14 Dec 2009 13:58:51 +0100 | Cezary Kaliszyk | Moved DETERM inside Repeat & added SOLVE around quotient_tac. | changeset | files | 
| Mon, 14 Dec 2009 13:57:39 +0100 | Cezary Kaliszyk | merge. | changeset | files | 
| Mon, 14 Dec 2009 13:56:24 +0100 | Cezary Kaliszyk | FIXME/TODO. | changeset | files | 
| Mon, 14 Dec 2009 10:19:27 +0100 | Cezary Kaliszyk | reply to question in code | changeset | files | 
| Mon, 14 Dec 2009 10:12:23 +0100 | Cezary Kaliszyk | Reply in code. | changeset | files | 
| Mon, 14 Dec 2009 10:09:49 +0100 | Cezary Kaliszyk | Replies to questions from the weekend: Uncommenting the renamed theorem commented out in 734. | changeset | files | 
| Sun, 13 Dec 2009 02:47:47 +0100 | Christian Urban | a few code annotations | changeset | files | 
| Sun, 13 Dec 2009 02:35:34 +0100 | Christian Urban | another pass on apply_rsp | changeset | files | 
| Sun, 13 Dec 2009 01:56:19 +0100 | Christian Urban | managed to simplify apply_rsp | changeset | files | 
| Sat, 12 Dec 2009 18:43:42 +0100 | Christian Urban | tried to simplify apply_rsp_tac; failed at the moment; added some questions | changeset | files | 
| Sat, 12 Dec 2009 18:01:22 +0100 | Christian Urban | some trivial changes | changeset | files | 
| Sat, 12 Dec 2009 16:40:29 +0100 | Christian Urban | trivial cleaning of make_inst | changeset | files | 
| Sat, 12 Dec 2009 15:23:58 +0100 | Christian Urban | tried to improve test; but fails | changeset | files | 
| Sat, 12 Dec 2009 15:08:25 +0100 | Christian Urban | merged | changeset | files | 
| Sat, 12 Dec 2009 15:07:59 +0100 | Christian Urban | annotated some questions to the code; some simple changes | changeset | files | 
| Sat, 12 Dec 2009 14:57:34 +0100 | Cezary Kaliszyk | Answering the question in code. | changeset | files | 
| Sat, 12 Dec 2009 13:54:01 +0100 | Christian Urban | merged | changeset | files | 
| Sat, 12 Dec 2009 13:53:46 +0100 | Christian Urban | trivial | changeset | files | 
| Sat, 12 Dec 2009 02:01:33 +0100 | Christian Urban | tuned code | changeset | files | 
| Sat, 12 Dec 2009 09:27:06 +0100 | Cezary Kaliszyk | Minor | changeset | files | 
| Sat, 12 Dec 2009 05:12:50 +0100 | Cezary Kaliszyk | Some proofs. | changeset | files | 
| Sat, 12 Dec 2009 04:48:43 +0100 | Cezary Kaliszyk | Proof of finite_set_storng_cases_raw. | changeset | files | 
| Sat, 12 Dec 2009 04:25:47 +0100 | Cezary Kaliszyk | A bracket was missing; with it proved the 'definitely false' lemma. | changeset | files | 
| Sat, 12 Dec 2009 01:44:56 +0100 | Christian Urban | renamed quotient.ML to quotient_typ.ML | changeset | files | 
| Fri, 11 Dec 2009 19:22:30 +0100 | Christian Urban | merged | changeset | files | 
| Fri, 11 Dec 2009 19:19:50 +0100 | Christian Urban | tuned | changeset | files | 
| Fri, 11 Dec 2009 19:19:24 +0100 | Christian Urban | started to have a look at it; redefined the relation | changeset | files | 
| Fri, 11 Dec 2009 17:59:29 +0100 | Cezary Kaliszyk | More name and indentation cleaning. | changeset | files | 
| Fri, 11 Dec 2009 17:22:26 +0100 | Cezary Kaliszyk | Merge + Added LarryInt & Fset3 to tests. | changeset | files | 
| Fri, 11 Dec 2009 17:19:38 +0100 | Cezary Kaliszyk | Renaming | changeset | files | 
| Fri, 11 Dec 2009 17:03:52 +0100 | Christian Urban | merged | changeset | files | 
| Fri, 11 Dec 2009 17:03:34 +0100 | Christian Urban | deleted struct_match by Pattern.match (fixes a problem in LarryInt) | changeset | files | 
| Fri, 11 Dec 2009 16:32:40 +0100 | Cezary Kaliszyk | FSet3 minor fixes + cases | changeset | files | 
| Fri, 11 Dec 2009 15:58:15 +0100 | Christian Urban | added Int example from Larry | changeset | files | 
| Fri, 11 Dec 2009 15:49:15 +0100 | Cezary Kaliszyk | Added FSet3 with a formalisation of finite sets based on Michael's one. | changeset | files | 
| Fri, 11 Dec 2009 13:51:08 +0100 | Cezary Kaliszyk | Updated TODO list together. | changeset | files | 
| Fri, 11 Dec 2009 11:32:29 +0100 | Cezary Kaliszyk | Merge | changeset | files | 
| Fri, 11 Dec 2009 11:30:00 +0100 | Cezary Kaliszyk | More theorem renaming. | changeset | files | 
| Fri, 11 Dec 2009 11:25:52 +0100 | Cezary Kaliszyk | Renamed theorems in IntEx2 to conform to names in Int. | changeset | files | 
| Fri, 11 Dec 2009 11:19:41 +0100 | Cezary Kaliszyk | Updated comments. | changeset | files | 
| Fri, 11 Dec 2009 11:14:05 +0100 | Christian Urban | merged | changeset | files | 
| Fri, 11 Dec 2009 11:12:53 +0100 | Christian Urban | tuned | changeset | files | 
| Fri, 11 Dec 2009 10:57:46 +0100 | Christian Urban | renamed Larrys example | changeset | files | 
| Fri, 11 Dec 2009 11:08:58 +0100 | Cezary Kaliszyk | New syntax for definitions. | changeset | files | 
| Fri, 11 Dec 2009 08:28:41 +0100 | Christian Urban | changed error message | changeset | files | 
| Fri, 11 Dec 2009 06:58:31 +0100 | Christian Urban | reformulated the lemma lifting_procedure as ML value; gave better warning message for injection case | changeset | files | 
| Thu, 10 Dec 2009 19:05:56 +0100 | Christian Urban | slightly tuned | changeset | files | 
| Thu, 10 Dec 2009 18:28:41 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 10 Dec 2009 18:28:30 +0100 | Christian Urban | added Larry's theory; introduced lemma equivpI; added something to the TODO about error messages | changeset | files | 
| Thu, 10 Dec 2009 16:56:03 +0100 | Christian Urban | added maps-printout and tuned some comments | changeset | files | 
| Thu, 10 Dec 2009 14:35:06 +0100 | Cezary Kaliszyk | Option and Sum quotients. | changeset | files | 
| Thu, 10 Dec 2009 12:25:12 +0100 | Cezary Kaliszyk | Regularized the hard lemma. | changeset | files | 
| Thu, 10 Dec 2009 11:19:34 +0100 | Cezary Kaliszyk | Simplification of Babses for regularize; will probably become injection | changeset | files | 
| Thu, 10 Dec 2009 10:54:45 +0100 | Cezary Kaliszyk | Found the problem with ttt3. | changeset | files | 
| Thu, 10 Dec 2009 10:36:05 +0100 | Cezary Kaliszyk | minor | changeset | files | 
| Thu, 10 Dec 2009 10:21:51 +0100 | Cezary Kaliszyk | Moved Unused part of locale to Unused QuotMain. | changeset | files | 
| Thu, 10 Dec 2009 08:55:30 +0100 | Cezary Kaliszyk | Moved 'int_induct' to IntEx to keep IntEx2 being just theory of integers in order. | changeset | files | 
| Thu, 10 Dec 2009 08:44:01 +0100 | Cezary Kaliszyk | Removed 'Presburger' as it introduces int & other minor cleaning in Int2. | changeset | files | 
| Thu, 10 Dec 2009 05:11:53 +0100 | Christian Urban | more tuning | changeset | files | 
| Thu, 10 Dec 2009 05:02:34 +0100 | Christian Urban | tuned | changeset | files | 
| Thu, 10 Dec 2009 04:53:48 +0100 | Christian Urban | simplified the instantiation of QUOT_TRUE in procedure_tac | changeset | files | 
| Thu, 10 Dec 2009 04:35:08 +0100 | Christian Urban | completed previous commit | changeset | files | 
| Thu, 10 Dec 2009 04:34:24 +0100 | Christian Urban | deleted DT/NDT diagnostic code | changeset | files | 
| Thu, 10 Dec 2009 04:23:13 +0100 | Christian Urban | moved the interpretation code into Unused.thy | changeset | files | 
| Thu, 10 Dec 2009 03:48:39 +0100 | Christian Urban | added an attempt to get a finite set theory | changeset | files | 
| Thu, 10 Dec 2009 03:47:10 +0100 | Christian Urban | removed memb and used standard mem (member from List.thy) | changeset | files | 
| Thu, 10 Dec 2009 03:25:42 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 10 Dec 2009 03:11:19 +0100 | Christian Urban | simplified proofs | changeset | files | 
| Thu, 10 Dec 2009 02:46:08 +0100 | Christian Urban | removed quot_respect attribute of a non-standard lemma | changeset | files | 
| Thu, 10 Dec 2009 02:42:09 +0100 | Cezary Kaliszyk | With int_of_nat as a quotient_def, lemmas about it can be easily lifted. | changeset | files | 
| Thu, 10 Dec 2009 01:48:39 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 10 Dec 2009 01:47:55 +0100 | Christian Urban | naming in this file cannot be made to agree to the original (PROBLEM?) | changeset | files | 
| Thu, 10 Dec 2009 01:39:47 +0100 | Cezary Kaliszyk | Lifted some kind of induction. | changeset | files | 
| Wed, 09 Dec 2009 23:32:16 +0100 | Christian Urban | more proofs in IntEx2 | changeset | files | 
| Wed, 09 Dec 2009 22:43:11 +0100 | Cezary Kaliszyk | Finished one proof in IntEx2. | changeset | files | 
| Wed, 09 Dec 2009 22:05:11 +0100 | Christian Urban | slightly more on IntEx2 | changeset | files | 
| Wed, 09 Dec 2009 20:35:52 +0100 | Christian Urban | proved (with a lot of pain) that times_raw is respectful | changeset | files | 
| Wed, 09 Dec 2009 17:31:19 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 09 Dec 2009 17:31:01 +0100 | Christian Urban | fixed minor stupidity | changeset | files | 
| Wed, 09 Dec 2009 17:16:39 +0100 | Cezary Kaliszyk | Exception handling. | changeset | files | 
| Wed, 09 Dec 2009 17:05:33 +0100 | Cezary Kaliszyk | Code cleaning. | changeset | files | 
| Wed, 09 Dec 2009 16:44:34 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 09 Dec 2009 16:43:12 +0100 | Cezary Kaliszyk | foldr_rsp. | changeset | files | 
| Wed, 09 Dec 2009 16:09:25 +0100 | Christian Urban | tuned | changeset | files | 
| Wed, 09 Dec 2009 15:59:02 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 09 Dec 2009 15:57:47 +0100 | Cezary Kaliszyk | Different syntax for definitions that allows overloading and retrieving of definitions by matching whole constants. | changeset | files | 
| Wed, 09 Dec 2009 15:35:21 +0100 | Christian Urban | deleted make_inst3 | changeset | files | 
| Wed, 09 Dec 2009 15:29:36 +0100 | Christian Urban | tuned | changeset | files | 
| Wed, 09 Dec 2009 15:28:01 +0100 | Christian Urban | tuned | changeset | files | 
| Wed, 09 Dec 2009 15:24:11 +0100 | Christian Urban | moved function and tuned comment | changeset | files | 
| Wed, 09 Dec 2009 15:11:49 +0100 | Christian Urban | improved fun_map_conv | changeset | files | 
| Wed, 09 Dec 2009 06:21:09 +0100 | Cezary Kaliszyk | Arbitrary number of fun_map_tacs. | changeset | files | 
| Wed, 09 Dec 2009 05:59:49 +0100 | Cezary Kaliszyk | Temporarily repeated fun_map_tac 4 times. Cleaning for all examples work. | changeset | files | 
| Wed, 09 Dec 2009 00:54:46 +0100 | Christian Urban | tuned code | changeset | files | 
| Wed, 09 Dec 2009 00:03:18 +0100 | Christian Urban | tuned the examples and flagged the problematic cleaning lemmas in FSet | changeset | files | 
| Tue, 08 Dec 2009 23:32:54 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 08 Dec 2009 23:30:47 +0100 | Christian Urban | implemented cleaning strategy with fun_map.simps on non-bounded variables; still a few rough edges | changeset | files | 
| Tue, 08 Dec 2009 23:04:40 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 08 Dec 2009 23:04:25 +0100 | Cezary Kaliszyk | manually cleaned the hard lemma. | changeset | files | 
| Tue, 08 Dec 2009 22:26:01 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 08 Dec 2009 22:24:24 +0100 | Christian Urban | decoupled QuotProd from QuotMain and also started new cleaning strategy | changeset | files | 
| Tue, 08 Dec 2009 22:05:01 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 08 Dec 2009 22:03:34 +0100 | Cezary Kaliszyk | An example which is hard to lift because of the interplay between lambda_prs and unfolding. | changeset | files | 
| Tue, 08 Dec 2009 22:02:14 +0100 | Christian Urban | proper formulation of all preservation theorems | changeset | files | 
| Tue, 08 Dec 2009 20:55:55 +0100 | Christian Urban | started to reformulate preserve lemmas | changeset | files | 
| Tue, 08 Dec 2009 20:34:00 +0100 | Christian Urban | properly set up the prs_rules | changeset | files | 
| Tue, 08 Dec 2009 17:43:32 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 08 Dec 2009 17:40:58 +0100 | Christian Urban | added preserve rules to the cleaning_tac | changeset | files | 
| Tue, 08 Dec 2009 17:39:34 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 08 Dec 2009 17:35:04 +0100 | Cezary Kaliszyk | cleaning. | changeset | files | 
| Tue, 08 Dec 2009 17:34:10 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 08 Dec 2009 17:33:51 +0100 | Christian Urban | chnaged syntax to "lifting theorem" | changeset | files | 
| Tue, 08 Dec 2009 17:30:00 +0100 | Christian Urban | changed names of attributes | changeset | files | 
| Tue, 08 Dec 2009 16:56:51 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 08 Dec 2009 16:56:37 +0100 | Cezary Kaliszyk | Manual regularization of a goal in FSet. | changeset | files | 
| Tue, 08 Dec 2009 16:36:01 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 08 Dec 2009 16:35:40 +0100 | Christian Urban | added methods for the lifting_tac and the other tacs | changeset | files | 
| Tue, 08 Dec 2009 15:42:29 +0100 | Cezary Kaliszyk | make_inst3 | changeset | files | 
| Tue, 08 Dec 2009 15:12:55 +0100 | Cezary Kaliszyk | Merge | changeset | files | 
| Tue, 08 Dec 2009 15:12:36 +0100 | Cezary Kaliszyk | trans2 replaced with equals_rsp_tac | changeset | files | 
| Tue, 08 Dec 2009 14:00:48 +0100 | Christian Urban | corrected name of FSet in ROOT.ML | changeset | files | 
| Tue, 08 Dec 2009 13:09:21 +0100 | Cezary Kaliszyk | Made fset work again to test all. | changeset | files | 
| Tue, 08 Dec 2009 13:08:56 +0100 | Cezary Kaliszyk | Finished the proof of ttt2 and found bug in regularize when trying ttt3. | changeset | files | 
| Tue, 08 Dec 2009 13:01:23 +0100 | Cezary Kaliszyk | Another lambda example theorem proved. Seems it starts working properly. | changeset | files | 
| Tue, 08 Dec 2009 13:00:36 +0100 | Cezary Kaliszyk | Removed pattern from quot_rel_rsp, since list_rel and all used introduced ones cannot be patterned | changeset | files | 
| Tue, 08 Dec 2009 12:59:38 +0100 | Cezary Kaliszyk | Proper checked map_rsp. | changeset | files | 
| Tue, 08 Dec 2009 12:36:28 +0100 | Cezary Kaliszyk | Nitpick found a counterexample for one lemma. | changeset | files | 
| Tue, 08 Dec 2009 11:59:16 +0100 | Cezary Kaliszyk | Added a 'rep_abs' in inj_repabs_trm of babs; and proved two lam examples. | changeset | files | 
| Tue, 08 Dec 2009 11:38:58 +0100 | Cezary Kaliszyk | It also regularizes. | changeset | files | 
| Tue, 08 Dec 2009 11:28:04 +0100 | Cezary Kaliszyk | inj_repabs also works. | changeset | files | 
| Tue, 08 Dec 2009 11:20:01 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 08 Dec 2009 11:17:56 +0100 | Cezary Kaliszyk | An example of working cleaning for lambda lifting. Still not sure why Babs helps. | changeset | files | 
| Tue, 08 Dec 2009 04:21:14 +0100 | Christian Urban | tuned | changeset | files | 
| Tue, 08 Dec 2009 04:14:02 +0100 | Christian Urban | the lift_tac produces a warning message if one of the three automatic proofs fails | changeset | files | 
| Tue, 08 Dec 2009 01:25:43 +0100 | Christian Urban | added a thm list for ids | changeset | files | 
| Tue, 08 Dec 2009 01:00:21 +0100 | Christian Urban | removed a fixme: map_info is now checked | changeset | files | 
| Mon, 07 Dec 2009 23:45:51 +0100 | Christian Urban | tuning of the code | changeset | files | 
| Mon, 07 Dec 2009 21:54:14 +0100 | Christian Urban | merged | changeset | files | 
| Mon, 07 Dec 2009 21:53:50 +0100 | Christian Urban | removed "global" data and lookup functions; had to move a tactic out from the inj_repabs_match tactic since apply_rsp interferes with a trans2 rule for ===> | changeset | files | 
| Mon, 07 Dec 2009 21:25:49 +0100 | Cezary Kaliszyk | 3 lambda examples in FSet. In the last one regularize_term fails. | changeset | files | 
| Mon, 07 Dec 2009 21:21:57 +0100 | Cezary Kaliszyk | Handling of errors in lambda_prs_conv. | changeset | files | 
| Mon, 07 Dec 2009 21:21:23 +0100 | Cezary Kaliszyk | babs_prs | changeset | files | 
| Mon, 07 Dec 2009 18:49:14 +0100 | Christian Urban | clarified the function examples | changeset | files | 
| Mon, 07 Dec 2009 17:57:33 +0100 | Christian Urban | first attempt to deal with Babs in regularise and cleaning (not yet working) | changeset | files | 
| Mon, 07 Dec 2009 15:21:51 +0100 | Christian Urban | isabelle make tests all examples | changeset | files | 
| Mon, 07 Dec 2009 15:18:44 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 07 Dec 2009 15:18:00 +0100 | Cezary Kaliszyk | make_inst for lambda_prs where the second quotient is not identity. | changeset | files | 
| Mon, 07 Dec 2009 14:37:10 +0100 | Christian Urban | added "end" to each example theory | changeset | files | 
| Mon, 07 Dec 2009 14:35:45 +0100 | Cezary Kaliszyk | List moved after QuotMain | changeset | files | 
| Mon, 07 Dec 2009 14:14:07 +0100 | Christian Urban | cleaning | changeset | files | 
| Mon, 07 Dec 2009 14:12:29 +0100 | Christian Urban | final move | changeset | files | 
| Mon, 07 Dec 2009 14:09:50 +0100 | Christian Urban | directory re-arrangement | changeset | files | 
| Mon, 07 Dec 2009 14:00:36 +0100 | Cezary Kaliszyk | inj_repabs_tac handles Babs now. | changeset | files | 
| Mon, 07 Dec 2009 12:14:25 +0100 | Cezary Kaliszyk | Fix of regularize for babs and proof of babs_rsp. | changeset | files | 
| Mon, 07 Dec 2009 11:14:21 +0100 | Cezary Kaliszyk | Using pair_prs; debugging the error in regularize of a lambda. | changeset | files | 
| Mon, 07 Dec 2009 08:45:04 +0100 | Cezary Kaliszyk | QuotProd with product_quotient and a 3 respects and preserves lemmas. | changeset | files | 
| Mon, 07 Dec 2009 04:41:42 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 07 Dec 2009 04:39:42 +0100 | Cezary Kaliszyk | 3 new example thms in MyInt; reveal problems with handling of lambdas; regularize fails with "Loose Bound". | changeset | files | 
| Mon, 07 Dec 2009 02:34:24 +0100 | Christian Urban | simplified the regularize simproc | changeset | files | 
| Mon, 07 Dec 2009 01:28:10 +0100 | Christian Urban | now simpler regularize_tac with added solver works | changeset | files | 
| Mon, 07 Dec 2009 01:22:20 +0100 | Christian Urban | removed usage of HOL_basic_ss by using a slighly extended version of empty_ss | changeset | files | 
| Mon, 07 Dec 2009 00:13:36 +0100 | Christian Urban | merged | changeset | files | 
| Mon, 07 Dec 2009 00:07:23 +0100 | Christian Urban | fixed examples | changeset | files | 
| Mon, 07 Dec 2009 00:03:12 +0100 | Cezary Kaliszyk | Fix IntEx2 for equiv_list | changeset | files | 
| Sun, 06 Dec 2009 23:35:02 +0100 | Christian Urban | merged | changeset | files | 
| Sun, 06 Dec 2009 23:32:27 +0100 | Christian Urban | working state again | changeset | files | 
| Sun, 06 Dec 2009 13:41:42 +0100 | Christian Urban | added a theorem list for equivalence theorems | changeset | files | 
| Sun, 06 Dec 2009 22:58:03 +0100 | Cezary Kaliszyk | Merge | changeset | files | 
| Sun, 06 Dec 2009 22:57:44 +0100 | Cezary Kaliszyk | Name changes. | changeset | files | 
| Sun, 06 Dec 2009 22:57:03 +0100 | Cezary Kaliszyk | Solved all quotient goals. | changeset | files | 
| Sun, 06 Dec 2009 11:39:34 +0100 | Christian Urban | updated Isabelle and deleted mono rules | changeset | files | 
| Sun, 06 Dec 2009 11:21:29 +0100 | Christian Urban | more tuning of the code | changeset | files | 
| Sun, 06 Dec 2009 11:09:51 +0100 | Christian Urban | puting code in separate sections | changeset | files | 
| Sun, 06 Dec 2009 06:58:24 +0100 | Cezary Kaliszyk | Handle 'find_qt_asm' exception. Now all inj_repabs_goals should be solved automatically. | changeset | files | 
| Sun, 06 Dec 2009 06:41:52 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Sun, 06 Dec 2009 06:39:32 +0100 | Cezary Kaliszyk | Simpler definition code that works with any type maps. | changeset | files | 
| Sun, 06 Dec 2009 04:03:08 +0100 | Christian Urban | working on lambda_prs with examples; polished code of clean_tac | changeset | files | 
| Sun, 06 Dec 2009 02:41:35 +0100 | Christian Urban | renamed lambda_allex_prs | changeset | files | 
| Sun, 06 Dec 2009 01:43:46 +0100 | Christian Urban | added more to IntEx2 | changeset | files | 
| Sun, 06 Dec 2009 00:19:45 +0100 | Christian Urban | merged | changeset | files | 
| Sun, 06 Dec 2009 00:13:35 +0100 | Christian Urban | added new example for Ints; regularise does not work in all instances | changeset | files | 
| Sun, 06 Dec 2009 00:00:47 +0100 | Cezary Kaliszyk | Definitions folded first. | changeset | files | 
| Sat, 05 Dec 2009 23:35:09 +0100 | Cezary Kaliszyk | Used symmetric definitions. Moved quotient_rsp to QuotMain. | changeset | files | 
| Sat, 05 Dec 2009 23:26:08 +0100 | Cezary Kaliszyk | Proved foldl_rsp and ho_map_rsp | changeset | files | 
| Sat, 05 Dec 2009 22:38:42 +0100 | Christian Urban | moved all_prs and ex_prs out from the conversion into the simplifier | changeset | files | 
| Sat, 05 Dec 2009 22:16:17 +0100 | Christian Urban | further cleaning | changeset | files | 
| Sat, 05 Dec 2009 22:07:46 +0100 | Cezary Kaliszyk | Merge | changeset | files | 
| Sat, 05 Dec 2009 22:05:09 +0100 | Cezary Kaliszyk | Added nil_rsp and cons_rsp to quotient_rsp; simplified IntEx. | changeset | files | 
| Sat, 05 Dec 2009 22:02:32 +0100 | Christian Urban | simplified inj_repabs_trm | changeset | files | 
| Sat, 05 Dec 2009 21:50:31 +0100 | Christian Urban | merged | changeset | files | 
| Sat, 05 Dec 2009 21:47:48 +0100 | Christian Urban | merged | changeset | files | 
| Sat, 05 Dec 2009 21:45:56 +0100 | Christian Urban | merged | changeset | files | 
| Sat, 05 Dec 2009 21:44:01 +0100 | Christian Urban | simpler version of clean_tac | changeset | files | 
| Sat, 05 Dec 2009 21:45:39 +0100 | Cezary Kaliszyk | Handling of respects in the fast inj_repabs_tac; includes respects with quotient assumptions. | changeset | files | 
| Sat, 05 Dec 2009 21:28:24 +0100 | Cezary Kaliszyk | Solutions to IntEx tests. | changeset | files | 
| Sat, 05 Dec 2009 16:26:18 +0100 | Christian Urban | made some slight simplifications to the examples | changeset | files | 
| Sat, 05 Dec 2009 13:49:35 +0100 | Christian Urban | added three examples to IntEx for testing ideas - regularisation and injection seem to be not quite right yet | changeset | files | 
| Sat, 05 Dec 2009 00:06:27 +0100 | Christian Urban | tuned code | changeset | files | 
| Fri, 04 Dec 2009 21:43:29 +0100 | Christian Urban | merged | changeset | files | 
| Fri, 04 Dec 2009 21:42:55 +0100 | Christian Urban | not yet quite functional treatment of constants | changeset | files | 
| Fri, 04 Dec 2009 19:47:58 +0100 | Cezary Kaliszyk | Changed FOCUS to SUBGOAL in rep_abs_rsp_tac; another 20% speedup :) | changeset | files | 
| Fri, 04 Dec 2009 19:06:53 +0100 | Cezary Kaliszyk | Changing FOCUS to CSUBGOAL (part 1) | changeset | files | 
| Fri, 04 Dec 2009 18:32:19 +0100 | Cezary Kaliszyk | abs_rep as == | changeset | files | 
| Fri, 04 Dec 2009 17:57:03 +0100 | Cezary Kaliszyk | Cleaning the Quotients file | changeset | files | 
| Fri, 04 Dec 2009 17:50:02 +0100 | Cezary Kaliszyk | Minor renames and moving | changeset | files | 
| Fri, 04 Dec 2009 17:36:45 +0100 | Cezary Kaliszyk | Cleaning/review of QuotScript. | changeset | files | 
| Fri, 04 Dec 2009 17:15:55 +0100 | Cezary Kaliszyk | More cleaning | changeset | files | 
| Fri, 04 Dec 2009 16:53:11 +0100 | Cezary Kaliszyk | more name cleaning and removing | changeset | files | 
| Fri, 04 Dec 2009 16:40:23 +0100 | Cezary Kaliszyk | More code cleaning and renaming: moved rsp and prs lemmas from Int to QuotList | changeset | files | 
| Fri, 04 Dec 2009 16:12:40 +0100 | Cezary Kaliszyk | Cleaning & Renaming coming from QuotList | changeset | files | 
| Fri, 04 Dec 2009 16:01:23 +0100 | Cezary Kaliszyk | Cleaning in Quotients | changeset | files | 
| Fri, 04 Dec 2009 15:50:57 +0100 | Cezary Kaliszyk | Even more name changes and cleaning | changeset | files | 
| Fri, 04 Dec 2009 15:41:09 +0100 | Cezary Kaliszyk | More code cleaning and name changes | changeset | files | 
| Fri, 04 Dec 2009 15:25:51 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Fri, 04 Dec 2009 15:25:26 +0100 | Cezary Kaliszyk | merged | changeset | files | 
| Fri, 04 Dec 2009 15:23:10 +0100 | Christian Urban | smaller theory footprint | changeset | files | 
| Fri, 04 Dec 2009 15:20:06 +0100 | Christian Urban | merged | changeset | files | 
| Fri, 04 Dec 2009 15:19:39 +0100 | Christian Urban | merge | changeset | files | 
| Fri, 04 Dec 2009 15:18:37 +0100 | Christian Urban | smaller theory footprint | changeset | files | 
| Fri, 04 Dec 2009 15:18:33 +0100 | Cezary Kaliszyk | More name changes | changeset | files | 
| Fri, 04 Dec 2009 15:04:05 +0100 | Cezary Kaliszyk | Naming changes | changeset | files | 
| Fri, 04 Dec 2009 14:35:36 +0100 | Cezary Kaliszyk | code cleaning and renaming | changeset | files | 
| Fri, 04 Dec 2009 14:11:20 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Fri, 04 Dec 2009 14:11:03 +0100 | Cezary Kaliszyk | Removed previous inj_repabs_tac | changeset | files | 
| Fri, 04 Dec 2009 13:58:23 +0100 | Christian Urban | some tuning | changeset | files | 
| Fri, 04 Dec 2009 12:21:15 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Fri, 04 Dec 2009 12:20:49 +0100 | Cezary Kaliszyk | rep_abs_rsp_tac to replace the last use of instantiate_tac with matching and unification. | changeset | files | 
| Fri, 04 Dec 2009 11:34:49 +0100 | Christian Urban | merged | changeset | files | 
| Fri, 04 Dec 2009 11:34:21 +0100 | Christian Urban | merged | changeset | files | 
| Fri, 04 Dec 2009 11:33:58 +0100 | Cezary Kaliszyk | Change equiv_trans2 to EQUALS_RSP, since we can prove it for any quotient type, not only for eqv relations. | changeset | files | 
| Fri, 04 Dec 2009 11:06:43 +0100 | Cezary Kaliszyk | compose_tac instead of rtac to avoid unification; some code cleaning. | changeset | files | 
| Fri, 04 Dec 2009 10:36:35 +0100 | Cezary Kaliszyk | Got to about 5 seconds for the longest proof. APPLY_RSP_TAC' solves the quotient internally without instantiation resulting in a faster proof. | changeset | files | 
| Fri, 04 Dec 2009 10:12:17 +0100 | Cezary Kaliszyk | Using APPLY_RSP1; again a little bit faster. | changeset | files | 
| Fri, 04 Dec 2009 09:33:32 +0100 | Cezary Kaliszyk | Fixes after big merge. | changeset | files | 
| Fri, 04 Dec 2009 09:25:27 +0100 | Cezary Kaliszyk | The big merge; probably non-functional. | changeset | files | 
| Fri, 04 Dec 2009 09:08:51 +0100 | Cezary Kaliszyk | Testing the new tactic everywhere | changeset | files | 
| Fri, 04 Dec 2009 09:01:13 +0100 | Cezary Kaliszyk | First version of the deterministic rep-abs-inj-tac. | changeset | files | 
| Fri, 04 Dec 2009 09:18:46 +0100 | Cezary Kaliszyk | Changing = to \<equiv> in case if we want to use simp. | changeset | files | 
| Fri, 04 Dec 2009 09:10:31 +0100 | Cezary Kaliszyk | Even better: Completely got rid of the simps in both quotient_tac and inj_repabs_tac | changeset | files | 
| Fri, 04 Dec 2009 08:19:56 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Fri, 04 Dec 2009 08:18:38 +0100 | Cezary Kaliszyk | Made your version work again with LIST_REL_EQ. | changeset | files | 
| Thu, 03 Dec 2009 19:06:14 +0100 | Christian Urban | the error occurs in APPLY_RSP_TAC where the wrong quotient (for LIST_REL) is applied | changeset | files | 
| Thu, 03 Dec 2009 15:03:31 +0100 | Christian Urban | removed quot argument...not all examples work anymore | changeset | files | 
| Thu, 03 Dec 2009 14:02:05 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 03 Dec 2009 14:00:43 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 03 Dec 2009 13:59:53 +0100 | Christian Urban | first version of internalised quotient theorems; added FIXME-TODO | changeset | files | 
| Thu, 03 Dec 2009 11:40:10 +0100 | Christian Urban | further dead code | changeset | files | 
| Thu, 03 Dec 2009 13:56:59 +0100 | Cezary Kaliszyk | Reintroduced varifyT; we still need it for permutation definition. | changeset | files | 
| Thu, 03 Dec 2009 13:45:52 +0100 | Cezary Kaliszyk | Updated the examples | changeset | files | 
| Thu, 03 Dec 2009 12:33:05 +0100 | Cezary Kaliszyk | Fixed previous mistake | changeset | files | 
| Thu, 03 Dec 2009 12:31:05 +0100 | Cezary Kaliszyk | defs used automatically by clean_tac | changeset | files | 
| Thu, 03 Dec 2009 12:22:19 +0100 | Cezary Kaliszyk | Added qoutient_consts dest for getting all the constant definitions in the cleaning step. | changeset | files | 
| Thu, 03 Dec 2009 12:17:23 +0100 | Cezary Kaliszyk | Added the definition to quotient constant data. | changeset | files | 
| Thu, 03 Dec 2009 11:58:46 +0100 | Cezary Kaliszyk | removing unused code | changeset | files | 
| Thu, 03 Dec 2009 11:34:34 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 03 Dec 2009 11:33:24 +0100 | Christian Urban | deleted some dead code | changeset | files | 
| Thu, 03 Dec 2009 11:28:19 +0100 | Cezary Kaliszyk | Included all_prs and ex_prs in the lambda_prs conversion. | changeset | files | 
| Thu, 03 Dec 2009 02:53:54 +0100 | Christian Urban | further simplification | changeset | files | 
| Thu, 03 Dec 2009 02:18:21 +0100 | Christian Urban | simplified lambda_prs_conv | changeset | files | 
| Wed, 02 Dec 2009 23:31:30 +0100 | Christian Urban | deleted now obsolete argument rty everywhere | changeset | files | 
| Wed, 02 Dec 2009 23:11:50 +0100 | Christian Urban | deleted tests at the beginning of QuotMain | changeset | files | 
| Wed, 02 Dec 2009 20:54:59 +0100 | Cezary Kaliszyk | Experiments with OPTION_map | changeset | files | 
| Wed, 02 Dec 2009 17:16:44 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 02 Dec 2009 17:15:36 +0100 | Cezary Kaliszyk | More experiments with higher order quotients and theorems with non-lifted constants. | changeset | files | 
| Wed, 02 Dec 2009 16:12:41 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 02 Dec 2009 14:37:21 +0100 | Cezary Kaliszyk | Lifting to 2 different types :) | changeset | files | 
| Wed, 02 Dec 2009 14:11:46 +0100 | Cezary Kaliszyk | New APPLY_RSP which finally does automatic partial lifting :). Doesn't support same relation yet. | changeset | files | 
| Wed, 02 Dec 2009 12:07:54 +0100 | Cezary Kaliszyk | Fixed unlam for non-abstractions and updated list_induct_part proof. | changeset | files | 
| Wed, 02 Dec 2009 11:30:40 +0100 | Cezary Kaliszyk | Removed the use of 'rty' from APPLY_RSP, finally LF proofs go automatically. | changeset | files | 
| Wed, 02 Dec 2009 10:56:35 +0100 | Cezary Kaliszyk | The conversion approach works. | changeset | files | 
| Wed, 02 Dec 2009 10:30:20 +0100 | Cezary Kaliszyk | Trying a conversion based approach. | changeset | files | 
| Wed, 02 Dec 2009 09:23:48 +0100 | Cezary Kaliszyk | A bit of progress; but the object-logic vs meta-logic distinction is troublesome. | changeset | files | 
| Wed, 02 Dec 2009 07:21:10 +0100 | Cezary Kaliszyk | Added tactic for dealing with QUOT_TRUE and introducing QUOT_TRUE. | changeset | files | 
| Tue, 01 Dec 2009 19:18:43 +0100 | Cezary Kaliszyk | back in working state | changeset | files | 
| Tue, 01 Dec 2009 19:01:51 +0100 | Cezary Kaliszyk | clean | changeset | files | 
| Tue, 01 Dec 2009 18:51:14 +0100 | Christian Urban | fixed previous commit | changeset | files | 
| Tue, 01 Dec 2009 18:48:52 +0100 | Christian Urban | fixed problems with FOCUS | changeset | files | 
| Tue, 01 Dec 2009 18:41:01 +0100 | Christian Urban | added a make_inst test | changeset | files | 
| Tue, 01 Dec 2009 18:22:48 +0100 | Cezary Kaliszyk | Transformation of QUOT_TRUE assumption by any given function | changeset | files | 
| Tue, 01 Dec 2009 16:27:42 +0100 | Christian Urban | QUOT_TRUE joke | changeset | files | 
| Tue, 01 Dec 2009 14:08:56 +0100 | Cezary Kaliszyk | Removed last HOL_ss | changeset | files | 
| Tue, 01 Dec 2009 14:04:00 +0100 | Cezary Kaliszyk | more cleaning | changeset | files | 
| Tue, 01 Dec 2009 12:16:45 +0100 | Cezary Kaliszyk | Cleaning 'aps'. | changeset | files | 
| Mon, 30 Nov 2009 15:40:22 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 30 Nov 2009 15:36:49 +0100 | Christian Urban | cleaned inj_regabs_trm | changeset | files | 
| Mon, 30 Nov 2009 15:33:06 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 30 Nov 2009 15:32:14 +0100 | Cezary Kaliszyk | clean_tac rewrites the definitions the other way | changeset | files | 
| Mon, 30 Nov 2009 13:58:05 +0100 | Christian Urban | merged | changeset | files | 
| Mon, 30 Nov 2009 12:26:08 +0100 | Christian Urban | added facilities to get all stored quotient data (equiv thms etc) | changeset | files | 
| Mon, 30 Nov 2009 12:14:20 +0100 | Cezary Kaliszyk | More code cleaning | changeset | files | 
| Mon, 30 Nov 2009 11:53:20 +0100 | Cezary Kaliszyk | Code cleaning. | changeset | files | 
| Mon, 30 Nov 2009 10:16:10 +0100 | Cezary Kaliszyk | Commented clean-tac | changeset | files | 
| Mon, 30 Nov 2009 02:05:22 +0100 | Cezary Kaliszyk | Added another induction to LFex | changeset | files | 
| Sun, 29 Nov 2009 23:59:37 +0100 | Christian Urban | tried to improve the inj_repabs_trm function but left the new part commented out | changeset | files | 
| Sun, 29 Nov 2009 19:48:55 +0100 | Christian Urban | added a new version of QuotMain to experiment with qids | changeset | files | 
| Sun, 29 Nov 2009 17:47:37 +0100 | Christian Urban | started functions for qid-insertion and fixed a bug in regularise | changeset | files | 
| Sun, 29 Nov 2009 09:38:07 +0100 | Cezary Kaliszyk | Removed unnecessary HOL_ss which proved one of the subgoals. | changeset | files | 
| Sun, 29 Nov 2009 08:48:06 +0100 | Cezary Kaliszyk | Added 'TRY' to refl in clean_tac to get as far as possible. Removed unnecessary [quot_rsp] in FSet. Added necessary [quot_rsp] and one lifted thm in LamEx. | changeset | files | 
| Sun, 29 Nov 2009 03:59:18 +0100 | Christian Urban | introduced a global list of respectfulness lemmas; the attribute is [quot_rsp] | changeset | files | 
| Sun, 29 Nov 2009 02:51:42 +0100 | Christian Urban | tuned | changeset | files | 
| Sat, 28 Nov 2009 19:14:12 +0100 | Christian Urban | improved pattern matching inside the inj_repabs_tacs | changeset | files | 
| Sat, 28 Nov 2009 18:49:39 +0100 | Christian Urban | selective debugging of the inj_repabs_tac (at the moment for step 3 and 4 debugging information is printed) | changeset | files | 
| Sat, 28 Nov 2009 14:45:22 +0100 | Christian Urban | removed old inj_repabs_tac; kept only the one with (selective) debugging information | changeset | files | 
| Sat, 28 Nov 2009 14:33:04 +0100 | Christian Urban | renamed r_mk_comb_tac to inj_repabs_tac | changeset | files | 
| Sat, 28 Nov 2009 14:15:05 +0100 | Christian Urban | tuning | changeset | files | 
| Sat, 28 Nov 2009 14:03:01 +0100 | Christian Urban | tuned comments | changeset | files | 
| Sat, 28 Nov 2009 13:54:48 +0100 | Christian Urban | renamed LAMBDA_RES_TAC and WEAK_LAMBDA_RES_TAC to lower case names | changeset | files | 
| Sat, 28 Nov 2009 08:46:24 +0100 | Cezary Kaliszyk | Manually finished LF induction. | changeset | files | 
| Sat, 28 Nov 2009 08:04:23 +0100 | Cezary Kaliszyk | Moved fast instantiation to QuotMain | changeset | files | 
| Sat, 28 Nov 2009 07:44:17 +0100 | Cezary Kaliszyk | LFex proof a bit further. | changeset | files | 
| Sat, 28 Nov 2009 06:15:06 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Sat, 28 Nov 2009 06:14:50 +0100 | Cezary Kaliszyk | Looking at repabs proof in LF. | changeset | files | 
| Sat, 28 Nov 2009 05:53:31 +0100 | Christian Urban | further proper merge | changeset | files | 
| Sat, 28 Nov 2009 05:49:16 +0100 | Christian Urban | merged | changeset | files | 
| Sat, 28 Nov 2009 05:47:13 +0100 | Christian Urban | more simplification | changeset | files | 
| Sat, 28 Nov 2009 05:43:18 +0100 | Cezary Kaliszyk | Merged and tested that all works. | changeset | files | 
| Sat, 28 Nov 2009 05:29:30 +0100 | Cezary Kaliszyk | Finished and tested the new regularize | changeset | files | 
| Sat, 28 Nov 2009 05:09:22 +0100 | Christian Urban | more tuning of the repabs-tactics | changeset | files | 
| Sat, 28 Nov 2009 04:46:03 +0100 | Christian Urban | fixed examples in IntEx and FSet | changeset | files | 
| Sat, 28 Nov 2009 04:37:30 +0100 | Christian Urban | merged | changeset | files | 
| Sat, 28 Nov 2009 04:37:04 +0100 | Christian Urban | fixed previous commit | changeset | files | 
| Sat, 28 Nov 2009 04:02:54 +0100 | Cezary Kaliszyk | Cleaned all lemmas about regularisation of Ball and Bex and moved in one place. Second Ball simprox. | changeset | files | 
| Sat, 28 Nov 2009 03:17:22 +0100 | Cezary Kaliszyk | Merged comment | changeset | files | 
| Sat, 28 Nov 2009 03:07:38 +0100 | Cezary Kaliszyk | Integrated Stefan's tactic and changed substs to simps with empty context. | changeset | files | 
| Sat, 28 Nov 2009 03:06:22 +0100 | Christian Urban | some slight tuning of the apply-tactic | changeset | files | 
| Sat, 28 Nov 2009 02:54:24 +0100 | Christian Urban | annotated a proof with all steps and simplified LAMBDA_RES_TAC | changeset | files | 
| Fri, 27 Nov 2009 18:38:44 +0100 | Cezary Kaliszyk | Merge | changeset | files | 
| Fri, 27 Nov 2009 18:38:09 +0100 | Cezary Kaliszyk | The magical code from Stefan, will need to be integrated in the Simproc. | changeset | files | 
| Fri, 27 Nov 2009 13:59:52 +0100 | Christian Urban | replaced FIRST' (map rtac list) with resolve_tac list | changeset | files | 
| Fri, 27 Nov 2009 10:04:49 +0100 | Cezary Kaliszyk | Simplifying arguments; got rid of trans2_thm. | changeset | files | 
| Fri, 27 Nov 2009 09:16:32 +0100 | Cezary Kaliszyk | Cleaning of LFex. Lambda_prs fails to unify in 2 places. | changeset | files | 
| Fri, 27 Nov 2009 08:22:46 +0100 | Cezary Kaliszyk | Recommit | changeset | files | 
| Fri, 27 Nov 2009 08:15:23 +0100 | Cezary Kaliszyk | Removing arguments of tactics: absrep, rel_refl, reps_same are computed. | changeset | files | 
| Fri, 27 Nov 2009 07:16:16 +0100 | Cezary Kaliszyk | More cleaning in QuotMain, identity handling. | changeset | files | 
| Fri, 27 Nov 2009 07:00:14 +0100 | Cezary Kaliszyk | Minor cleaning | changeset | files | 
| Fri, 27 Nov 2009 04:02:20 +0100 | Christian Urban | tuned | changeset | files | 
| Fri, 27 Nov 2009 03:56:18 +0100 | Christian Urban | some tuning | changeset | files | 
| Fri, 27 Nov 2009 03:33:30 +0100 | Christian Urban | simplified gen_frees_tac and properly named abstracted variables | changeset | files | 
| Fri, 27 Nov 2009 02:58:28 +0100 | Christian Urban | removed CHANGED' | changeset | files | 
| Fri, 27 Nov 2009 02:55:56 +0100 | Christian Urban | introduced a separate lemma for id_simps | changeset | files | 
| Fri, 27 Nov 2009 02:45:54 +0100 | Christian Urban | renamed inj_REPABS to inj_repabs_trm | changeset | files | 
| Fri, 27 Nov 2009 02:44:11 +0100 | Christian Urban | tuned comments and moved slightly some code | changeset | files | 
| Fri, 27 Nov 2009 02:35:50 +0100 | Christian Urban | deleted obsolete qenv code | changeset | files | 
| Fri, 27 Nov 2009 02:23:49 +0100 | Christian Urban | renamed REGULARIZE to be regularize | changeset | files | 
| Thu, 26 Nov 2009 21:16:59 +0100 | Christian Urban | more tuning | changeset | files | 
| Thu, 26 Nov 2009 21:04:17 +0100 | Christian Urban | deleted get_fun_old and stuff | changeset | files | 
| Thu, 26 Nov 2009 21:01:53 +0100 | Christian Urban | recommited changes of comments | changeset | files | 
| Thu, 26 Nov 2009 20:32:56 +0100 | Cezary Kaliszyk | Merge Again | changeset | files | 
| Thu, 26 Nov 2009 20:32:33 +0100 | Cezary Kaliszyk | Merged | changeset | files | 
| Thu, 26 Nov 2009 20:18:36 +0100 | Christian Urban | tuned comments | changeset | files | 
| Thu, 26 Nov 2009 19:51:31 +0100 | Christian Urban | some diagnostic code for r_mk_comb | changeset | files | 
| Thu, 26 Nov 2009 16:23:24 +0100 | Christian Urban | introduced a new property for Ball and ===> on the left | changeset | files | 
| Thu, 26 Nov 2009 13:52:46 +0100 | Christian Urban | fixed QuotList | changeset | files | 
| Thu, 26 Nov 2009 13:46:00 +0100 | Christian Urban | changed left-res | changeset | files | 
| Thu, 26 Nov 2009 12:21:47 +0100 | Cezary Kaliszyk | Manually regularized akind_aty_atrm.induct | changeset | files | 
| Thu, 26 Nov 2009 10:52:24 +0100 | Cezary Kaliszyk | Playing with Monos in LFex. | changeset | files | 
| Thu, 26 Nov 2009 10:32:31 +0100 | Cezary Kaliszyk | Fixed FSet after merge. | changeset | files | 
| Thu, 26 Nov 2009 03:18:38 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 26 Nov 2009 02:31:00 +0100 | Christian Urban | test with monos | changeset | files | 
| Wed, 25 Nov 2009 21:48:32 +0100 | Cezary Kaliszyk | applic_prs | changeset | files | 
| Wed, 25 Nov 2009 15:43:12 +0100 | Christian Urban | polishing | changeset | files | 
| Wed, 25 Nov 2009 15:20:10 +0100 | Christian Urban | reordered the code | changeset | files | 
| Wed, 25 Nov 2009 14:25:29 +0100 | Cezary Kaliszyk | Moved exception handling to QuotMain and cleaned FSet. | changeset | files | 
| Wed, 25 Nov 2009 14:16:33 +0100 | Cezary Kaliszyk | Merge | changeset | files | 
| Wed, 25 Nov 2009 14:15:34 +0100 | Cezary Kaliszyk | Finished manual lifting of list_induct_part :) | changeset | files | 
| Wed, 25 Nov 2009 12:27:28 +0100 | Christian Urban | comments tuning and slight reordering | changeset | files | 
| Wed, 25 Nov 2009 11:59:49 +0100 | Cezary Kaliszyk | Merge | changeset | files | 
| Wed, 25 Nov 2009 11:58:56 +0100 | Cezary Kaliszyk | More moving from QuotMain to UnusedQuotMain | changeset | files | 
| Wed, 25 Nov 2009 11:46:59 +0100 | Christian Urban | deleted some obsolete diagnostic code | changeset | files | 
| Wed, 25 Nov 2009 11:41:42 +0100 | Cezary Kaliszyk | Removed unused things from QuotMain. | changeset | files | 
| Wed, 25 Nov 2009 10:52:21 +0100 | Cezary Kaliszyk | All examples work again. | changeset | files | 
| Wed, 25 Nov 2009 10:39:53 +0100 | Cezary Kaliszyk | cleaning in MyInt | changeset | files | 
| Wed, 25 Nov 2009 10:34:03 +0100 | Cezary Kaliszyk | lambda_prs and cleaning the existing examples. | changeset | files | 
| Wed, 25 Nov 2009 03:47:07 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 25 Nov 2009 03:45:44 +0100 | Christian Urban | fixed the problem with generalising variables; at the moment it is quite a hack | changeset | files | 
| Tue, 24 Nov 2009 20:13:16 +0100 | Cezary Kaliszyk | Ho-matching failures... | changeset | files | 
| Tue, 24 Nov 2009 19:09:29 +0100 | Christian Urban | changed unification to matching | changeset | files | 
| Tue, 24 Nov 2009 18:13:57 +0100 | Christian Urban | unification | changeset | files | 
| Tue, 24 Nov 2009 18:13:18 +0100 | Cezary Kaliszyk | Lambda & SOLVED' for new quotient_tac | changeset | files | 
| Tue, 24 Nov 2009 17:35:31 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 24 Nov 2009 17:00:53 +0100 | Cezary Kaliszyk | Conversion | changeset | files | 
| Tue, 24 Nov 2009 16:20:34 +0100 | Cezary Kaliszyk | The non-working procedure_tac. | changeset | files | 
| Tue, 24 Nov 2009 16:10:31 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 24 Nov 2009 15:31:29 +0100 | Christian Urban | use error instead of raising our own exception | changeset | files | 
| Tue, 24 Nov 2009 15:18:00 +0100 | Cezary Kaliszyk | Fixes to the tactic after quotient_tac changed. | changeset | files | 
| Tue, 24 Nov 2009 15:15:33 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 24 Nov 2009 15:15:10 +0100 | Christian Urban | added a prepare_tac | changeset | files | 
| Tue, 24 Nov 2009 14:41:47 +0100 | Cezary Kaliszyk | TRY' for clean_tac | changeset | files | 
| Tue, 24 Nov 2009 14:19:54 +0100 | Cezary Kaliszyk | Moved cleaning to QuotMain | changeset | files | 
| Tue, 24 Nov 2009 14:16:57 +0100 | Cezary Kaliszyk | New cleaning tactic | changeset | files | 
| Tue, 24 Nov 2009 13:46:36 +0100 | Christian Urban | explicit phases for the cleaning | changeset | files | 
| Tue, 24 Nov 2009 12:25:04 +0100 | Cezary Kaliszyk | Separate regularize_tac | changeset | files | 
| Tue, 24 Nov 2009 08:36:28 +0100 | Cezary Kaliszyk | Another theorem for which the new regularize differs from old one, so the goal is not proved. But it seems, that the new one is better. | changeset | files | 
| Tue, 24 Nov 2009 08:35:04 +0100 | Cezary Kaliszyk | More fixes for inj_REPABS | changeset | files | 
| Tue, 24 Nov 2009 01:36:50 +0100 | Christian Urban | addded a tactic, which sets up the three goals of the `algorithm' | changeset | files | 
| Mon, 23 Nov 2009 23:09:03 +0100 | Christian Urban | fixed the error by a temporary fix (the data of the eqivalence relation should be only its name) | changeset | files | 
| Mon, 23 Nov 2009 22:00:54 +0100 | Christian Urban | merged | changeset | files | 
| Mon, 23 Nov 2009 21:59:57 +0100 | Christian Urban | tuned some comments | changeset | files | 
| Mon, 23 Nov 2009 21:56:30 +0100 | Cezary Kaliszyk | Another not-typechecking regularized term. | changeset | files | 
| Mon, 23 Nov 2009 21:48:44 +0100 | Cezary Kaliszyk | domain_type in regularizing equality | changeset | files | 
| Mon, 23 Nov 2009 21:12:16 +0100 | Cezary Kaliszyk | More theorems lifted in the goal-directed way. | changeset | files | 
| Mon, 23 Nov 2009 20:10:39 +0100 | Cezary Kaliszyk | Finished temporary goal-directed lift_theorem wrapper. | changeset | files | 
| Mon, 23 Nov 2009 16:13:19 +0100 | Christian Urban | merged | changeset | files | 
| Mon, 23 Nov 2009 16:12:50 +0100 | Christian Urban | a version of inj_REPABS (needs to be looked at again later) | changeset | files | 
| Mon, 23 Nov 2009 15:47:14 +0100 | Cezary Kaliszyk | Fixes for atomize | changeset | files | 
| Mon, 23 Nov 2009 15:08:25 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Mon, 23 Nov 2009 15:08:09 +0100 | Cezary Kaliszyk | lift_thm with a goal. | changeset | files | 
| Mon, 23 Nov 2009 15:02:48 +0100 | Christian Urban | slight change in code layout | changeset | files | 
| Mon, 23 Nov 2009 14:40:53 +0100 | Cezary Kaliszyk | Fixes for new code | changeset | files | 
| Mon, 23 Nov 2009 14:32:11 +0100 | Cezary Kaliszyk | Removing dead code | changeset | files | 
| Mon, 23 Nov 2009 14:16:41 +0100 | Cezary Kaliszyk | Move atomize_goal to QuotMain | changeset | files | 
| Mon, 23 Nov 2009 14:05:02 +0100 | Cezary Kaliszyk | Removed second implementation of Regularize/Inject from FSet. | changeset | files | 
| Mon, 23 Nov 2009 13:55:31 +0100 | Cezary Kaliszyk | Moved new repabs_inj code to QuotMain | changeset | files | 
| Mon, 23 Nov 2009 13:46:14 +0100 | Cezary Kaliszyk | New repabs behaves the same way as old one. | changeset | files | 
| Mon, 23 Nov 2009 13:24:12 +0100 | Christian Urban | code review with Cezary | changeset | files | 
| Mon, 23 Nov 2009 10:26:59 +0100 | Cezary Kaliszyk | The other branch does not seem to work... | changeset | files | 
| Mon, 23 Nov 2009 10:04:35 +0100 | Cezary Kaliszyk | Fixes for recent changes. | changeset | files | 
| Sun, 22 Nov 2009 15:30:23 +0100 | Christian Urban | updated to Isabelle 22nd November | changeset | files | 
| Sun, 22 Nov 2009 00:01:06 +0100 | Christian Urban | a little tuning of comments | changeset | files | 
| Sat, 21 Nov 2009 23:23:01 +0100 | Christian Urban | slight tuning | changeset | files | 
| 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 | changeset | files | 
| Sat, 21 Nov 2009 14:18:31 +0100 | Christian Urban | tried to prove the repabs_inj lemma, but failed for the moment | changeset | files | 
| Sat, 21 Nov 2009 13:14:35 +0100 | Christian Urban | my first version of repabs injection | changeset | files | 
| Sat, 21 Nov 2009 11:16:48 +0100 | Christian Urban | tuned | changeset | files | 
| Sat, 21 Nov 2009 10:58:08 +0100 | Christian Urban | tunded | changeset | files | 
| Sat, 21 Nov 2009 03:12:50 +0100 | Christian Urban | tuned | changeset | files | 
| Sat, 21 Nov 2009 02:53:23 +0100 | Christian Urban | flagged qenv-stuff as obsolete | changeset | files | 
| Sat, 21 Nov 2009 02:49:39 +0100 | Christian Urban | simplified get_fun so that it uses directly rty and qty, instead of qenv | changeset | files | 
| Fri, 20 Nov 2009 13:03:01 +0100 | Christian Urban | started regularize of rtrm/qtrm version; looks quite promising | changeset | files | 
| Thu, 19 Nov 2009 14:17:10 +0100 | Christian Urban | updated to new Isabelle | changeset | files | 
| Wed, 18 Nov 2009 23:52:48 +0100 | Christian Urban | fixed the storage of qconst definitions | changeset | files | 
| Fri, 13 Nov 2009 19:32:12 +0100 | Cezary Kaliszyk | Still don't know how to do the proof automatically. | changeset | files | 
| Fri, 13 Nov 2009 16:44:36 +0100 | Christian Urban | added some tracing information to all phases of lifting to the function lift_thm | changeset | files | 
| Thu, 12 Nov 2009 13:57:20 +0100 | Cezary Kaliszyk | merge of the merge? | changeset | files | 
| Thu, 12 Nov 2009 13:56:07 +0100 | Cezary Kaliszyk | merged | changeset | files | 
| Thu, 12 Nov 2009 12:15:41 +0100 | Christian Urban | added a FIXME commment | changeset | files | 
| Thu, 12 Nov 2009 12:07:33 +0100 | Christian Urban | looking up data in quot_info works now (needs qualified string) | changeset | files | 
| Thu, 12 Nov 2009 02:54:40 +0100 | Christian Urban | changed the quotdata to be a symtab table (needs fixing) | changeset | files | 
| Thu, 12 Nov 2009 02:18:36 +0100 | Christian Urban | added a container for quotient constants (does not work yet though) | changeset | files | 
| Wed, 11 Nov 2009 22:30:43 +0100 | Cezary Kaliszyk | Lifting towards goal and manually finished the proof. | changeset | files | 
| Wed, 11 Nov 2009 18:51:59 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 11 Nov 2009 18:49:46 +0100 | Cezary Kaliszyk | Modifications while preparing the goal-directed version. | changeset | files | 
| Wed, 11 Nov 2009 11:59:22 +0100 | Christian Urban | updated to new Theory_Data and to new Isabelle | changeset | files | 
| Wed, 11 Nov 2009 10:22:47 +0100 | Cezary Kaliszyk | Removed 'Toplevel.program' for polyml 5.3 | changeset | files | 
| Tue, 10 Nov 2009 17:43:05 +0100 | Cezary Kaliszyk | Atomizing a "goal" theorems. | changeset | files | 
| Tue, 10 Nov 2009 09:32:16 +0100 | Cezary Kaliszyk | More code cleaning and commenting | changeset | files | 
| Mon, 09 Nov 2009 15:40:43 +0100 | Cezary Kaliszyk | Minor cleaning and removing of some 'handle _'. | changeset | files | 
| Mon, 09 Nov 2009 15:23:33 +0100 | Cezary Kaliszyk | Cleaning and commenting | changeset | files | 
| Mon, 09 Nov 2009 13:47:46 +0100 | Cezary Kaliszyk | Fixes for the other get_fun implementation. | changeset | files | 
| Fri, 06 Nov 2009 19:43:09 +0100 | Christian Urban | permutation lifting works now also | changeset | files | 
| Fri, 06 Nov 2009 19:26:32 +0100 | Christian Urban | merged | changeset | files | 
| Fri, 06 Nov 2009 19:26:08 +0100 | Christian Urban | updated to new Isabelle version and added a new example file | changeset | files | 
| Fri, 06 Nov 2009 17:42:20 +0100 | Cezary Kaliszyk | Minor changes | changeset | files | 
| Fri, 06 Nov 2009 11:02:11 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Fri, 06 Nov 2009 11:01:22 +0100 | Cezary Kaliszyk | fold_rsp | changeset | files | 
| Fri, 06 Nov 2009 09:48:37 +0100 | Christian Urban | tuned the code in quotient and quotient_def | changeset | files | 
| Thu, 05 Nov 2009 16:43:57 +0100 | Cezary Kaliszyk | More functionality for lifting list.cases and list.recs. | changeset | files | 
| Thu, 05 Nov 2009 13:47:41 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 05 Nov 2009 13:47:04 +0100 | Christian Urban | removed typing information from get_fun in quotient_def; *potentially* dangerous | changeset | files | 
| Thu, 05 Nov 2009 13:36:46 +0100 | Cezary Kaliszyk | Remaining fixes for polymorphic types. map_append now lifts properly with 'a list and 'b list. | changeset | files | 
| Thu, 05 Nov 2009 10:46:54 +0100 | Christian Urban | removed Simplifier.context | changeset | files | 
| Thu, 05 Nov 2009 10:23:27 +0100 | Christian Urban | replaced check_term o parse_term by read_term | changeset | files | 
| Thu, 05 Nov 2009 09:55:21 +0100 | Christian Urban | merged | changeset | files | 
| Thu, 05 Nov 2009 09:38:34 +0100 | Cezary Kaliszyk | Infrastructure for polymorphic types | changeset | files | 
| Wed, 04 Nov 2009 16:10:39 +0100 | Cezary Kaliszyk | Two new tests for get_fun. Second one fails. | changeset | files | 
| Wed, 04 Nov 2009 15:27:32 +0100 | Cezary Kaliszyk | Type instantiation in regularize | changeset | files | 
| Wed, 04 Nov 2009 14:03:46 +0100 | Cezary Kaliszyk | Description of regularize | changeset | files | 
| Wed, 04 Nov 2009 13:33:13 +0100 | Cezary Kaliszyk | Experiments with lifting partially applied constants. | changeset | files | 
| Wed, 04 Nov 2009 12:19:04 +0100 | Christian Urban | more tuning | changeset | files | 
| Wed, 04 Nov 2009 12:07:22 +0100 | Christian Urban | slightly tuned | changeset | files | 
| Wed, 04 Nov 2009 11:59:48 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 04 Nov 2009 11:59:15 +0100 | Christian Urban | separated the quotient_def into a separate file | changeset | files | 
| Wed, 04 Nov 2009 11:08:05 +0100 | Cezary Kaliszyk | Experiments in Int | changeset | files | 
| Wed, 04 Nov 2009 10:43:33 +0100 | Christian Urban | fixed definition of PLUS | changeset | files | 
| Wed, 04 Nov 2009 10:31:20 +0100 | Christian Urban | simplified the quotient_def code | changeset | files | 
| Wed, 04 Nov 2009 09:52:31 +0100 | Cezary Kaliszyk | Lifting 'fold1.simps(2)' and some cleaning. | changeset | files | 
| Tue, 03 Nov 2009 18:09:59 +0100 | Cezary Kaliszyk | Playing with alpha_refl. | changeset | files | 
| Tue, 03 Nov 2009 17:51:10 +0100 | Cezary Kaliszyk | Alpha.induct now lifts automatically. | changeset | files | 
| Tue, 03 Nov 2009 17:30:43 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 03 Nov 2009 17:30:27 +0100 | Cezary Kaliszyk | applic_prs | changeset | files | 
| 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 | changeset | files | 
| Tue, 03 Nov 2009 16:17:19 +0100 | Cezary Kaliszyk | Automatic FORALL_PRS. 'list.induct' lifts automatically. Faster ALLEX_RSP | changeset | files | 
| Tue, 03 Nov 2009 14:04:45 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Tue, 03 Nov 2009 14:04:21 +0100 | Cezary Kaliszyk | Preparing infrastructure for general FORALL_PRS | changeset | files | 
| Mon, 02 Nov 2009 18:26:55 +0100 | Christian Urban | split quotient.ML into two files | changeset | files | 
| Mon, 02 Nov 2009 18:16:19 +0100 | Christian Urban | slightly saner way of parsing the quotient_def | changeset | files | 
| Mon, 02 Nov 2009 15:39:25 +0100 | Christian Urban | merged | changeset | files | 
| Mon, 02 Nov 2009 15:38:49 +0100 | Christian Urban | changed Type.typ_match to Sign.typ_match | changeset | files | 
| Mon, 02 Nov 2009 15:38:03 +0100 | Cezary Kaliszyk | Fixes after optimization and preparing for a general FORALL_PRS | changeset | files | 
| Mon, 02 Nov 2009 14:57:56 +0100 | Cezary Kaliszyk | Optimization | changeset | files | 
| Mon, 02 Nov 2009 11:51:50 +0100 | Cezary Kaliszyk | Map does not fully work yet. | changeset | files | 
| Mon, 02 Nov 2009 11:15:26 +0100 | Cezary Kaliszyk | Fixed quotdata_lookup. | changeset | files | 
| Mon, 02 Nov 2009 09:47:49 +0100 | Christian Urban | fixed problem with maps_update | changeset | files | 
| Mon, 02 Nov 2009 09:39:29 +0100 | Christian Urban | merged | changeset | files | 
| Mon, 02 Nov 2009 09:33:48 +0100 | Christian Urban | fixed the problem with types in map | changeset | files | 
| Sat, 31 Oct 2009 11:20:55 +0100 | Cezary Kaliszyk | Automatic computation of application preservation and manually finished "alpha.induct". Slow... | changeset | files | 
| Fri, 30 Oct 2009 19:03:53 +0100 | Cezary Kaliszyk | Regularize for equalities and a better tactic. "alpha.cases" now lifts. | changeset | files | 
| Fri, 30 Oct 2009 18:31:06 +0100 | Cezary Kaliszyk | Regularization | changeset | files | 
| Fri, 30 Oct 2009 16:37:09 +0100 | Christian Urban | merged | changeset | files | 
| Fri, 30 Oct 2009 16:35:43 +0100 | Christian Urban | added some facts about fresh and support of lam | changeset | files | 
| Fri, 30 Oct 2009 16:24:07 +0100 | Cezary Kaliszyk | Finally merged the code of the versions of regularize and tested examples. | changeset | files | 
| Fri, 30 Oct 2009 15:52:47 +0100 | Cezary Kaliszyk | Lemmas about fv. | changeset | files | 
| Fri, 30 Oct 2009 15:35:42 +0100 | Christian Urban | changed the order of rfv and reformulated a3 with rfv | changeset | files | 
| Fri, 30 Oct 2009 15:32:04 +0100 | Christian Urban | merged | changeset | files | 
| Fri, 30 Oct 2009 15:30:33 +0100 | Christian Urban | not sure what changed here | changeset | files | 
| Fri, 30 Oct 2009 15:28:44 +0100 | Christian Urban | added fv-function | changeset | files | 
| Fri, 30 Oct 2009 15:22:59 +0100 | Cezary Kaliszyk | The proper real_alpha | changeset | files | 
| Fri, 30 Oct 2009 14:25:37 +0100 | Cezary Kaliszyk | Finding applications and duplicates filtered out in abstractions | changeset | files | 
| Fri, 30 Oct 2009 12:22:03 +0100 | Cezary Kaliszyk | Cleaning also in Lam | changeset | files | 
| Fri, 30 Oct 2009 11:25:29 +0100 | Cezary Kaliszyk | Cleaning of the interface to lift. | changeset | files | 
| Thu, 29 Oct 2009 17:35:03 +0100 | Cezary Kaliszyk | Tried manually lifting real_alpha | changeset | files | 
| Thu, 29 Oct 2009 13:30:11 +0100 | Cezary Kaliszyk | More tests in Lam | changeset | files | 
| Thu, 29 Oct 2009 13:29:03 +0100 | Cezary Kaliszyk | Cleaning of 'map id' and 'prod_fun id id' in lower_defs. | changeset | files | 
| Thu, 29 Oct 2009 12:09:31 +0100 | Cezary Kaliszyk | Using subst for identity definition. | changeset | files | 
| Thu, 29 Oct 2009 08:46:34 +0100 | Cezary Kaliszyk | Lifting of the 3 lemmas in LamEx | changeset | files | 
| Thu, 29 Oct 2009 08:06:49 +0100 | Cezary Kaliszyk | Fixed wrong CARD definition and removed the "Does not work anymore" comment. | changeset | files | 
| Thu, 29 Oct 2009 07:29:12 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 28 Oct 2009 20:01:20 +0100 | Christian Urban | updated some definitions; had to give sometimes different names; somewhere I introduced a bug, since not everything is working anymore (needs fixing!) | changeset | files | 
| Wed, 28 Oct 2009 19:46:15 +0100 | Christian Urban | ported all constant definitions to new scheme | changeset | files | 
| Wed, 28 Oct 2009 19:36:52 +0100 | Christian Urban | fixed the definition of alpha; this *breaks* some of the experiments | changeset | files | 
| Wed, 28 Oct 2009 18:08:38 +0100 | Cezary Kaliszyk | disambiguate ===> syntax | changeset | files | 
| Wed, 28 Oct 2009 17:38:37 +0100 | Cezary Kaliszyk | More cleaning in Lam code | changeset | files | 
| Wed, 28 Oct 2009 17:17:21 +0100 | Cezary Kaliszyk | cleaned FSet | changeset | files | 
| Wed, 28 Oct 2009 16:48:57 +0100 | Cezary Kaliszyk | Some cleaning | changeset | files | 
| Wed, 28 Oct 2009 16:16:38 +0100 | Cezary Kaliszyk | Cleaning the unnecessary theorems in 'IntEx'. | changeset | files | 
| Wed, 28 Oct 2009 16:11:28 +0100 | Cezary Kaliszyk | Fix also in the general procedure. | changeset | files | 
| Wed, 28 Oct 2009 16:06:19 +0100 | Cezary Kaliszyk | merge | changeset | files | 
| Wed, 28 Oct 2009 16:05:59 +0100 | Cezary Kaliszyk | Fixes | changeset | files | 
| Wed, 28 Oct 2009 15:48:38 +0100 | Christian Urban | updated all definitions | changeset | files | 
| Wed, 28 Oct 2009 15:25:36 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 28 Oct 2009 15:25:11 +0100 | Christian Urban | added infrastructure for defining lifted constants | changeset | files | 
| Wed, 28 Oct 2009 14:59:24 +0100 | Cezary Kaliszyk | First experiments with Lambda | changeset | files | 
| Wed, 28 Oct 2009 12:22:06 +0100 | Cezary Kaliszyk | Fixed mistake in const generation, will postpone this. | changeset | files | 
| Wed, 28 Oct 2009 10:29:00 +0100 | Cezary Kaliszyk | More finshed proofs and cleaning | changeset | files | 
| Wed, 28 Oct 2009 10:17:07 +0100 | Cezary Kaliszyk | Proof of append_rsp | changeset | files | 
| Wed, 28 Oct 2009 01:49:31 +0100 | Christian Urban | merged | changeset | files | 
| Wed, 28 Oct 2009 01:48:45 +0100 | Christian Urban | added a function for matching types | changeset | files | 
| Tue, 27 Oct 2009 18:05:45 +0100 | Cezary Kaliszyk | Manual conversion of equality to equivalence allows lifting append_assoc. | changeset | files | 
| Tue, 27 Oct 2009 18:02:35 +0100 | Cezary Kaliszyk | Simplfied interface to repabs_injection. | changeset | files | 
| Tue, 27 Oct 2009 17:08:47 +0100 | Cezary Kaliszyk | map_append lifted automatically. | changeset | files | 
| Tue, 27 Oct 2009 16:15:56 +0100 | Cezary Kaliszyk | Manually lifted Map_Append. | changeset | files | 
| Tue, 27 Oct 2009 15:00:15 +0100 | Cezary Kaliszyk | Merged | changeset | files | 
| Tue, 27 Oct 2009 14:59:00 +0100 | Cezary Kaliszyk | Fixed APPLY_RSP vs Cong in the InjRepAbs tactic. | changeset | files | 
| Tue, 27 Oct 2009 14:46:38 +0100 | Christian Urban | tuned | changeset | files | 
| Tue, 27 Oct 2009 14:15:40 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 27 Oct 2009 14:14:30 +0100 | Christian Urban | added equiv-thm to the quot_info | changeset | files | 
| Tue, 27 Oct 2009 12:20:57 +0100 | Cezary Kaliszyk | Simplifying FSet with new functions. | changeset | files | 
| Tue, 27 Oct 2009 11:43:02 +0100 | Christian Urban | added an example about lambda-terms | changeset | files | 
| Tue, 27 Oct 2009 11:27:53 +0100 | Christian Urban | made quotients compatiple with Nominal; updated keyword file | changeset | files | 
| Tue, 27 Oct 2009 11:03:38 +0100 | Christian Urban | merged | changeset | files | 
| Tue, 27 Oct 2009 09:01:12 +0100 | Cezary Kaliszyk | Completely cleaned Int. | changeset | files | 
| Tue, 27 Oct 2009 07:46:52 +0100 | Cezary Kaliszyk | Further reordering in Int code. | changeset | files | 
| Mon, 26 Oct 2009 19:35:30 +0100 | Cezary Kaliszyk | Simplifying Int. | changeset | files | 
| Mon, 26 Oct 2009 15:32:17 +0100 | Cezary Kaliszyk | Merge | changeset | files | 
| Mon, 26 Oct 2009 15:31:53 +0100 | Cezary Kaliszyk | Simplifying Int and Working on map | changeset | files | 
| Mon, 26 Oct 2009 14:18:26 +0100 | Christian Urban | merged | changeset | files | 
| Mon, 26 Oct 2009 14:16:32 +0100 | Cezary Kaliszyk | Simplifying code in int | changeset | files | 
| Mon, 26 Oct 2009 13:33:28 +0100 | Cezary Kaliszyk | Symmetry of integer addition | changeset | files | 
| Mon, 26 Oct 2009 11:55:36 +0100 | Cezary Kaliszyk | Finished the code for adding lower defs, and more things moved to QuotMain | changeset | files | 
| Mon, 26 Oct 2009 11:34:02 +0100 | Cezary Kaliszyk | Making all the definitions from the original ones | changeset | files | 
| Mon, 26 Oct 2009 10:20:20 +0100 | Cezary Kaliszyk | Finished COND_PRS proof. | changeset | files | 
| Mon, 26 Oct 2009 10:02:50 +0100 | Cezary Kaliszyk | Cleaning and fixing. | changeset | files | 
| Mon, 26 Oct 2009 02:06:01 +0100 | Christian Urban | updated with quotient_def | changeset | files | 
| Sun, 25 Oct 2009 23:44:41 +0100 | Christian Urban | added code for declaring map-functions | changeset | files | 
| Sun, 25 Oct 2009 01:31:04 +0200 | Christian Urban | added "print_quotients" command to th ekeyword file | changeset | files | 
| Sun, 25 Oct 2009 01:15:03 +0200 | Christian Urban | proved the two lemmas in QuotScript (reformulated them without leading forall) | changeset | files | 
| Sun, 25 Oct 2009 00:14:40 +0200 | Christian Urban | added data-storage about the quotients | changeset | files | 
| Sat, 24 Oct 2009 22:52:23 +0200 | Christian Urban | added another example file about integers (see HOL/Int.thy) | changeset | files | 
| Sat, 24 Oct 2009 18:17:38 +0200 | Christian Urban | changed the definitions of liftet constants to use fun_maps | changeset | files | 
| Sat, 24 Oct 2009 17:29:20 +0200 | cek | Merge | changeset | files | 
| Sat, 24 Oct 2009 17:29:27 +0200 | Cezary Kaliszyk | Finally lifted induction, with some manually added simplification lemmas. | changeset | files | 
| Sat, 24 Oct 2009 16:31:07 +0200 | Christian Urban | changed encoding from utf8 to ISO8 (needed to work with xemacs) | changeset | files | 
| Sat, 24 Oct 2009 16:15:33 +0200 | cek | Merge | changeset | files | 
| Sat, 24 Oct 2009 16:15:58 +0200 | Cezary Kaliszyk | Preparing infrastructire for LAMBDA_PRS | changeset | files | 
| Sat, 24 Oct 2009 16:09:05 +0200 | Christian Urban | moved the map_funs setup into QuotMain | changeset | files | 
| Sat, 24 Oct 2009 14:00:18 +0200 | Cezary Kaliszyk | Finally completely lift the previously lifted theorems + clean some old stuff | changeset | files | 
| Sat, 24 Oct 2009 13:00:54 +0200 | Cezary Kaliszyk | More infrastructure for automatic lifting of theorems lifted before | changeset | files | 
| Sat, 24 Oct 2009 10:16:53 +0200 | Cezary Kaliszyk | More infrastructure for automatic lifting of theorems lifted before | changeset | files | 
| Sat, 24 Oct 2009 08:34:14 +0200 | cek | Undid wrong merge | changeset | files | 
| Sat, 24 Oct 2009 08:29:11 +0200 | cek | Tried rolling back | changeset | files | 
| Sat, 24 Oct 2009 08:24:26 +0200 | cek | Cleaning the mess | changeset | files | 
| Sat, 24 Oct 2009 08:09:40 +0200 | cek | Merge | changeset | files | 
| Sat, 24 Oct 2009 08:09:09 +0200 | cek | Better tactic and simplified the proof further | changeset | files | 
| Sat, 24 Oct 2009 01:33:29 +0200 | Christian Urban | fixed problem with incorrect ABS/REP name | changeset | files | 
| Fri, 23 Oct 2009 18:20:06 +0200 | Cezary Kaliszyk | Stronger tactic, simpler proof. | changeset | files | 
| Fri, 23 Oct 2009 16:34:20 +0200 | Cezary Kaliszyk | Split Finite Set example into separate file | changeset | files | 
| Fri, 23 Oct 2009 16:01:13 +0200 | Cezary Kaliszyk | eqsubst_tac | changeset | files | 
| Fri, 23 Oct 2009 11:24:43 +0200 | Cezary Kaliszyk | Trying to get a simpler lemma with the whole infrastructure | changeset | files | 
| Fri, 23 Oct 2009 09:21:45 +0200 | Cezary Kaliszyk | Using RANGE tactical allows getting rid of the quotients immediately. | changeset | files | 
| Thu, 22 Oct 2009 17:35:40 +0200 | Cezary Kaliszyk | Further developing the tactic and simplifying the proof | changeset | files | 
| Thu, 22 Oct 2009 16:24:02 +0200 | Cezary Kaliszyk | res_forall_rsp_tac further simplifies the proof | changeset | files | 
| Thu, 22 Oct 2009 16:10:06 +0200 | Cezary Kaliszyk | Working on the proof and the tactic. | changeset | files | 
| Thu, 22 Oct 2009 15:45:05 +0200 | Cezary Kaliszyk | The proof gets simplified | changeset | files | 
| Thu, 22 Oct 2009 15:44:16 +0200 | Cezary Kaliszyk | Removed an assumption | changeset | files | 
| Thu, 22 Oct 2009 15:02:01 +0200 | Cezary Kaliszyk | The proof now including manually unfolded higher-order RES_FORALL_RSP. | changeset | files | 
| Thu, 22 Oct 2009 13:45:48 +0200 | Cezary Kaliszyk | The problems with 'abs' term. | changeset | files | 
| Thu, 22 Oct 2009 11:43:12 +0200 | Cezary Kaliszyk | Simplified the proof with some tactic... Still hangs sometimes. | changeset | files | 
| Thu, 22 Oct 2009 10:45:33 +0200 | Cezary Kaliszyk | More proof | changeset | files | 
| Thu, 22 Oct 2009 10:38:00 +0200 | Cezary Kaliszyk | Got rid of instantiations in the proof | changeset | files | 
| Thu, 22 Oct 2009 06:51:27 +0200 | Cezary Kaliszyk | Removed some debugging messages | changeset | files | 
| Thu, 22 Oct 2009 01:59:17 +0200 | Christian Urban | tuned and attempted to store data about the quotients (does not work yet) | changeset | files | 
| Thu, 22 Oct 2009 01:16:42 +0200 | Christian Urban | tuned | changeset | files | 
| Thu, 22 Oct 2009 01:15:01 +0200 | Christian Urban | slight tuning | changeset | files | 
| Wed, 21 Oct 2009 18:30:42 +0200 | Christian Urban | fixed my_reg | changeset | files | 
| Wed, 21 Oct 2009 16:13:39 +0200 | Cezary Kaliszyk | Reorganization of the construction part | changeset | files | 
| Wed, 21 Oct 2009 15:01:50 +0200 | Cezary Kaliszyk | Simplified proof more | changeset | files | 
| Wed, 21 Oct 2009 14:30:29 +0200 | Cezary Kaliszyk | Cleaning the code | changeset | files | 
| Wed, 21 Oct 2009 14:15:22 +0200 | Cezary Kaliszyk | Further reorganization | changeset | files | 
| Wed, 21 Oct 2009 14:09:06 +0200 | Cezary Kaliszyk | Further reorganizing the file | changeset | files | 
| Wed, 21 Oct 2009 13:47:39 +0200 | Cezary Kaliszyk | Reordering | changeset | files | 
| Wed, 21 Oct 2009 11:50:53 +0200 | Cezary Kaliszyk | cterm_instantiate also fails for some strange reason... | changeset | files | 
| Wed, 21 Oct 2009 10:55:32 +0200 | Cezary Kaliszyk | preparing arguments for res_inst_tac | changeset | files | 
| Wed, 21 Oct 2009 10:30:29 +0200 | Cezary Kaliszyk | Trying res_inst_tac | changeset | files | 
| Tue, 20 Oct 2009 19:46:22 +0200 | Christian Urban | started to write code for storing data about the quotients | changeset | files | 
| Tue, 20 Oct 2009 09:37:22 +0200 | Christian Urban | some minor tuning | changeset | files | 
| Tue, 20 Oct 2009 09:31:34 +0200 | Christian Urban | tuned and fixed the earlier fix | changeset | files | 
| Tue, 20 Oct 2009 09:21:18 +0200 | Christian Urban | fixed the abs case in my_reg and added an app case | changeset | files | 
| Tue, 20 Oct 2009 01:17:22 +0200 | Christian Urban | my version of regularise (still needs to be completed) | changeset | files | 
| Tue, 20 Oct 2009 00:12:05 +0200 | Christian Urban | moved the map-info and fun-info section to quotient.ML | changeset | files | 
| Sun, 18 Oct 2009 10:34:53 +0200 | Cezary Kaliszyk | Test if we can already do sth with the transformed theorem. | changeset | files | 
| Sun, 18 Oct 2009 08:44:16 +0200 | Christian Urban | slight fix and tuning | changeset | files | 
| Sun, 18 Oct 2009 00:52:10 +0200 | Christian Urban | the command "quotient" can now define more than one quotient at the same time; quotients need to be separated by and | changeset | files | 
| Sat, 17 Oct 2009 16:06:54 +0200 | Cezary Kaliszyk | Partial simplification of the proof | changeset | files | 
| Sat, 17 Oct 2009 15:42:57 +0200 | Cezary Kaliszyk | Some QUOTIENTS | changeset | files | 
| Sat, 17 Oct 2009 14:16:57 +0200 | Cezary Kaliszyk | Only QUOTIENSs are left to fnish proof | changeset | files | 
| Sat, 17 Oct 2009 12:44:58 +0200 | Cezary Kaliszyk | More higher order unification problems | changeset | files | 
| Sat, 17 Oct 2009 12:31:48 +0200 | Cezary Kaliszyk | Merged | changeset | files | 
| Sat, 17 Oct 2009 12:31:36 +0200 | Cezary Kaliszyk | Simplified | changeset | files | 
| Sat, 17 Oct 2009 12:20:56 +0200 | Cezary Kaliszyk | Further in the proof | changeset | files | 
| Sat, 17 Oct 2009 11:54:50 +0200 | Cezary Kaliszyk | compose_tac works with the full instantiation. | changeset | files | 
| Sat, 17 Oct 2009 12:19:06 +0200 | Christian Urban | slightly simplified get_fun function | changeset | files | 
| Sat, 17 Oct 2009 10:40:54 +0200 | Cezary Kaliszyk | The instantiated version is the same modulo beta | changeset | files | 
| Sat, 17 Oct 2009 10:07:52 +0200 | Cezary Kaliszyk | Fully manually instantiated. Still fails... | changeset | files | 
| Sat, 17 Oct 2009 09:04:24 +0200 | Cezary Kaliszyk | Little progress with match/instantiate | changeset | files | 
| Fri, 16 Oct 2009 19:21:05 +0200 | Cezary Kaliszyk | Fighting with the instantiation | changeset | files | 
| Fri, 16 Oct 2009 17:05:52 +0200 | Cezary Kaliszyk | Symmetric version of REP_ABS_RSP | changeset | files | 
| Fri, 16 Oct 2009 16:51:01 +0200 | Cezary Kaliszyk | Progressing with the proof | changeset | files | 
| Fri, 16 Oct 2009 10:54:31 +0200 | Cezary Kaliszyk | Finally fix get_fun. | changeset | files | 
| Fri, 16 Oct 2009 08:48:56 +0200 | Cezary Kaliszyk | A fix for one fun_map; doesn't work for more. | changeset | files | 
| Fri, 16 Oct 2009 03:26:54 +0200 | Christian Urban | fixed the problem with function types; but only type_of works; cterm_of does not work | changeset | files | 
| Thu, 15 Oct 2009 16:51:24 +0200 | Cezary Kaliszyk | Description of the problem with get_fun. | changeset | files | 
| Thu, 15 Oct 2009 16:36:20 +0200 | Cezary Kaliszyk | A proper build_goal_term function. | changeset | files | 
| Thu, 15 Oct 2009 12:06:00 +0200 | Cezary Kaliszyk | Cleaning the code | changeset | files | 
| Thu, 15 Oct 2009 11:57:33 +0200 | Cezary Kaliszyk | Merged | changeset | files | 
| Thu, 15 Oct 2009 11:56:30 +0200 | Cezary Kaliszyk | Cleaning the proofs | changeset | files | 
| Thu, 15 Oct 2009 11:55:52 +0200 | Cezary Kaliszyk | Cleaning the code, part 4 | changeset | files | 
| Thu, 15 Oct 2009 11:53:11 +0200 | Christian Urban | slightly improved tyRel | changeset | files | 
| Thu, 15 Oct 2009 11:42:14 +0200 | Cezary Kaliszyk | Reordering the code, part 3 | changeset | files | 
| Thu, 15 Oct 2009 11:29:38 +0200 | Cezary Kaliszyk | Reordering the code, part 2. | changeset | files | 
| Thu, 15 Oct 2009 11:25:25 +0200 | Cezary Kaliszyk | Reordering the code, part 1. | changeset | files | 
| Thu, 15 Oct 2009 11:20:50 +0200 | Cezary Kaliszyk | Minor cleaning. | changeset | files | 
| Thu, 15 Oct 2009 11:17:27 +0200 | Cezary Kaliszyk | The definition of Fold1 | changeset | files | 
| Thu, 15 Oct 2009 10:25:23 +0200 | Cezary Kaliszyk | A number of lemmas for REGULARIZE_TAC and regularizing card1. | changeset | files | 
| Wed, 14 Oct 2009 18:13:16 +0200 | Cezary Kaliszyk | Proving the proper RepAbs version | changeset | files | 
| Wed, 14 Oct 2009 16:23:49 +0200 | Cezary Kaliszyk | Forgot to save, second part of the commit | changeset | files | 
| Wed, 14 Oct 2009 16:23:32 +0200 | Cezary Kaliszyk | Manually regularized list_induct2 | changeset | files | 
| Wed, 14 Oct 2009 12:05:39 +0200 | Cezary Kaliszyk | Fixed bug in regularise types. Now we can regularise list.induct. | changeset | files | 
| Wed, 14 Oct 2009 11:23:55 +0200 | Cezary Kaliszyk | Function for checking recursively if lifting is needed | changeset | files | 
| Wed, 14 Oct 2009 09:50:13 +0200 | Cezary Kaliszyk | Merge | changeset | files | 
| Wed, 14 Oct 2009 09:47:16 +0200 | Cezary Kaliszyk | Proper handling of non-lifted quantifiers, testing type freezing. | changeset | files | 
| Tue, 13 Oct 2009 22:22:15 +0200 | Christian Urban | slight simplification of atomize_thm | changeset | files | 
| Tue, 13 Oct 2009 18:01:54 +0200 | Cezary Kaliszyk | atomize_thm and meta_quantify. | changeset | files | 
| Tue, 13 Oct 2009 13:37:07 +0200 | Cezary Kaliszyk | Regularizing HOL all. | changeset | files | 
| Tue, 13 Oct 2009 11:38:35 +0200 | Cezary Kaliszyk | ":" is used for being in a set, "IN" means something else... | changeset | files | 
| Tue, 13 Oct 2009 11:03:55 +0200 | Cezary Kaliszyk | First (untested) version of regularize for abstractions. | changeset | files | 
| Tue, 13 Oct 2009 09:26:19 +0200 | Christian Urban | restored old version | changeset | files | 
| Tue, 13 Oct 2009 00:02:22 +0200 | Christian Urban | tuned | changeset | files | 
| Mon, 12 Oct 2009 23:39:14 +0200 | Christian Urban | slightly modified the parser | changeset | files | 
| Mon, 12 Oct 2009 23:16:20 +0200 | Christian Urban | deleted diagnostic code | changeset | files | 
| Mon, 12 Oct 2009 23:06:14 +0200 | Christian Urban | added quotient command (you need to update isar-keywords-prove.el) | changeset | files | 
| Mon, 12 Oct 2009 22:44:16 +0200 | Christian Urban | added new keyword | changeset | files | 
| Mon, 12 Oct 2009 16:31:29 +0200 | Cezary Kaliszyk | Bounded quantifier | changeset | files | 
| Mon, 12 Oct 2009 15:47:27 +0200 | Cezary Kaliszyk | The tyREL function. | changeset | files | 
| Mon, 12 Oct 2009 14:30:50 +0200 | Christian Urban | started some strange functions | changeset | files | 
| Mon, 12 Oct 2009 13:58:31 +0200 | Cezary Kaliszyk | Further with the manual proof | changeset | files | 
| Fri, 09 Oct 2009 17:05:45 +0200 | Cezary Kaliszyk | Further experiments with proving induction manually | changeset | files | 
| Fri, 09 Oct 2009 15:03:43 +0200 | Cezary Kaliszyk | Testing if I can prove the regularized version of induction manually | changeset | files | 
| Thu, 08 Oct 2009 14:27:50 +0200 | Christian Urban | exported parts of QuotMain into a separate ML-file | changeset | files | 
| Tue, 06 Oct 2009 15:11:30 +0200 | Christian Urban | consistent usage of rty (for the raw, unquotient type); tuned a bit the Isar | changeset | files | 
| Tue, 06 Oct 2009 11:56:23 +0200 | Christian Urban | simplified typedef_quot_type_tac (using MetaSimplifier.rewrite_rule instead of the simplifier) | changeset | files | 
| Tue, 06 Oct 2009 11:41:35 +0200 | Christian Urban | renamed unlam_def to unabs_def (matching the function abs_def in drule.ML) | changeset | files | 
| Tue, 06 Oct 2009 11:36:08 +0200 | Christian Urban | tuned; nothing serious | changeset | files | 
| Tue, 06 Oct 2009 09:28:59 +0200 | Christian Urban | another improvement to unlam_def | changeset | files | 
| Tue, 06 Oct 2009 02:02:51 +0200 | Christian Urban | one further improvement to unlam_def | changeset | files | 
| Tue, 06 Oct 2009 01:50:13 +0200 | Christian Urban | simplified the unlam_def function | changeset | files | 
| Mon, 05 Oct 2009 11:54:02 +0200 | Christian Urban | added an explicit syntax-argument to the function make_def (is needed if the user gives an syntax annotation for quotient types) | changeset | files | 
| Mon, 05 Oct 2009 11:24:32 +0200 | Christian Urban | used prop_of to get the term of a theorem (replaces crep_thm) | changeset | files | 
| Fri, 02 Oct 2009 11:10:21 +0200 | Cezary Kaliszyk | Merged | changeset | files | 
| Fri, 02 Oct 2009 11:09:33 +0200 | Cezary Kaliszyk | First theorem with quantifiers. Learned how to use sledgehammer. | changeset | files | 
| Thu, 01 Oct 2009 16:10:14 +0200 | Christian Urban | simplified the storage of the map-functions by using TheoryDataFun | changeset | files | 
| Wed, 30 Sep 2009 16:57:09 +0200 | Cezary Kaliszyk | Just one atomize is enough for the currently lifted theorems. Properly lift 'all' and 'Ex'. | changeset | files | 
| Tue, 29 Sep 2009 22:35:48 +0200 | Christian Urban | used new cong_tac | changeset | files | 
| Tue, 29 Sep 2009 17:46:18 +0200 | Cezary Kaliszyk | First version of handling of the universal quantifier | changeset | files | 
| Tue, 29 Sep 2009 15:58:14 +0200 | Cezary Kaliszyk | Handling abstraction correctly. | changeset | files | 
| Tue, 29 Sep 2009 13:38:27 +0200 | Cezary Kaliszyk | second test | changeset | files | 
| Tue, 29 Sep 2009 13:24:57 +0200 | Cezary Kaliszyk | Test line | changeset | files | 
| Tue, 29 Sep 2009 11:55:37 +0200 | Cezary Kaliszyk | Partially fix lifting of card_suc. The quantified variable still needs to be changed. | changeset | files | 
| Tue, 29 Sep 2009 10:49:31 +0200 | Cezary Kaliszyk | Tested new build_goal and removed old one, eq_reflection is included in atomize, card_suc tests. | changeset | files | 
| Tue, 29 Sep 2009 09:58:02 +0200 | Cezary Kaliszyk | Checked again with the version on my hard-drive backedup yesterday and fixed small whitespace issues. | changeset | files | 
| Tue, 29 Sep 2009 09:26:22 +0200 | Cezary Kaliszyk | Merged | changeset | files | 
| Mon, 28 Sep 2009 23:17:29 +0200 | Christian Urban | added name to prove | changeset | files | 
| Mon, 28 Sep 2009 19:24:55 +0200 | Christian Urban | consistent state | changeset | files | 
| Mon, 28 Sep 2009 19:22:28 +0200 | Christian Urban | some tuning of my code | changeset | files | 
| Mon, 28 Sep 2009 19:15:19 +0200 | Cezary Kaliszyk | Cleanup | changeset | files | 
| Mon, 28 Sep 2009 19:10:27 +0200 | Cezary Kaliszyk | Merged | changeset | files | 
| Mon, 28 Sep 2009 18:59:04 +0200 | Cezary Kaliszyk | Cleaning the code with Makarius | changeset | files | 
| Mon, 28 Sep 2009 15:37:38 +0200 | Cezary Kaliszyk | Instnatiation with a schematic variable | changeset | files | 
| Mon, 28 Sep 2009 02:39:44 +0200 | Christian Urban | added ctxt as explicit argument to build_goal; tuned | changeset | files | 
| Fri, 25 Sep 2009 19:26:18 +0200 | Christian Urban | slightly tuned the comment for unlam | changeset | files | 
| Fri, 25 Sep 2009 17:08:50 +0200 | Christian Urban | fixed a bug in my code: function typedef_term constructs now now the correct term when the relation is called x | changeset | files | 
| Fri, 25 Sep 2009 16:50:11 +0200 | Christian Urban | tuned slightly one proof | changeset | files | 
| Fri, 25 Sep 2009 14:50:35 +0200 | Cezary Kaliszyk | A version of the tactic that exports variables correctly. | changeset | files | 
| Fri, 25 Sep 2009 09:38:16 +0200 | Cezary Kaliszyk | Minor cleaning: whitespace, commas etc. | changeset | files | 
| Thu, 24 Sep 2009 17:43:26 +0200 | Cezary Kaliszyk | Correctly handling abstractions while building goals | changeset | files | 
| Thu, 24 Sep 2009 13:32:52 +0200 | Cezary Kaliszyk | Minor cleanup | changeset | files | 
| Thu, 24 Sep 2009 11:38:20 +0200 | Cezary Kaliszyk | Found the source for the exception and added a handle for it. | changeset | files | 
| Thu, 24 Sep 2009 09:09:46 +0200 | Cezary Kaliszyk | Make the tactic use Trueprop_cong and atomize. | changeset | files | 
| Wed, 23 Sep 2009 16:57:56 +0200 | Cezary Kaliszyk | Proper code for getting the prop out of the theorem. | changeset | files | 
| Wed, 23 Sep 2009 16:44:56 +0200 | Cezary Kaliszyk | Using "atomize" the versions with arbitrary Trueprops can be proven. | changeset | files | 
| Tue, 22 Sep 2009 17:39:52 +0200 | Cezary Kaliszyk | Proper definition of CARD and some properties of it. | changeset | files | 
| Tue, 22 Sep 2009 09:42:27 +0200 | Christian Urban | some comments | changeset | files | 
| Mon, 21 Sep 2009 18:18:29 +0200 | Christian Urban | merged | changeset | files | 
| Mon, 21 Sep 2009 18:18:01 +0200 | Christian Urban | slight tuning | changeset | files | 
| Mon, 21 Sep 2009 16:45:44 +0200 | Cezary Kaliszyk | The tactic with REPEAT, CHANGED and a proper simpset. | changeset | files | 
| Mon, 21 Sep 2009 10:53:01 +0200 | Cezary Kaliszyk | Merged with my changes from the morning: | changeset | files | 
| Sun, 20 Sep 2009 05:48:49 +0100 | Ning | some more beautification | changeset | files | 
| Sun, 20 Sep 2009 05:18:36 +0100 | Ning | beautification of some proofs | changeset | files | 
| Fri, 18 Sep 2009 17:30:33 +0200 | Cezary Kaliszyk | Added more useful quotient facts. | changeset | files | 
| Fri, 18 Sep 2009 13:44:06 +0200 | Cezary Kaliszyk | Testing the tactic further. | changeset | files | 
| Thu, 17 Sep 2009 16:55:11 +0200 | Cezary Kaliszyk | The tactic still only for fset | changeset | files | 
| Thu, 17 Sep 2009 12:06:06 +0200 | Cezary Kaliszyk | Infrastructure for the tactic | changeset | files | 
| Wed, 16 Sep 2009 11:50:41 +0200 | Cezary Kaliszyk | More naming/binding suggestions from Makarius | changeset | files | 
| Tue, 15 Sep 2009 11:31:35 +0200 | Cezary Kaliszyk | Code cleanup | changeset | files | 
| Tue, 15 Sep 2009 10:00:34 +0200 | Cezary Kaliszyk | Cleaning the code | changeset | files | 
| Tue, 15 Sep 2009 09:59:56 +0200 | Cezary Kaliszyk | Generalized interpretation, works for all examples. | changeset | files | 
| Fri, 28 Aug 2009 17:12:19 +0200 | Cezary Kaliszyk | Fixes after suggestions from Makarius: | changeset | files | 
| Fri, 28 Aug 2009 10:01:25 +0200 | Cezary Kaliszyk | More examples. | changeset | files | 
| Thu, 27 Aug 2009 09:04:39 +0200 | Cezary Kaliszyk | Use metavariables in the 'non-lambda' definitions | changeset | files | 
| Wed, 26 Aug 2009 11:31:55 +0200 | Cezary Kaliszyk | Make both kinds of definitions. | changeset | files | 
| Tue, 25 Aug 2009 17:37:50 +0200 | Cezary Kaliszyk | Changed to the use of "modern interface" | changeset | files | 
| Tue, 25 Aug 2009 14:37:11 +0200 | Cezary Kaliszyk | Initial version of the function that builds goals. | changeset | files | 
| Tue, 25 Aug 2009 10:35:28 +0200 | Cezary Kaliszyk | - Build an interpretation for fset from ML level and use it | changeset | files | 
| Tue, 25 Aug 2009 00:30:23 +0200 | Christian Urban | added the prove command | changeset | files | 
| Fri, 21 Aug 2009 13:56:20 +0200 | Cezary Kaliszyk | Fixed | changeset | files | 
| Fri, 21 Aug 2009 13:36:58 +0200 | Christian Urban | tuned | changeset | files | 
| Thu, 20 Aug 2009 14:44:29 +0200 | cek | UNION - Append theorem | changeset | files | 
| Thu, 20 Aug 2009 10:31:44 +0200 | Christian Urban | update | changeset | files | 
| Tue, 18 Aug 2009 14:04:51 +0200 | Christian Urban | updated slightly | changeset | files | 
| Tue, 11 Aug 2009 12:29:15 +0200 | Christian Urban | initial commit | changeset | files |