src/HOL/Update.thy
author wenzelm
Mon, 22 Jun 1998 17:26:46 +0200
changeset 5069 3ea049f7979d
parent 4898 68fd1a2b8b7b
child 5070 c42429b3e2f2
permissions -rw-r--r--
isatool fixgoal;

(*  Title:      HOL/Update.thy
    ID:         $Id$
    Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
    Copyright   1998  University of Cambridge

Function updates: like theory Map, but for ordinary functions
*)

Update = Fun +

consts
  update  :: "('a => 'b) => 'a => 'b => ('a => 'b)"
           ("_/[_/:=/_]" [900,0,0] 900)

defs
  update_def "f[a:=b] == %x. if x=a then b else f x"

end