src/HOL/NanoJava/TypeRel.thy
changeset 63167 0909deb8059b
parent 62390 842917225d56
child 67443 3abf6a722518
--- a/src/HOL/NanoJava/TypeRel.thy	Thu May 26 16:57:14 2016 +0200
+++ b/src/HOL/NanoJava/TypeRel.thy	Thu May 26 17:51:22 2016 +0200
@@ -8,7 +8,7 @@
 imports Decl
 begin
 
-text{* Direct subclass relation *}
+text\<open>Direct subclass relation\<close>
 
 definition subcls1 :: "(cname \<times> cname) set"
 where
@@ -24,7 +24,7 @@
 
 subsection "Declarations and properties not used in the meta theory"
 
-text{* Widening, viz. method invocation conversion *}
+text\<open>Widening, viz. method invocation conversion\<close>
 inductive
   widen :: "ty => ty => bool"  ("_ \<preceq> _" [71,71] 70)
 where
@@ -103,7 +103,7 @@
 apply (subst cut_apply, auto intro: subcls1I)
 done
 
---{* Methods of a class, with inheritance and hiding *}
+\<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
 
 
---{* Fields of a class, with inheritance and hiding *}
+\<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"