src/HOL/MicroJava/JVM/Store.thy
changeset 8034 6fc37b5c5e98
parent 8011 d14c4e9e9c8e
child 8038 a13c3b80d3d4
equal deleted inserted replaced
8033:325b8e754523 8034:6fc37b5c5e98
    10 *)
    10 *)
    11 
    11 
    12 Store = Conform +  
    12 Store = Conform +  
    13 
    13 
    14 syntax
    14 syntax
    15  value	:: "['a \\<leadsto> 'b,'a] \\<Rightarrow> 'b"			("_ \\<And> _")		
    15  map_apply :: "['a \\<leadsto> 'b,'a] \\<Rightarrow> 'b"	("_ !! _")
    16 translations
    16 translations
    17  "t \\<And> x"  == "the (t x)"
    17  "t !! x"  == "the (t x)"
    18 
    18 
    19 constdefs
    19 constdefs
    20  newref :: "('a \\<leadsto> 'b) \\<Rightarrow> 'a"
    20  newref :: "('a \\<leadsto> 'b) \\<Rightarrow> 'a"
    21  "newref s \\<equiv> \\<epsilon>v. s v = None"
    21  "newref s \\<equiv> \\<epsilon>v. s v = None"
    22 
    22