src/HOL/Bali/Eval.thy
changeset 16417 9bc16273c2d4
parent 14981 e73f8140af78
child 17589 58eeffd73be1
equal deleted inserted replaced
16416:6061ae1f90f2 16417:9bc16273c2d4
     4 *)
     4 *)
     5 header {* Operational evaluation (big-step) semantics of Java expressions and 
     5 header {* Operational evaluation (big-step) semantics of Java expressions and 
     6           statements
     6           statements
     7 *}
     7 *}
     8 
     8 
     9 theory Eval = State + DeclConcepts:
     9 theory Eval imports State DeclConcepts begin
    10 
    10 
    11 text {*
    11 text {*
    12 
    12 
    13 improvements over Java Specification 1.0:
    13 improvements over Java Specification 1.0:
    14 \begin{itemize}
    14 \begin{itemize}