src/HOL/MicroJava/JVM/Store.thy
author oheimb
Tue, 17 Oct 2000 08:41:42 +0200
changeset 10229 10e2d29a77de
parent 10057 8c8d2d0d3ef8
permissions -rw-r--r--
cosmetics

(*  Title:      HOL/MicroJava/JVM/Store.thy
    ID:         $Id$
    Author:     Cornelia Pusch
    Copyright   1999 Technische Universitaet Muenchen
*)

header {* Store of the JVM *}

theory Store = Conform:

text {*
The JVM builds on many notions already defined in Java.
Conform provides notions for the type safety proof of the Bytecode Verifier.
*}


constdefs
 newref :: "('a \<leadsto> 'b) => 'a"
 "newref s == SOME v. s v = None"


lemma newref_None:
  "hp x = None ==> hp (newref hp) = None"
by (auto intro: someI2_ex simp add: newref_def)

end