Nominal/Parser.thy
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.
Tue, 23 Mar 2010 08:33:48 +0100 Cezary Kaliszyk Move examples which create more permutations out
Mon, 22 Mar 2010 18:29:29 +0100 Cezary Kaliszyk equivp_cheat can be removed for all one-permutation examples.
Mon, 22 Mar 2010 17:21:27 +0100 Cezary Kaliszyk Got rid of alpha_bn_rsp_cheat.
Mon, 22 Mar 2010 14:07:07 +0100 Cezary Kaliszyk fv_rsp proved automatically.
Sat, 20 Mar 2010 09:27:28 +0100 Cezary Kaliszyk Use 'alpha_bn_refl' to get rid of one of the sorrys.
Sat, 20 Mar 2010 08:04:59 +0100 Cezary Kaliszyk Prove reflp for all relations.
Fri, 19 Mar 2010 18:42:57 +0100 Cezary Kaliszyk Automatically derive support for datatypes with at-most one binding per constructor.
Fri, 19 Mar 2010 14:54:30 +0100 Cezary Kaliszyk Use fs typeclass in showing finite support + some cheat cleaning.
Fri, 19 Mar 2010 10:24:16 +0100 Cezary Kaliszyk Remove atom_decl from the parser.
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.
Thu, 18 Mar 2010 15:13:20 +0100 Cezary Kaliszyk Rename "_property" to ".property"
Thu, 18 Mar 2010 14:05:49 +0100 Cezary Kaliszyk case names also for _induct
Thu, 18 Mar 2010 12:32:03 +0100 Cezary Kaliszyk Case_Names for _inducts. Does not work for _induct yet.
Thu, 18 Mar 2010 12:09:59 +0100 Cezary Kaliszyk Added fv,bn,distinct,perm to the simplifier.
Thu, 18 Mar 2010 08:03:42 +0100 Cezary Kaliszyk Move most of the exporting out of the parser.
Thu, 18 Mar 2010 07:43:44 +0100 Cezary Kaliszyk Prove pseudo-inject (eq-iff) on the exported level and rename appropriately.
Thu, 18 Mar 2010 07:35:44 +0100 Cezary Kaliszyk Prove eqvts on exported terms.
Thu, 18 Mar 2010 07:26:36 +0100 Cezary Kaliszyk Clean 'Lift', start working only on exported things in Parser.
Wed, 17 Mar 2010 17:11:23 +0100 Christian Urban merged
Wed, 17 Mar 2010 15:13:31 +0100 Christian Urban made paper to compile
Wed, 17 Mar 2010 12:18:35 +0100 Cezary Kaliszyk cheat_alpha_eqvt no longer needed. Cleaned the tracing messages.
Wed, 17 Mar 2010 08:39:46 +0100 Cezary Kaliszyk Lifting theorems with compound fv and compound alpha.
Tue, 16 Mar 2010 20:07:13 +0100 Cezary Kaliszyk Revert 7c8cd6eae8e2, now all proofs in Term5 go through, both recursive and not.
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.
Mon, 15 Mar 2010 17:42:17 +0100 Cezary Kaliszyk fv_eqvt_cheat no longer needed.
Mon, 15 Mar 2010 14:32:05 +0100 Cezary Kaliszyk derive "inducts" from "induct" instead of lifting again is much faster.
Mon, 15 Mar 2010 11:50:12 +0100 Cezary Kaliszyk cheat_alpha_eqvt no longer needed; the proofs work.
Mon, 15 Mar 2010 10:07:15 +0100 Cezary Kaliszyk explicit flag "cheat_equivp"
Sat, 13 Mar 2010 13:49:15 +0100 Christian Urban started supp-fv proofs (is going to work)
Fri, 12 Mar 2010 12:42:35 +0100 Cezary Kaliszyk Still don't know how to prove supp=fv for simplest Let...
Thu, 11 Mar 2010 20:49:31 +0100 Cezary Kaliszyk Do not fail if the finite support proof fails.
Thu, 11 Mar 2010 19:41:11 +0100 Christian Urban support of atoms at the end of Abs.thy
Thu, 11 Mar 2010 17:47:29 +0100 Cezary Kaliszyk Show that the new types are in finite support typeclass.
Thu, 11 Mar 2010 15:11:57 +0100 Cezary Kaliszyk Remove "_raw" from lifted theorems.
Thu, 11 Mar 2010 14:05:36 +0100 Cezary Kaliszyk The cheats described explicitely.
Thu, 11 Mar 2010 13:34:45 +0100 Cezary Kaliszyk With the 4 cheats, all examples fully lift.
Thu, 11 Mar 2010 12:30:53 +0100 Cezary Kaliszyk Lift alpha_bn_constants.
Thu, 11 Mar 2010 12:26:24 +0100 Cezary Kaliszyk Lifting constants.
Thu, 11 Mar 2010 11:32:37 +0100 Cezary Kaliszyk Lifting constants works for all examples.
Thu, 11 Mar 2010 11:25:18 +0100 Cezary Kaliszyk Equivp working only on the standard alpha-equivalences.
Thu, 11 Mar 2010 11:20:50 +0100 Cezary Kaliszyk explicit cheat_fv_eqvt
Thu, 11 Mar 2010 11:15:14 +0100 Cezary Kaliszyk extract build_eqvts_tac.
Thu, 11 Mar 2010 10:39:29 +0100 Cezary Kaliszyk build_eqvts no longer requires permutations.
Thu, 11 Mar 2010 10:22:24 +0100 Cezary Kaliszyk Add explicit alpha_eqvt_cheat.
Thu, 11 Mar 2010 10:10:23 +0100 Cezary Kaliszyk Export tactic out of alpha_eqvt.
Wed, 10 Mar 2010 16:51:15 +0100 Christian Urban merged
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)
Wed, 10 Mar 2010 15:34:13 +0100 Cezary Kaliszyk Undoing mistakenly committed parser experiments.
Wed, 10 Mar 2010 15:32:51 +0100 Cezary Kaliszyk alpha_eqvt for recursive term1.
Wed, 10 Mar 2010 13:10:00 +0100 Cezary Kaliszyk Linked parser to fv and alpha.
Wed, 10 Mar 2010 12:48:38 +0100 Christian Urban parser produces ordered bn-fun information
Tue, 09 Mar 2010 22:08:38 +0100 Christian Urban added bn-information, but it is not yet ordered according to the dts
Tue, 09 Mar 2010 16:24:39 +0100 Cezary Kaliszyk A version of Fv that takes into account recursive and non-recursive bindings.
Mon, 08 Mar 2010 15:01:26 +0100 Christian Urban merged
Mon, 08 Mar 2010 15:01:01 +0100 Christian Urban updated to new Isabelle
Mon, 08 Mar 2010 11:12:15 +0100 Cezary Kaliszyk More fine-grained nominal restriction for debugging.
Fri, 05 Mar 2010 14:55:21 +0100 Cezary Kaliszyk Lift fv and bn eqvts; no need to lift alpha_eqvt.
Thu, 04 Mar 2010 18:57:23 +0100 Cezary Kaliszyk Lift distinct.
Thu, 04 Mar 2010 15:55:53 +0100 Cezary Kaliszyk Added lifting of pseudo-injectivity, commented out the code again and enabled the weird examples.
less more (0) -60 tip