src/HOL/MicroJava/J/SystemClasses.thy
changeset 61361 8b5f00202e1a
parent 58886 8a6cac7c7247
child 62042 6c6ccf573479
--- a/src/HOL/MicroJava/J/SystemClasses.thy	Wed Oct 07 19:45:00 2015 +0200
+++ b/src/HOL/MicroJava/J/SystemClasses.thy	Wed Oct 07 23:28:49 2015 +0200
@@ -3,14 +3,14 @@
     Copyright   2002 Technische Universitaet Muenchen
 *)
 
-section {* System Classes *}
+section \<open>System Classes\<close>
 
 theory SystemClasses imports Decl begin
 
-text {*
+text \<open>
   This theory provides definitions for the @{text Object} class,
   and the system exceptions.
-*}
+\<close>
 
 definition ObjectC :: "'c cdecl" where
   [code_unfold]: "ObjectC \<equiv> (Object, (undefined,[],[]))"