History log of /seL4-l4v-master/l4v/isabelle/src/HOL/Bali/Trans.thy
Revision Date Author Comments
# 5385dbfa 16-Jan-2018 wenzelm <none@none>

standardized towards new-style formal comments: isabelle update_comments;


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

more canonical names


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

isabelle update_cartouches -c -t;


# 713cd402 13-Mar-2014 nipkow <none@none>

enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions

--HG--
extra : rebase_source : 4103bf02b2df95e1e84808f766f131292beef893


# 1f0f0995 27-Mar-2012 wenzelm <none@none>

simplified statements and proofs;


# 48096e82 03-Dec-2010 wenzelm <none@none>

recoded latin1 as utf8;
use textcomp for some text symbols where it appears appropriate;


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

modernized/unified some specifications;


# 518f89a0 28-Jun-2010 haftmann <none@none>

modernized specifications


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

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


# e9e35adb 09-Feb-2010 wenzelm <none@none>

removed obsolete CVS Ids;


# 803f34cc 09-Feb-2010 wenzelm <none@none>

modernized syntax translations, using mostly abbreviation/notation;
minor tuning;


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

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


# 39f27693 20-Apr-2009 haftmann <none@none>

power operation on functions with syntax o^; power operation on relations with syntax ^^


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

arbitrary is undefined


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

Renamed inductive2 to inductive.


# fd8a9d0e 11-Dec-2006 berghofe <none@none>

Adapted to new inductive definition package.


# 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


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


# ee7e563d 16-Jul-2002 schirmer <none@none>

Added conditional and (&&) and or (||).


# 2f4a8a50 12-Jul-2002 schirmer <none@none>

little Bugfix


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