Invoke instruction gets fully qualified method name (class+name+sig) as
in Sun's JVM spec
(* 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";