diff -r 67110d6c66de -r 66c68453455c src/HOL/NanoJava/AxSem.thy --- a/src/HOL/NanoJava/AxSem.thy Tue Dec 13 14:04:20 2011 +0100 +++ b/src/HOL/NanoJava/AxSem.thy Tue Dec 13 15:18:52 2011 +0100 @@ -99,17 +99,18 @@ subsection "Fully polymorphic variants, required for Example only" -axioms - +axiomatization where Conseq:"[| \Z. A \ {P' Z} c {Q' Z}; \s t. (\Z. P' Z s --> Q' Z t) --> (P s --> Q t) |] ==> A \ {P} c {Q }" - eConseq:"[| \Z. A \\<^sub>e {P' Z} e {Q' Z}; +axiomatization where + eConseq:"[| \Z. 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 }" - Impl: "\Z. A\ (\Z. (\Cm. (P Z Cm, Impl Cm, Q Z Cm))`Ms) |\ +axiomatization where + Impl: "\Z. 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"