diff -r f7157bdc1e70 -r 8f32860eac3a src/HOL/NanoJava/AxSem.thy --- a/src/HOL/NanoJava/AxSem.thy Wed Aug 08 15:16:38 2001 +0200 +++ b/src/HOL/NanoJava/AxSem.thy Wed Aug 08 16:57:43 2001 +0200 @@ -9,7 +9,7 @@ theory AxSem = State: types assn = "state => bool" - vassn = "val \ assn" + vassn = "val => assn" triple = "assn \ stmt \ assn" etriple = "assn \ expr \ vassn" translations @@ -24,9 +24,9 @@ "@hoare" :: "[triple set, triple set ] => bool" ("_ |\/ _" [61,61] 60) "@hoare1" :: "[triple set, assn,stmt,assn] => bool" ("_ \/ ({(1_)}/ (_)/ {(1_)})" [61,3,90,3]60) -"@ehoare" :: "[triple set, etriple ] => bool" ("_ |\e/ _"[61,61]60) +"@ehoare" :: "[triple set, etriple ] => bool" ("_ |\\<^sub>e/ _"[61,61]60) "@ehoare1" :: "[triple set, assn,expr,vassn]=> bool" - ("_ \e/ ({(1_)}/ (_)/ {(1_)})" [61,3,90,3]60) + ("_ \\<^sub>e/ ({(1_)}/ (_)/ {(1_)})" [61,3,90,3]60) syntax "@hoare" :: "[triple set, triple set ] => bool" ("_ ||-/ _" [61,61] 60) "@hoare1" :: "[triple set, assn,stmt,assn] => bool" @@ -37,9 +37,9 @@ translations "A |\ C" \ "(A,C) \ hoare" "A \ {P}c{Q}" \ "A |\ {(P,c,Q)}" - "A |\e t" \ "(A,t) \ ehoare" - "A |\e (P,e,Q)" \ "(A,P,e,Q) \ ehoare" (** shouldn't be necess.**) - "A \e{P}e{Q}" \ "A |\e (P,e,Q)" + "A |\\<^sub>e t" \ "(A,t) \ ehoare" + "A |\\<^sub>e (P,e,Q)" \ "(A,P,e,Q) \ ehoare" (** shouldn't be necess.**) + "A \\<^sub>e {P}e{Q}" \ "A |\\<^sub>e (P,e,Q)" inductive hoare ehoare @@ -124,13 +124,13 @@ apply fast done -lemma eConseq1: "\A \e {P'} e {Q}; \s. P s \ P' s\ \ A \e {P} e {Q}" +lemma eConseq1: "\A \\<^sub>e {P'} e {Q}; \s. P s \ P' s\ \ A \\<^sub>e {P} e {Q}" apply (rule hoare_ehoare.eConseq) apply (rule allI, assumption) apply fast done -lemma eConseq2: "\A \e {P} e {Q'}; \v t. Q' v t \ Q v t\ \ A \e {P} e {Q}" +lemma eConseq2: "\A \\<^sub>e {P} e {Q'}; \v t. Q' v t \ Q v t\ \ A \\<^sub>e {P} e {Q}" apply (rule hoare_ehoare.eConseq) apply (rule allI, assumption) apply fast