src/HOL/Int.thy
changeset 64996 b316cd527a11
parent 64849 766db3539859
child 66035 de6cd60b1226
--- a/src/HOL/Int.thy	Tue Feb 07 22:15:03 2017 +0100
+++ b/src/HOL/Int.thy	Tue Feb 07 22:15:04 2017 +0100
@@ -1721,7 +1721,7 @@
 
 text \<open>Implementations.\<close>
 
-lemma one_int_code [code, code_unfold]: "1 = Pos Num.One"
+lemma one_int_code [code]: "1 = Pos Num.One"
   by simp
 
 lemma plus_int_code [code]: