diff -r c8a2755bf220 -r ff784d5a5bfb src/HOL/Hoare/Heap.thy --- a/src/HOL/Hoare/Heap.thy Sat Jan 05 17:00:43 2019 +0100 +++ b/src/HOL/Hoare/Heap.thy Sat Jan 05 17:24:33 2019 +0100 @@ -60,11 +60,11 @@ definition distPath :: "('a \ 'a ref) \ 'a ref \ 'a list \ 'a ref \ bool" where "distPath h x as y \ Path h x as y \ distinct as" -text\The term @{term"distPath h x as y"} expresses the fact that a -non-repeating path @{term as} connects location @{term x} to location -@{term y} by means of the @{term h} field. In the case where \x -= y\, and there is a cycle from @{term x} to itself, @{term as} can -be both @{term "[]"} and the non-repeating list of nodes in the +text\The term \<^term>\distPath h x as y\ expresses the fact that a +non-repeating path \<^term>\as\ connects location \<^term>\x\ to location +\<^term>\y\ by means of the \<^term>\h\ field. In the case where \x += y\, and there is a cycle from \<^term>\x\ to itself, \<^term>\as\ can +be both \<^term>\[]\ and the non-repeating list of nodes in the cycle.\ lemma neq_dP: "p \ q \ Path h p Ps q \ distinct Ps \