diff -r 46f59511b7bb -r d97fdabd9e2b src/HOL/NanoJava/TypeRel.thy --- a/src/HOL/NanoJava/TypeRel.thy Fri Sep 20 19:07:10 2024 +0200 +++ b/src/HOL/NanoJava/TypeRel.thy Fri Sep 20 19:51:08 2024 +0200 @@ -15,10 +15,10 @@ "subcls1 \ {(C,D). C\Object \ (\c. class C = Some c \ super c=D)}" abbreviation - subcls1_syntax :: "[cname, cname] => bool" ("_ \C1 _" [71,71] 70) + subcls1_syntax :: "[cname, cname] => bool" (\_ \C1 _\ [71,71] 70) where "C \C1 D == (C,D) \ subcls1" abbreviation - subcls_syntax :: "[cname, cname] => bool" ("_ \C _" [71,71] 70) + subcls_syntax :: "[cname, cname] => bool" (\_ \C _\ [71,71] 70) where "C \C D \ (C,D) \ subcls1\<^sup>*" @@ -26,7 +26,7 @@ text\Widening, viz. method invocation conversion\ inductive - widen :: "ty => ty => bool" ("_ \ _" [71,71] 70) + widen :: "ty => ty => bool" (\_ \ _\ [71,71] 70) where refl [intro!, simp]: "T \ T" | subcls: "C\C D \ Class C \ Class D"