tuned;
authorwenzelm
Mon, 28 Jan 2002 18:48:25 +0100
changeset 12856 17ae8bbb46cb
parent 12855 21225338f8db
child 12857 a4386cc9b1c3
tuned;
src/HOL/Bali/document/root.tex
--- a/src/HOL/Bali/document/root.tex	Mon Jan 28 17:52:13 2002 +0100
+++ b/src/HOL/Bali/document/root.tex	Mon Jan 28 18:48:25 2002 +0100
@@ -1,22 +1,10 @@
 
 \documentclass[11pt,a4paper]{book}
 \usepackage{isabelle,isabellesym}
-
-% further packages required for unusual symbols (see also isabellesym.sty)
 \usepackage{latexsym}
-%\usepackage{amssymb}
-%\usepackage[english]{babel}
-%\usepackage[latin1]{inputenc}
-%\usepackage[only,bigsqcap]{stmaryrd}
-%\usepackage{wasysym}
-%\usepackage{eufrak}
-%\usepackage{textcomp}
-%\usepackage{marvosym}
-
-% this should be the last package used
+\usepackage{graphicx}
 \usepackage{pdfsetup}
 
-% proper setup for best-style documents
 \urlstyle{rm}
 \isabellestyle{it}
 
@@ -37,16 +25,20 @@
 {\begin{isabellebody}}
 {\end{isabellebody}}
 
+
 \begin{document}
 
-\title{Java Source and Bytecode Formalizations in Isabelle: Bali\\
-  {\large -- VerifiCard Project Deliverables -- }}
+\title{Java Source and Bytecode Formalizations in Isabelle: Bali}
 \author{Gerwin Klein \and Tobias Nipkow \and David von Oheimb \and
   Leonor Prensa Nieto \and Norbert Schirmer \and Martin Strecker}
 \maketitle
 
 \tableofcontents
 
+\begin{center}
+  \includegraphics[scale=0.7]{session_graph}
+\end{center}
+
 \parindent 0pt\parskip 0.5ex
 \chapter{Overview}
 These theories, called Bali,  model and analyse different aspects of the 
@@ -95,142 +87,136 @@
 
 Overview of the theories:
 \begin{description}
-\item [Basis.thy] 
+\item[Basis] 
 Some basic definitions and settings not specific to JavaCard but missing in HOL.
 
-\item [Table.thy]
+\item[Table]
 Definition and some properties of a lookup table to map various names 
 (like class names or method names) to some content (like classes or methods).
 
-\item[Name.thy]
+\item[Name]
 Definition of various names (class names, variable names, package names,...)
 
-\item[Value.thy]
+\item[Value]
 JavaCard expression values (Boolean, Integer, Addresses,...)
 
-\item[Type.thy]
+\item[Type]
 JavaCard types. Primitive types (Boolean, Integer,...) and reference types 
 (Classes, Interfaces, Arrays,...)
 
-\item[Term.thy]
+\item[Term]
 JavaCard terms. Variables, expressions and statements.
 
-\item[Decl.thy]
+\item[Decl]
 Class, interface and program declarations. Recursion operators for the
 class and the interface hierarchy. 
 
-\item[TypeRel.thy]
+\item[TypeRel]
 Various relations on types like the subclass-, subinterface-, widening-, 
 narrowing- and casting-relation.
 
-\item[DeclConcepts.thy]
+\item[DeclConcepts]
 Advanced concepts on the class and interface hierarchy like inheritance, 
 overriding, hiding, accessibility of types and members according to the access 
 modifiers, method lookup.
 
-\item[WellType.thy]
+\item[WellType]
 Typesystem on the JavaCard term level.
 
-\item[WellForm.thy]
+\item[WellForm]
 Typesystem on the JavaCard class, interface and program level.
 
-\item[State.thy]
+\item[State]
 The program state (like object store) for the execution of JavaCard.
 Abrupt completion (exceptions, break, continue, return) is modelled as flag
 inside the state.
 
-\item[Eval.thy]
+\item[Eval]
 Operational (big step) semantics for JavaCard.
 
-\item[Example.thy]
+\item[Example]
 An concrete example of a JavaCard program to validate the typesystem and the
 operational semantics.
 
-\item[Conform.thy]
+\item[Conform]
 Conformance predicate for states. When does an execution state conform to the
 static types of the program given by the typesystem.
 
-\item[TypeSafe.thy]
+\item[TypeSafe]
 Typesafety proof of the execution of JavaCard. ''Welltyped programs don't go
 wrong'' or more technical: The execution of a welltyped JavaCard program 
 preserves the conformance of execution states.
 
-\item[Evaln.thy]
-Copy of the operational semantics given in Eval.thy expanded with an annotation
+\item[Evaln]
+Copy of the operational semantics given in theory Eval expanded with an annotation
 for the maximal recursive depth. The semantics is not altered. The annotation
 is needed for the soundness proof of the axiomatic semantics.
 
-\item[AxSem.thy]
+\item[AxSem]
 An axiomatic semantics (Hoare logic) for JavaCard.
 
-\item[AxSound.thy]
+\item[AxSound]
 The soundness proof of the axiomatic semantics with respect to the operational
 semantics.
 
-\item[AxCompl.thy]
+\item[AxCompl]
 The proof of (relative) completeness of the axiomatic semantics with respect
 to the operational semantics. 
 
-\item[AxExample.thy]
+\item[AxExample]
 An concrete example of the axiomatic semantics at work, applied to prove 
-some properties of the JavaCard example given in Example.thy.
+some properties of the JavaCard example given in theory Example.
 \end{description}
 
-% include generated text of all theories
-\chapter{Basis.thy}
-\input{../generated/Basis.tex}
-\chapter{Table.thy}
-\input{../generated/Table.tex}    
+
+\chapter{Basis}
+\input{Basis}
+\chapter{Table}
+\input{Table}    
 
-\chapter{Name.thy}
-\input{../generated/Name.tex}
-\chapter{Value.thy}     
-\input{../generated/Value.tex}
-\chapter{Type.thy}
-\input{../generated/Type.tex}      
-\chapter{Term.thy}
-\input{../generated/Term.tex}     
-\chapter{Decl.thy}
-\input{../generated/Decl.tex}          
-\chapter{TypeRel.thy}
-\input{../generated/TypeRel.tex}   
-\chapter{DeclConcepts.thy}
-\input{../generated/DeclConcepts.tex}  
-
-\chapter{WellType.thy}
-\input{../generated/WellType.tex}
-\chapter{WellForm.thy}
-\input{../generated/WellForm.tex}
+\chapter{Name}
+\input{Name}
+\chapter{Value}     
+\input{Value}
+\chapter{Type}
+\input{Type}      
+\chapter{Term}
+\input{Term}     
+\chapter{Decl}
+\input{Decl}          
+\chapter{TypeRel}
+\input{TypeRel}   
+\chapter{DeclConcepts}
+\input{DeclConcepts}  
 
-\chapter{State.thy}
-\input{../generated/State.tex}    
-\chapter{Eval.thy}
-\input{../generated/Eval.tex}          
+\chapter{WellType}
+\input{WellType}
+\chapter{WellForm}
+\input{WellForm}
 
-\chapter{Example.thy}
-\input{../generated/Example.tex}  
+\chapter{State}
+\input{State}    
+\chapter{Eval}
+\input{Eval}          
 
-\chapter{Conform.thy}
-\input{../generated/Conform.tex}       
-\chapter{TypeSafe.thy}
-\input{../generated/TypeSafe.tex}
+\chapter{Example}
+\input{Example}  
 
-\chapter{Evaln.thy}
-\input{../generated/Evaln.tex}         
-\chapter{AxSem.thy}
-\input{../generated/AxSem.tex}      
-\chapter{AxSound.thy}
-\input{../generated/AxSound.tex}    
-\chapter{AxCompl.thy}
-\input{../generated/AxCompl.tex}    
-\chapter{AxExample.thy}
-\input{../generated/AxExample.tex}  
+\chapter{Conform}
+\input{Conform}       
+\chapter{TypeSafe}
+\input{TypeSafe}
 
-
-
-
-
-
+\chapter{Evaln}
+\input{Evaln}         
+\chapter{AxSem}
+\input{AxSem}      
+\chapter{AxSound}
+\input{AxSound}    
+\chapter{AxCompl}
+\input{AxCompl}    
+\chapter{AxExample}
+\input{AxExample}  
 
 %\bibliographystyle{abbrv}
 %\bibliography{root}