src/HOL/MicroJava/J/Conform.thy
changeset 14134 0fdf5708c7a8
parent 13672 b95d12325b51
child 14174 f3cafd2929d5
--- a/src/HOL/MicroJava/J/Conform.thy	Fri Jul 25 10:52:15 2003 +0200
+++ b/src/HOL/MicroJava/J/Conform.thy	Fri Jul 25 17:21:22 2003 +0200
@@ -8,7 +8,7 @@
 
 theory Conform = State + WellType + Exceptions:
 
-types 'c env_ = "'c prog \<times> (vname \<leadsto> ty)"  -- "same as @{text env} of @{text WellType.thy}"
+types 'c env_ = "'c prog \<times> (vname \<rightharpoonup> ty)"  -- "same as @{text env} of @{text WellType.thy}"
 
 constdefs
 
@@ -19,7 +19,7 @@
                                    ("_,_ |- _ ::<= _"  [51,51,51,51] 50)
  "G,h|-v::<=T == \<exists>T'. typeof (option_map obj_ty o h) v = Some T' \<and> G\<turnstile>T'\<preceq>T"
 
-  lconf :: "'c prog => aheap => ('a \<leadsto> val) => ('a \<leadsto> ty) => bool"
+  lconf :: "'c prog => aheap => ('a \<rightharpoonup> val) => ('a \<rightharpoonup> ty) => bool"
                                    ("_,_ |- _ [::<=] _" [51,51,51,51] 50)
  "G,h|-vs[::<=]Ts == \<forall>n T. Ts n = Some T --> (\<exists>v. vs n = Some v \<and> G,h|-v::<=T)"
 
@@ -45,7 +45,7 @@
   conf     :: "'c prog => aheap => val => ty => bool"
               ("_,_ \<turnstile> _ ::\<preceq> _" [51,51,51,51] 50)
 
-  lconf    :: "'c prog => aheap => ('a \<leadsto> val) => ('a \<leadsto> ty) => bool"
+  lconf    :: "'c prog => aheap => ('a \<rightharpoonup> val) => ('a \<rightharpoonup> ty) => bool"
               ("_,_ \<turnstile> _ [::\<preceq>] _" [51,51,51,51] 50)
 
   oconf    :: "'c prog => aheap => obj => bool"