src/HOL/String.thy
changeset 59621 291934bac95e
parent 59484 a130ae7a9398
child 59631 34030d67afb9
--- a/src/HOL/String.thy	Fri Mar 06 14:01:08 2015 +0100
+++ b/src/HOL/String.thy	Fri Mar 06 15:58:56 2015 +0100
@@ -248,7 +248,7 @@
 
 setup {*
 let
-  val nibbles = map_range (Thm.cterm_of @{theory} o HOLogic.mk_nibble) 16;
+  val nibbles = map_range (Thm.global_cterm_of @{theory} o HOLogic.mk_nibble) 16;
   val simpset =
     put_simpset HOL_ss @{context}
       addsimps @{thms nat_of_nibble.simps mult_0 mult_1 add_0 add_0_right arith_simps numeral_plus_one};