diff -r 457240e42972 -r e6e412406a2d thys/Hoare_gen.thy --- a/thys/Hoare_gen.thy Thu Mar 27 13:06:27 2014 +0000 +++ b/thys/Hoare_gen.thy Thu Mar 27 15:12:33 2014 +0000 @@ -203,6 +203,8 @@ shows "((EXS x. P(x)) \* r) s" by (metis assms pred_ex_def sep_globalise) + +(* Interpreted Hoare triples *) definition IHoare :: "('b::sep_algebra \ 'a \ bool) \ ('b \ bool) \ ('a \ bool) \ ('b \ bool) \ bool" ("(1_).(\(1_)\/ (_)/ \(1_)\)" 50)