History log of /seL4-l4v-master/l4v/isabelle/src/HOL/Nominal/Examples/Lam_Funs.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;


# 06329277 13-Aug-2013 wenzelm <none@none>

standardized symbols via "isabelle update_sub_sup", excluding src/Pure and src/Tools/WWW_Find;


# 1ff366c9 13-Dec-2008 berghofe <none@none>

Modified nominal_primrec to make it work with local theories, unified syntax
with the one used by fun(ction) and new version of primrec command.


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

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


# 40225442 01-May-2008 urbanc <none@none>

extended to be a library of general facts about the lambda calculus


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

tuned proofs and comments


# b0bfde44 03-May-2007 urbanc <none@none>

deleted some unnecessary type-annotations


# 6384e974 01-May-2007 urbanc <none@none>

tuned some proofs and changed variable names in some definitions of Nominal.thy


# 72455713 28-Mar-2007 urbanc <none@none>

adapted to new nominal_inductive


# a1877829 21-Mar-2007 krauss <none@none>

Unified function syntax


# 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


# 7d38f996 27-Nov-2006 urbanc <none@none>

added the function for free variables of a lambda-term, which is a
tad more difficult to define than capture-avoiding substitution


# ef19da37 27-Nov-2006 urbanc <none@none>

adapted function definitions to new syntax


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

more robust syntax for definition/abbreviation/notation;


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

new file for defining functions in the lambda-calculus