src/HOL/NanoJava/TypeRel.thy
changeset 67443 3abf6a722518
parent 63167 0909deb8059b
child 67613 ce654b0e6d69
--- a/src/HOL/NanoJava/TypeRel.thy	Tue Jan 16 09:12:16 2018 +0100
+++ b/src/HOL/NanoJava/TypeRel.thy	Tue Jan 16 09:30:00 2018 +0100
@@ -103,7 +103,7 @@
 apply (subst cut_apply, auto intro: subcls1I)
 done
 
-\<comment>\<open>Methods of a class, with inheritance and hiding\<close>
+\<comment> \<open>Methods of a class, with inheritance and hiding\<close>
 definition "method" :: "cname => (mname \<rightharpoonup> methd)" where
   "method C \<equiv> class_rec C methods"
 
@@ -115,7 +115,7 @@
 done
 
 
-\<comment>\<open>Fields of a class, with inheritance and hiding\<close>
+\<comment> \<open>Fields of a class, with inheritance and hiding\<close>
 definition field  :: "cname => (fname \<rightharpoonup> ty)" where
   "field C \<equiv> class_rec C flds"