src/HOL/MicroJava/J/Eval.thy
changeset 11070 cc421547e744
parent 11040 194406da4e43
child 11372 648795477bb5
--- a/src/HOL/MicroJava/J/Eval.thy	Mon Feb 05 14:59:44 2001 +0100
+++ b/src/HOL/MicroJava/J/Eval.thy	Mon Feb 05 20:14:15 2001 +0100
@@ -2,10 +2,9 @@
     ID:         $Id$
     Author:     David von Oheimb
     Copyright   1999 Technische Universitaet Muenchen
+*)
 
-Operational evaluation (big-step) semantics of the 
-execution of Java expressions and statements
-*)
+header "Operational Evaluation (big-step) Semantics"
 
 theory Eval = State + WellType: