author | wenzelm |
Wed, 02 Aug 2000 19:40:14 +0200 | |
changeset 9502 | 50ec59aff389 |
parent 8038 | a13c3b80d3d4 |
child 10042 | 7164dc0d24d8 |
permissions | -rw-r--r-- |
(* Title: HOL/MicroJava/JVM/Store.thy ID: $Id$ Author: Cornelia Pusch Copyright 1999 Technische Universitaet Muenchen The store. The JVM builds on many notions already defined in Java. Conform provides notions for the type safety proof of the Bytecode Verifier. *) Store = Conform + constdefs newref :: "('a \\<leadsto> 'b) \\<Rightarrow> 'a" "newref s \\<equiv> \\<epsilon>v. s v = None" end