src/HOL/NanoJava/TypeRel.thy
changeset 61990 39e4a93ad36e
parent 59682 d662d096f72b
child 62390 842917225d56
--- a/src/HOL/NanoJava/TypeRel.thy	Wed Dec 30 19:57:37 2015 +0100
+++ b/src/HOL/NanoJava/TypeRel.thy	Wed Dec 30 20:07:59 2015 +0100
@@ -15,15 +15,11 @@
   "subcls1 \<equiv> {(C,D). C\<noteq>Object \<and> (\<exists>c. class C = Some c \<and> super c=D)}"
 
 abbreviation
-  subcls1_syntax :: "[cname, cname] => bool"  ("_ <=C1 _" [71,71] 70)
-  where "C <=C1 D == (C,D) \<in> subcls1"
+  subcls1_syntax :: "[cname, cname] => bool"  ("_ \<prec>C1 _" [71,71] 70)
+  where "C \<prec>C1 D == (C,D) \<in> subcls1"
 abbreviation
-  subcls_syntax  :: "[cname, cname] => bool" ("_ <=C _"  [71,71] 70)
-  where "C <=C D == (C,D) \<in> subcls1^*"
-
-notation (xsymbols)
-  subcls1_syntax  ("_ \<prec>C1 _"  [71,71] 70) and
-  subcls_syntax  ("_ \<preceq>C _"   [71,71] 70)
+  subcls_syntax  :: "[cname, cname] => bool" ("_ \<preceq>C _"  [71,71] 70)
+  where "C \<preceq>C D == (C,D) \<in> subcls1^*"
 
 
 subsection "Declarations and properties not used in the meta theory"