diff -r 1a0c129bb2e0 -r b1fd1d756e20 src/HOL/Statespace/StateFun.thy --- a/src/HOL/Statespace/StateFun.thy Thu Feb 11 22:19:58 2010 +0100 +++ b/src/HOL/Statespace/StateFun.thy Thu Feb 11 22:55:16 2010 +0100 @@ -1,5 +1,4 @@ (* Title: StateFun.thy - ID: $Id$ Author: Norbert Schirmer, TU Muenchen *) @@ -34,12 +33,12 @@ lemma K_statefun_cong [cong]: "K_statefun c x = K_statefun c x" by (rule refl) -constdefs lookup:: "('v \ 'a) \ 'n \ ('n \ 'v) \ 'a" -"lookup destr n s \ destr (s n)" +definition lookup:: "('v \ 'a) \ 'n \ ('n \ 'v) \ 'a" + where "lookup destr n s = destr (s n)" -constdefs update:: +definition update:: "('v \ 'a1) \ ('a2 \ 'v) \ 'n \ ('a1 \ 'a2) \ ('n \ 'v) \ ('n \ 'v)" -"update destr constr n f s \ s(n := constr (f (destr (s n))))" + where "update destr constr n f s = s(n := constr (f (destr (s n))))" lemma lookup_update_same: "(\v. destr (constr v) = v) \ lookup destr n (update destr constr n f s) =