src/HOL/Bali/Decl.thy
changeset 55518 1ddb2edf5ceb
parent 54703 499f92dc6e45
child 58249 180f1b3508ed
--- a/src/HOL/Bali/Decl.thy	Sun Feb 16 17:50:13 2014 +0100
+++ b/src/HOL/Bali/Decl.thy	Sun Feb 16 18:39:40 2014 +0100
@@ -818,7 +818,7 @@
   --{* methods of an interface, with overriding and inheritance, cf. 9.2 *}
   "imethds G I = iface_rec G I
               (\<lambda>I i ts. (Un_tables ts) \<oplus>\<oplus> 
-                        (Option.set \<circ> table_of (map (\<lambda>(s,m). (s,I,m)) (imethods i))))"
+                        (set_option \<circ> table_of (map (\<lambda>(s,m). (s,I,m)) (imethods i))))"