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

isabelle update -u control_cartouches;


# d4c96e26 15-Jun-2018 nipkow <none@none>

empty -> Map.empty


# f5796e6d 14-Feb-2018 wenzelm <none@none>

more symbols;


# 5385dbfa 16-Jan-2018 wenzelm <none@none>

standardized towards new-style formal comments: isabelle update_comments;


# d9ef7419 02-Jan-2016 wenzelm <none@none>

isabelle update_cartouches -c -t;


# 883895af 31-Aug-2015 wenzelm <none@none>

prefer symbols;


# 4eae0352 10-Nov-2014 wenzelm <none@none>

proper context for assume_tac (atac remains as fall-back without context);


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

modernized header;


# e91e0c03 16-Feb-2014 blanchet <none@none>

folded 'Option.set' into BNF-generated 'set_option'


# ee5744a6 21-Feb-2012 wenzelm <none@none>

tuned proofs;


# 450834a8 14-Jan-2012 wenzelm <none@none>

tuned white space;


# f4961062 20-Nov-2011 wenzelm <none@none>

eliminated obsolete "standard";


# 3ec8ee77 18-Feb-2011 wenzelm <none@none>

modernized specifications;


# 5b59da77 13-Sep-2010 nipkow <none@none>

renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI


# bb8268b1 07-Sep-2010 nipkow <none@none>

expand_fun_eq -> ext_iff
expand_set_eq -> set_ext_iff
Naming in line now with multisets


# 9d68725b 26-Jul-2010 wenzelm <none@none>

modernized/unified some specifications;


# 6bc0017f 02-Mar-2010 wenzelm <none@none>

cleanup type translations;


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

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


# 942a6e5f 24-Feb-2010 wenzelm <none@none>

modernized syntax declarations, and make them actually work with authentic syntax;


# f7c6aef2 16-Jan-2010 haftmann <none@none>

modernized syntax


# b391ac6a 04-Mar-2009 nipkow <none@none>

Made Option a separate theory and renamed option_map to Option.map


# 61bc019f 09-Aug-2007 haftmann <none@none>

re-eliminated Option.thy


# c32053dd 29-Jul-2007 wenzelm <none@none>

replaced make_imp by rev_mp;


# d9f4c279 20-Dec-2005 paulson <none@none>

removed or modified some instances of [iff]


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

migrated theory headers to new format


# 33b1b845 21-Jun-2004 kleing <none@none>

Merged in license change from Isabelle2004


# 67a49057 25-Jul-2003 nipkow <none@none>

Replaced \<leadsto> by \<rightharpoonup>


# efd5dc29 14-May-2003 nipkow <none@none>

*** empty log message ***


# c4a5cd8d 31-Oct-2002 schirmer <none@none>

"Definite Assignment Analysis" included, with proof of correctness. Large adjustments of type safety proof and soundness proof of the axiomatic semantics were necessary. Completeness proof of the loop rule of the axiomatic semantic was altered. So the additional polymorphic variants of some rules could be removed.


# 74d67fdb 30-Sep-2002 berghofe <none@none>

Adapted to new simplifier.


# 4803de87 26-Sep-2002 paulson <none@none>

Converted Fun to Isar style.
Moved Pi, funcset, restrict from Fun.thy to Library/FuncSet.thy.
Renamed constant "Fun.op o" to "Fun.comp"


# e5e60fc1 10-Jul-2002 schirmer <none@none>

Added unary and binary operations like (+,-,<, ...); Added smallstep semantics (no proofs about it yet).


# 55bc1056 22-Feb-2002 schirmer <none@none>

Added check for field/method access to operational semantics and proved the acesses valid.


# 2dc32281 28-Jan-2002 wenzelm <none@none>

GPLed;


# 8af5fde7 28-Jan-2002 wenzelm <none@none>

tuned header;


# 77d49ccc 28-Jan-2002 schirmer <none@none>

Isabelle/Bali sources;