History log of /seL4-l4v-10.1.1/isabelle/src/HOL/MicroJava/JVM/JVMListExample.thy
Revision Date Author Comments
# d9ef7419 02-Jan-2016 wenzelm <none@none>

isabelle update_cartouches -c -t;


# ba266305 07-Oct-2015 wenzelm <none@none>

isabelle update_cartouches;


# ba81fa63 02-Nov-2014 wenzelm <none@none>

modernized header;


# 3e0fffd8 24-Feb-2013 wenzelm <none@none>

prefer stateless 'ML_val' for tests;


# 5c541a07 13-Dec-2011 wenzelm <none@none>

modernized specifications;


# 39224b86 21-Oct-2011 bulwahn <none@none>

replacing code_inline by code_unfold, removing obsolete code_unfold, code_inline del now that the ancient code generator is removed


# 45dbe2de 05-Aug-2011 Andreas Lochbihler <none@none>

replace old SML code generator by new code generator in MicroJava/JVM and /BV


# baea5702 01-Mar-2010 haftmann <none@none>

replaced a couple of constsdefs by definitions (also some old primrecs by modern ones)


# c040dd23 24-Nov-2009 haftmann <none@none>

backported parts of abstract byte code verifier from AFP/Jinja

--HG--
extra : rebase_source : 1d943bc92831d0a92004a43f72ff37eb352bf23f


# 6df0cf4c 11-Aug-2009 haftmann <none@none>

temporary adjustment to dubious state of eta expansion in recfun_codegen


# 16362266 07-Oct-2008 haftmann <none@none>

arbitrary is undefined


# e900a18c 29-Sep-2008 wenzelm <none@none>

code example: back to individual ML commands, which are now thread-safe;


# 26e57f9b 30-Sep-2007 wenzelm <none@none>

avoid internal names;


# dcff929a 20-Aug-2007 wenzelm <none@none>

theory header: more precise imports;


# ab8c4365 10-Aug-2007 haftmann <none@none>

dropped code generator setup garbage


# c7efe280 30-Jul-2007 wenzelm <none@none>

tuned ML declarations;


# 5c5055dc 10-May-2007 haftmann <none@none>

consts in consts_code Isar commands are now referred to by usual term syntax


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

more robust syntax for definition/abbreviation/notation;


# d4c61f5a 31-Oct-2006 haftmann <none@none>

adapted to new serializer syntax


# 1cb68668 20-Oct-2006 haftmann <none@none>

slight cleanup


# ef558aa9 11-Oct-2006 haftmann <none@none>

added code generator setup


# 5940937f 14-Jan-2006 wenzelm <none@none>

generated code: raise Match instead of ERROR;


# 4f793cc3 25-Aug-2005 berghofe <none@none>

Adapted to new code generator syntax.


# c2997950 12-Jul-2005 berghofe <none@none>

Auxiliary functions to be used in generated code are now defined using "attach".


# 2c59a0ee 01-Jul-2005 berghofe <none@none>

Corrected implementation of arbitrary on cname.


# a7060872 17-Jun-2005 haftmann <none@none>

migrated theory headers to new format


# f2b06eca 30-Apr-2002 kleing <none@none>

tuned


# e9d3ce8e 19-Apr-2002 berghofe <none@none>

wf is no longer implemented by true (due to change in definition of class_rec).


# d1d14dc6 09-Mar-2002 kleing <none@none>

canonical start state


# 0ce3fe7b 28-Feb-2002 kleing <none@none>

fixed missing label


# 6c89dca9 26-Feb-2002 kleing <none@none>

introduces SystemClasses and BVExample


# 0e7365d8 21-Feb-2002 kleing <none@none>

new document


# 55d58ddc 20-Dec-2001 berghofe <none@none>

cast_ok and match_exception_entry no longer disabled (thanks to
improvement of code generator).


# 70d75cca 17-Dec-2001 kleing <none@none>

fixed JVMListExample


# db94ef87 15-Dec-2001 kleing <none@none>

exception merge, doesn't work yet


# 6be7ad2c 10-Dec-2001 berghofe <none@none>

Example for code generator.