Removed some traces of UNITY
authorpaulson
Wed, 06 May 1998 13:01:30 +0200
changeset 4898 68fd1a2b8b7b
parent 4897 be11be0b6ea1
child 4899 447d6b2956ba
Removed some traces of UNITY
src/HOL/Update.ML
src/HOL/Update.thy
--- a/src/HOL/Update.ML	Wed May 06 11:46:00 1998 +0200
+++ b/src/HOL/Update.ML	Wed May 06 13:01:30 1998 +0200
@@ -1,9 +1,9 @@
-(*  Title:      HOL/UNITY/Update.thy
+(*  Title:      HOL/Update.thy
     ID:         $Id$
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1998  University of Cambridge
 
-Function updates: like the standard theory Map, but for ordinary functions
+Function updates: like theory Map, but for ordinary functions
 *)
 
 open Update;
--- a/src/HOL/Update.thy	Wed May 06 11:46:00 1998 +0200
+++ b/src/HOL/Update.thy	Wed May 06 13:01:30 1998 +0200
@@ -1,9 +1,9 @@
-(*  Title:      HOL/UNITY/Update.thy
+(*  Title:      HOL/Update.thy
     ID:         $Id$
     Author:     Lawrence C Paulson, Cambridge University Computer Laboratory
     Copyright   1998  University of Cambridge
 
-Function updates: like the standard theory Map, but for ordinary functions
+Function updates: like theory Map, but for ordinary functions
 *)
 
 Update = Fun +
@@ -12,10 +12,6 @@
   update  :: "('a => 'b) => 'a => 'b => ('a => 'b)"
            ("_/[_/:=/_]" [900,0,0] 900)
 
-syntax (symbols)
-  update    :: "('a => 'b) => 'a => 'b => ('a => 'b)"
-               ("_/[_/\\<mapsto>/_]" [900,0,0] 900)
-
 defs
   update_def "f[a:=b] == %x. if x=a then b else f x"