diff -r f075640b8868 -r 3abf6a722518 src/HOL/NanoJava/Decl.thy --- a/src/HOL/NanoJava/Decl.thy Tue Jan 16 09:12:16 2018 +0100 +++ b/src/HOL/NanoJava/Decl.thy Tue Jan 16 09:30:00 2018 +0100 @@ -8,8 +8,8 @@ theory Decl imports Term begin datatype ty - = NT \\null type\ - | Class cname \\class type\ + = NT \ \null type\ + | Class cname \ \class type\ text\Field declaration\ type_synonym fdecl @@ -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