diff -r 66b62cbeaab3 -r 6539627881e8 src/HOL/NanoJava/TypeRel.thy --- a/src/HOL/NanoJava/TypeRel.thy Mon Sep 10 13:57:57 2001 +0200 +++ b/src/HOL/NanoJava/TypeRel.thy Mon Sep 10 17:35:22 2001 +0200 @@ -9,8 +9,8 @@ theory TypeRel = Decl: consts - widen :: "(ty \ ty ) set" (* widening *) - subcls1 :: "(cname \ cname) set" (* subclass *) + widen :: "(ty \ ty ) set" --{* widening *} + subcls1 :: "(cname \ cname) set" --{* subclass *} syntax (xsymbols) widen :: "[ty , ty ] => bool" ("_ \ _" [71,71] 70) @@ -28,17 +28,17 @@ consts method :: "cname => (mname \ methd)" - field :: "cname => (vnam \ ty)" + field :: "cname => (fname \ ty)" text {* The rest of this theory is not actually used. *} +text{* direct subclass relation *} defs - (* direct subclass relation *) subcls1_def: "subcls1 \ {(C,D). C\Object \ (\c. class C = Some c \ super c=D)}" - -inductive widen intros (*widening, viz. method invocation conversion, - i.e. sort of syntactic subtyping *) + +text{* widening, viz. method invocation conversion *} +inductive widen intros refl [intro!, simp]: "T \ T" subcls : "C\C D \ Class C \ Class D" null [intro!]: "NT \ R" @@ -121,7 +121,7 @@ apply simp done -(* methods of a class, with inheritance and hiding *) +--{* methods of a class, with inheritance and hiding *} defs method_def: "method C \ class_rec C methods" lemma method_rec: "\class C = Some m; ws_prog\ \ @@ -132,7 +132,7 @@ done -(* fields of a class, with inheritance and hiding *) +--{* fields of a class, with inheritance and hiding *} defs field_def: "field C \ class_rec C fields" lemma fields_rec: "\class C = Some m; ws_prog\ \