History log of /seL4-l4v-master/l4v/isabelle/src/HOL/Nominal/Examples/Crary.thy
Revision Date Author Comments
# ed7a971e 05-Jan-2019 wenzelm <none@none>

isabelle update -u control_cartouches;


# 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;


# 7237bdd9 02-Sep-2013 wenzelm <none@none>

tuned proofs -- clarified flow of facts wrt. calculation;


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

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


# e4ce7496 05-Sep-2012 wenzelm <none@none>

tuned proofs;


# 7a4b6a89 21-Feb-2011 wenzelm <none@none>

modernized specifications;


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

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


# d7136b86 21-Sep-2009 Christian Urban <urbanc@in.tum.de>

tuned some proofs


# 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.


# 65b87b21 28-Aug-2008 krauss <none@none>

more function -> fun


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

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


# bb8359f5 15-Apr-2008 urbanc <none@none>

removed test artefacts


# 3e9d6497 14-Apr-2008 wenzelm <none@none>

avoid duplicate fact bindings;


# f37f3054 19-Oct-2007 wenzelm <none@none>

tuned proofs: avoid implicit prems;


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

added type constraints to resolve syntax ambiguities;


# 9b2ff487 31-Jul-2007 narboux <none@none>

undo a change in last commit : give a single name to the inversion lemmas for the same inductive type


# e49ecba4 30-Jul-2007 urbanc <none@none>

updated some of the definitions and proofs


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

Renamed inductive2 to inductive.


# 2d5eacb6 21-Jun-2007 narboux <none@none>

fine tune automatic generation of inversion lemmas


# 9ad1fb76 14-Jun-2007 wenzelm <none@none>

tuned proofs: avoid implicit prems;


# f65d7568 12-Jun-2007 urbanc <none@none>

added the Q_Unit rule (was missing) and adjusted the proof accordingly


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

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


# 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


# a3f83b1e 07-Apr-2007 narboux <none@none>

perm_simp can now simplify using the rules (a,b) o a = b and (a,b) o b = a


# 750e2c22 04-Apr-2007 narboux <none@none>

add a few details in the Fst and Snd cases of unicity proof


# 95572f33 28-Mar-2007 berghofe <none@none>

- Renamed <predicate>_eqvt to <predicate>.eqvt
- Renamed induct_weak to weak_induct


# 33050f45 27-Mar-2007 urbanc <none@none>

tuned proofs (taking full advantage of nominal_inductive)


# fcd84069 27-Mar-2007 berghofe <none@none>

Adapted to changes in nominal_inductive.


# ffb06a8d 22-Mar-2007 krauss <none@none>

fixed function syntax


# 0b0f967d 22-Mar-2007 urbanc <none@none>

tuned some proofs


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

Unified function syntax


# 7e86f9a9 06-Mar-2007 narboux <none@none>

correct typo in latex output


# 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


# d284efa6 17-Jan-2007 urbanc <none@none>

tuned a bit the proofs


# 670d91f6 16-Jan-2007 urbanc <none@none>

formalisation of Crary's chapter on logical relations
(in the book on Advanced Topics in Type Systems) done
by Narboux and Urban