diff -r 143f58bb34f9 -r 0909deb8059b src/HOL/NanoJava/Decl.thy --- a/src/HOL/NanoJava/Decl.thy Thu May 26 16:57:14 2016 +0200 +++ b/src/HOL/NanoJava/Decl.thy Thu May 26 17:51:22 2016 +0200 @@ -8,10 +8,10 @@ theory Decl imports Term begin datatype ty - = NT --{* null type *} - | Class cname --{* class type *} + = NT \\null type\ + | Class cname \\class type\ -text{* Field declaration *} +text\Field declaration\ type_synonym fdecl = "fname \ ty" @@ -21,7 +21,7 @@ lcl ::"(vname \ ty) list" bdy :: stmt -text{* Method declaration *} +text\Method declaration\ type_synonym mdecl = "mname \ methd" @@ -30,7 +30,7 @@ flds ::"fdecl list" methods ::"mdecl list" -text{* Class declaration *} +text\Class declaration\ type_synonym cdecl = "cname \ class" @@ -45,9 +45,9 @@ (type) "prog " \ (type) "cdecl list" axiomatization - Prog :: prog --{* program as a global value *} + Prog :: prog \\program as a global value\ and - Object :: cname --{* name of root class *} + Object :: cname \\name of root class\ definition "class" :: "cname \ class" where