Sat, 25 Jun 2011 21:28:24 +0100 |
Christian Urban |
an alternative FCB for Abs_lst1; seems simpler but not as simple as I thought; not sure whether it generalises to multiple binders.
|
file |
diff |
annotate
|
Thu, 23 Jun 2011 22:21:43 +0100 |
Christian Urban |
the simplifier can simplify "sort (atom a)" if a is a concrete atom type declared with atom_decl
|
file |
diff |
annotate
|
Thu, 16 Jun 2011 20:07:03 +0100 |
Christian Urban |
got rid of the boolean flag in the raw_equivariance function
|
file |
diff |
annotate
|
Tue, 14 Jun 2011 19:11:44 +0100 |
Christian Urban |
tuned some proofs
|
file |
diff |
annotate
|
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
|
file |
diff |
annotate
|
Tue, 14 Jun 2011 11:43:06 +0100 |
Christian Urban |
tuned
|
file |
diff |
annotate
|
Mon, 06 Jun 2011 13:11:04 +0100 |
Christian Urban |
slightly stronger property in fundef_ex_prop
|
file |
diff |
annotate
|
Sun, 05 Jun 2011 16:58:18 +0100 |
Christian Urban |
added a more general lemma fro fundef_ex1
|
file |
diff |
annotate
|
Thu, 02 Jun 2011 15:35:33 +0100 |
Christian Urban |
removed dead code
|
file |
diff |
annotate
|
Tue, 10 May 2011 07:47:06 +0100 |
Christian Urban |
updated to new Isabelle (> 9 May)
|
file |
diff |
annotate
|
Mon, 09 May 2011 04:49:58 +0100 |
Christian Urban |
merged
|
file |
diff |
annotate
|
Tue, 03 May 2011 13:09:08 +0100 |
Christian Urban |
proved that lfp is equivariant (that simplifies equivariance proofs of inductively defined predicates)
|
file |
diff |
annotate
|
Mon, 09 May 2011 04:46:43 +0100 |
Christian Urban |
more on pearl-paper
|
file |
diff |
annotate
|
Fri, 22 Apr 2011 00:18:25 +0800 |
Christian Urban |
more to the pearl paper
|
file |
diff |
annotate
|
Sun, 10 Apr 2011 07:41:52 +0800 |
Christian Urban |
eqvt of supp and fresh is proved using equivariance infrastructure
|
file |
diff |
annotate
|
Fri, 08 Apr 2011 03:47:50 +0800 |
Christian Urban |
eqvt_lambda without eta-expansion
|
file |
diff |
annotate
|
Mon, 14 Mar 2011 16:35:59 +0100 |
Christian Urban |
equivariance for All and Ex can be proved in terms of their definition
|
file |
diff |
annotate
|
Fri, 11 Mar 2011 08:51:39 +0000 |
Christian Urban |
more on the paper
|
file |
diff |
annotate
|
Tue, 01 Mar 2011 00:14:02 +0000 |
Christian Urban |
a bit more tuning
|
file |
diff |
annotate
|
Mon, 28 Feb 2011 15:21:10 +0000 |
Christian Urban |
split the library into a basics file; merged Nominal_Eqvt into Nominal_Base
|
file |
diff |
annotate
|
Fri, 25 Feb 2011 21:23:30 +0000 |
Christian Urban |
some slight polishing
|
file |
diff |
annotate
|
Thu, 24 Feb 2011 16:26:11 +0000 |
Christian Urban |
added a lemma about fresh_star and Abs
|
file |
diff |
annotate
|
Thu, 27 Jan 2011 04:24:17 +0100 |
Christian Urban |
the proofs with eqvt_at
|
file |
diff |
annotate
|
Wed, 19 Jan 2011 19:41:50 +0100 |
Christian Urban |
added obtain_fresh lemma; tuned Lambda.thy
|
file |
diff |
annotate
|
Wed, 19 Jan 2011 18:56:28 +0100 |
Christian Urban |
ported some of the old proofs to serve as testcases
|
file |
diff |
annotate
|
Wed, 19 Jan 2011 17:11:10 +0100 |
Christian Urban |
added Minimal file to test things
|
file |
diff |
annotate
|
Tue, 18 Jan 2011 19:27:30 +0100 |
Christian Urban |
defined properly substitution
|
file |
diff |
annotate
|
Tue, 18 Jan 2011 17:19:50 +0100 |
Christian Urban |
removed finiteness assumption from set_rename_perm
|
file |
diff |
annotate
|
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
|
file |
diff |
annotate
|
Tue, 18 Jan 2011 06:55:18 +0100 |
Christian Urban |
modified the renaming_perm lemmas
|
file |
diff |
annotate
|
Mon, 17 Jan 2011 12:34:11 +0000 |
Christian Urban |
moved high level code from LamTest into the main libraries.
|
file |
diff |
annotate
|
Fri, 14 Jan 2011 14:22:25 +0000 |
Christian Urban |
strengthened renaming lemmas
|
file |
diff |
annotate
|
Mon, 10 Jan 2011 11:36:55 +0000 |
Christian Urban |
a few lemmas about freshness for at and at_base
|
file |
diff |
annotate
|
Thu, 06 Jan 2011 13:28:04 +0000 |
Christian Urban |
some further lemmas for fsets
|
file |
diff |
annotate
|
Mon, 03 Jan 2011 16:19:27 +0000 |
Christian Urban |
simple cases for string rule inductions
|
file |
diff |
annotate
|
Fri, 31 Dec 2010 12:12:59 +0000 |
Christian Urban |
added small example for strong inductions; functions still need a sorry
|
file |
diff |
annotate
|
Sun, 19 Dec 2010 07:43:32 +0000 |
Christian Urban |
a stronger statement for at_set_avoiding
|
file |
diff |
annotate
|
Thu, 16 Dec 2010 08:42:48 +0000 |
Christian Urban |
simple cases for strong inducts done; infrastructure for the difficult ones is there
|
file |
diff |
annotate
|
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)
|
file |
diff |
annotate
|
Tue, 07 Dec 2010 19:16:09 +0000 |
Christian Urban |
moved general theorems into the libraries
|
file |
diff |
annotate
|
Mon, 29 Nov 2010 08:01:09 +0000 |
Christian Urban |
isarfied some of the high-level proofs
|
file |
diff |
annotate
|
Mon, 29 Nov 2010 05:10:02 +0000 |
Christian Urban |
completed proofs in Foo2
|
file |
diff |
annotate
|
Sun, 28 Nov 2010 16:37:34 +0000 |
Christian Urban |
completed the strong exhausts rules for Foo2 using general lemmas
|
file |
diff |
annotate
|
Sat, 27 Nov 2010 23:00:16 +0000 |
Christian Urban |
tuned proof to reduce number of warnings
|
file |
diff |
annotate
|
Sat, 27 Nov 2010 22:55:29 +0000 |
Christian Urban |
disabled the Foo examples, because of heavy work
|
file |
diff |
annotate
|
Sun, 21 Nov 2010 02:17:19 +0000 |
Christian Urban |
added example Foo2.thy
|
file |
diff |
annotate
|
Sun, 14 Nov 2010 16:34:47 +0000 |
Christian Urban |
merged Nominal-General directory into Nominal; renamed Abs.thy to Nominal2_Abs.thy
|
file |
diff |
annotate
| base
|
Sat, 20 Mar 2010 02:46:07 +0100 |
Christian Urban |
moved infinite_Un into mainstream Isabelle; moved permute_boolI/E lemmas
|
file |
diff |
annotate
|
Tue, 02 Mar 2010 15:05:35 +0100 |
Christian Urban |
updated (added lemma about commuting permutations)
|
file |
diff |
annotate
|
Thu, 25 Feb 2010 07:48:33 +0100 |
Christian Urban |
moved Nominal to "toplevel"
|
file |
diff |
annotate
| base
|