src/HOL/String.thy
changeset 51717 9e7d1c139569
parent 51160 599ff65b85e2
child 52365 95186e6e4bf4
--- a/src/HOL/String.thy	Tue Apr 16 17:54:14 2013 +0200
+++ b/src/HOL/String.thy	Thu Apr 18 17:07:01 2013 +0200
@@ -252,8 +252,9 @@
 setup {*
 let
   val nibbles = map_range (Thm.cterm_of @{theory} o HOLogic.mk_nibble) 16;
-  val simpset = HOL_ss addsimps
-    @{thms nat_of_nibble.simps mult_0 mult_1 add_0 add_0_right arith_simps numeral_plus_one};
+  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};
   fun mk_code_eqn x y =
     Drule.instantiate' [] [SOME x, SOME y] @{thm nat_of_char_Char}
     |> simplify simpset;