diff -r 4dc65845eab3 -r d8d7d1b785af src/HOL/Hoare/Pointer_Examples.thy --- a/src/HOL/Hoare/Pointer_Examples.thy Wed Feb 24 11:55:52 2010 +0100 +++ b/src/HOL/Hoare/Pointer_Examples.thy Mon Mar 01 13:40:23 2010 +0100 @@ -216,10 +216,10 @@ text"This is still a bit rough, especially the proof." -constdefs - cor :: "bool \ bool \ bool" +definition cor :: "bool \ bool \ bool" where "cor P Q == if P then True else Q" - cand :: "bool \ bool \ bool" + +definition cand :: "bool \ bool \ bool" where "cand P Q == if P then Q else False" consts merge :: "'a list * 'a list * ('a \ 'a \ bool) \ 'a list" @@ -481,7 +481,7 @@ subsection "Storage allocation" -constdefs new :: "'a set \ 'a" +definition new :: "'a set \ 'a" where "new A == SOME a. a \ A"