src/HOL/NanoJava/TypeRel.thy
changeset 14134 0fdf5708c7a8
parent 13867 1fdecd15437f
child 14171 0cab06e3bbd0
--- a/src/HOL/NanoJava/TypeRel.thy	Fri Jul 25 10:52:15 2003 +0200
+++ b/src/HOL/NanoJava/TypeRel.thy	Fri Jul 25 17:21:22 2003 +0200
@@ -27,8 +27,8 @@
   "S \<preceq>   T" == "(S,T) \<in> widen"
 
 consts
-  method :: "cname => (mname \<leadsto> methd)"
-  field  :: "cname => (fname \<leadsto> ty)"
+  method :: "cname => (mname \<rightharpoonup> methd)"
+  field  :: "cname => (fname \<rightharpoonup> ty)"
 
 
 subsection "Declarations and properties not used in the meta theory"
@@ -102,7 +102,7 @@
 by (auto intro: finite_acyclic_wf_converse finite_subcls1 subcls1_acyclic)
 
 
-consts class_rec ::"cname \<Rightarrow> (class \<Rightarrow> ('a \<times> 'b) list) \<Rightarrow> ('a \<leadsto> 'b)"
+consts class_rec ::"cname \<Rightarrow> (class \<Rightarrow> ('a \<times> 'b) list) \<Rightarrow> ('a \<rightharpoonup> 'b)"
 
 recdef (permissive) class_rec "subcls1\<inverse>"
       "class_rec C = (\<lambda>f. case class C of None   \<Rightarrow> arbitrary