diff -r 6539627881e8 -r 65d98faa2182 src/HOL/NanoJava/AxSem.thy --- a/src/HOL/NanoJava/AxSem.thy Mon Sep 10 17:35:22 2001 +0200 +++ b/src/HOL/NanoJava/AxSem.thy Mon Sep 10 18:18:04 2001 +0200 @@ -86,8 +86,8 @@ Impl (D,m) {Q} ==> A |- {P} Meth (C,m) {Q}" - --{*\z instead of \z in the conclusion and - z restricted to type state due to limitations of the inductive package *} + --{* @{text "\z"} instead of @{text "\z"} in the conclusion and + z restricted to type state due to limitations of the inductive package *} Impl: "\z::state. A\ (\z. (\Cm. (P z Cm, Impl Cm, Q z Cm))`Ms) ||- (\Cm. (P z Cm, body Cm, Q z Cm))`Ms ==> A ||- (\Cm. (P z Cm, Impl Cm, Q z Cm))`Ms"