History log of /seL4-l4v-master/l4v/isabelle/src/HOL/Nominal/Examples/Weakening.thy
Revision Date Author Comments
# 17bc899d 18-Aug-2017 wenzelm <none@none>

session-qualified theory imports: isabelle imports -U -i -d '~~/src/Benchmarks' -a;


# 66281660 26-May-2016 wenzelm <none@none>

isabelle update_cartouches -c -t;


# 35f7dccd 23-Feb-2016 nipkow <none@none>

more canonical names


# 079cde2d 17-Oct-2009 wenzelm <none@none>

eliminated hard tabulators, guessing at each author's individual tab-width;
tuned headers;


# 2932189d 22-May-2008 urbanc <none@none>

made the naming of the induction principles consistent: weak_induct is
induct and induct is strong_induct


# cd5ecf2a 12-Mar-2008 urbanc <none@none>

tuned


# 56bcf215 11-Feb-2008 urbanc <none@none>

tuned proofs and comments


# 5a64f8c1 31-Dec-2007 urbanc <none@none>

tuned proofs and comments


# 28e1a742 19-Dec-2007 urbanc <none@none>

polishing of some proofs


# b99031e1 21-Oct-2007 urbanc <none@none>

further comments


# 0a6d3df1 21-Oct-2007 urbanc <none@none>

polished the proofs and added a version of the weakening lemma that does not use the variable convention


# a62c3c6d 12-Aug-2007 wenzelm <none@none>

added type constraints to resolve syntax ambiguities;


# ffa009b0 11-Jul-2007 berghofe <none@none>

Renamed inductive2 to inductive.


# f86abfd6 19-Apr-2007 berghofe <none@none>

nominal_inductive no longer proves equivariance.


# ead401a2 12-Apr-2007 urbanc <none@none>

tuned the proof of lemma pt_list_set_fresh (as suggested by Randy Pollack) and tuned the syntax for sub_contexts


# aeeb8c2a 27-Mar-2007 urbanc <none@none>

adapted to new nominal_inductive infrastructure


# 228c94bd 06-Mar-2007 urbanc <none@none>

major update of the nominal package; there is now an infrastructure
for equivariance lemmas which eases definitions of nominal functions


# 1601d366 02-Feb-2007 urbanc <none@none>

added an infrastructure that allows the user to declare lemmas to be equivariance lemmas; the intention is to use these lemmas in automated tools but also can be employed by the user


# 64a24614 23-Nov-2006 urbanc <none@none>

fixed some typos


# ec4eb96e 23-Nov-2006 urbanc <none@none>

tuned the proof of the strong induction principle


# 8951a9fe 17-Nov-2006 urbanc <none@none>

added an intro lemma for freshness of products; set up
the simplifier so that it can deal with the compact and
long notation for freshness constraints (FIXME: it should
also be able to deal with the special case of freshness
of atoms)


# cd65d9bc 16-Nov-2006 wenzelm <none@none>

more robust syntax for definition/abbreviation/notation;


# 20a0be49 15-Nov-2006 urbanc <none@none>

replaced exists_fresh lemma with a version formulated with obtains;
old lemma is available as exists_fresh' (still needed in apply-scripts)


# f6d23f77 14-Nov-2006 wenzelm <none@none>

inductive2: canonical specification syntax;


# 07b16468 30-Oct-2006 urbanc <none@none>

new file for defining functions in the lambda-calculus


# 45dc766b 18-Oct-2006 urbanc <none@none>

adapted to Stefan's new inductive package and cleaning up


# 6def9b19 10-Oct-2006 urbanc <none@none>

made some proof look more like the ones in Barendregt


# 7517dca8 11-Sep-2006 wenzelm <none@none>

induct method: renamed 'fixing' to 'arbitrary';


# 2f44ec19 02-Jul-2006 urbanc <none@none>

added more infrastructure for the recursion combinator


# c9c286d8 28-Apr-2006 berghofe <none@none>

Capitalized theory names.


# 3d1cbf70 11-Jan-2006 urbanc <none@none>

tuned proofs


# 44150cfb 11-Jan-2006 urbanc <none@none>

tuned the eqvt-proof


# 50a00001 05-Dec-2005 urbanc <none@none>

tuned


# 040d25a8 05-Dec-2005 urbanc <none@none>

tuned


# e6991bfb 03-Dec-2005 urbanc <none@none>

tuned


# 58bada02 30-Nov-2005 urbanc <none@none>

changed "fresh:" to "avoiding:" and cleaned up the weakening example


# 07822287 30-Nov-2005 urbanc <none@none>

adapted to the new nominal_induction


# 2f93a07d 27-Nov-2005 urbanc <none@none>

some small tuning


# 67c74de6 07-Nov-2005 urbanc <none@none>

Initial commit of the theory "Weakening".