diff -r f075640b8868 -r 3abf6a722518 src/HOL/NanoJava/AxSem.thy --- a/src/HOL/NanoJava/AxSem.thy Tue Jan 16 09:12:16 2018 +0100 +++ b/src/HOL/NanoJava/AxSem.thy Tue Jan 16 09:30:00 2018 +0100 @@ -72,13 +72,13 @@ Impl (D,m) {Q} ==> A \ {P} Meth (C,m) {Q}" - \\\\Z\ instead of \\Z\ in the conclusion and\\ + \ \\\Z\ instead of \\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" -\\structural rules\ +\ \structural rules\ | Asm: " a \ A ==> A |\ {a}" @@ -86,12 +86,12 @@ | ConjE: "[|A |\ C; c \ C |] ==> A |\ {c}" - \\Z restricted to type state due to limitations of the inductive package\ + \ \Z restricted to type state due to limitations of the inductive package\ | Conseq:"[| \Z::state. A \ {P' Z} c {Q' Z}; \s t. (\Z. P' Z s --> Q' Z t) --> (P s --> Q t) |] ==> A \ {P} c {Q }" - \\Z restricted to type state due to limitations of the inductive package\ + \ \Z restricted to type state due to limitations of the inductive package\ | eConseq:"[| \Z::state. A \\<^sub>e {P' Z} e {Q' Z}; \s v t. (\Z. P' Z s --> Q' Z v t) --> (P s --> Q v t) |] ==> A \\<^sub>e {P} e {Q }"