src/HOL/List.thy
changeset 28965 1de908189869
parent 28823 dcbef866c9e2
child 29223 e09c53289830
--- a/src/HOL/List.thy	Wed Dec 03 21:00:39 2008 -0800
+++ b/src/HOL/List.thy	Thu Dec 04 14:43:33 2008 +0100
@@ -3423,7 +3423,7 @@
    (fn n => fn m => Drule.instantiate' [] [SOME n, SOME m] @{thm nibble_pair_of_char.simps})
       nibbles nibbles;
 in
-  PureThy.note_thmss Thm.lemmaK [((Name.binding "nibble_pair_of_char_simps", []), [(thms, [])])]
+  PureThy.note_thmss Thm.lemmaK [((Binding.name "nibble_pair_of_char_simps", []), [(thms, [])])]
   #-> (fn [(_, thms)] => fold_rev Code.add_eqn thms)
 end
 *}