src/HOL/Fun.thy
changeset 55414 eab03e9cee8a
parent 55066 4e5ddf3162ac
child 55467 a5c9002bc54d
--- a/src/HOL/Fun.thy	Wed Feb 12 08:35:56 2014 +0100
+++ b/src/HOL/Fun.thy	Wed Feb 12 08:35:57 2014 +0100
@@ -662,10 +662,10 @@
   "_Update f (_updbinds b bs)" == "_Update (_Update f b) bs"
   "f(x:=y)" == "CONST fun_upd f x y"
 
-(* Hint: to define the sum of two functions (or maps), use sum_case.
+(* Hint: to define the sum of two functions (or maps), use case_sum.
          A nice infix syntax could be defined (in Datatype.thy or below) by
 notation
-  sum_case  (infixr "'(+')"80)
+  case_sum  (infixr "'(+')"80)
 *)
 
 lemma fun_upd_idem_iff: "(f(x:=y) = f) = (f x = y)"