src/HOL/MicroJava/JVM/Store.ML
author kleing
Thu, 09 Mar 2000 13:50:58 +0100
changeset 8386 3e56677d3b98
parent 8011 d14c4e9e9c8e
child 9969 4753185f1dd2
permissions -rw-r--r--
minor adjustments in branch and method invocation for completeness of LBV

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

Goalw [newref_def]
 "hp x = None \\<longrightarrow> hp (newref hp) = None";
by (fast_tac (claset() addIs [selectI2EX] addss (simpset())) 1);
qed_spec_mp "newref_None";