src/HOL/Hoare/HeapSyntaxAbort.thy
changeset 69597 ff784d5a5bfb
parent 62042 6c6ccf573479
child 72990 db8f94656024
--- a/src/HOL/Hoare/HeapSyntaxAbort.thy	Sat Jan 05 17:00:43 2019 +0100
+++ b/src/HOL/Hoare/HeapSyntaxAbort.thy	Sat Jan 05 17:24:33 2019 +0100
@@ -7,8 +7,8 @@
 
 subsection "Field access and update"
 
-text\<open>Heap update \<open>p^.h := e\<close> is now guarded against @{term p}
-being Null. However, @{term p} may still be illegal,
+text\<open>Heap update \<open>p^.h := e\<close> is now guarded against \<^term>\<open>p\<close>
+being Null. However, \<^term>\<open>p\<close> may still be illegal,
 e.g. uninitialized or dangling. To guard against that, one needs a
 more detailed model of the heap where allocated and free addresses are
 distinguished, e.g. by making the heap a map, or by carrying the set