src/HOL/HOLCF/IOA/RefCorrectness.thy
changeset 67613 ce654b0e6d69
parent 63680 6e1e8b5abbfa
--- a/src/HOL/HOLCF/IOA/RefCorrectness.thy	Tue Feb 13 14:24:50 2018 +0100
+++ b/src/HOL/HOLCF/IOA/RefCorrectness.thy	Thu Feb 15 12:11:00 2018 +0100
@@ -147,7 +147,7 @@
 
 lemma move_subprop3:
   "is_ref_map f C A \<Longrightarrow> reachable C s \<Longrightarrow> (s, a, t) \<in> trans_of C \<Longrightarrow>
-     laststate (f s,@x. move A x (f s) a (f t)) = (f t)"
+     laststate (f s, SOME x. move A x (f s) a (f t)) = (f t)"
   apply (cut_tac move_is_move)
   defer
   apply assumption+