src/HOL/Library/Efficient_Nat.thy
changeset 28562 4e74209f113e
parent 28522 eacb54d9e78d
child 28683 59c01ec6cb8d
--- a/src/HOL/Library/Efficient_Nat.thy	Fri Oct 10 06:45:50 2008 +0200
+++ b/src/HOL/Library/Efficient_Nat.thy	Fri Oct 10 06:45:53 2008 +0200
@@ -232,7 +232,6 @@
    of NONE => NONE
     | SOME thms4 => if Thm.eq_thms (map fst eqns2, thms4)
         then NONE else SOME (map (apfst (AxClass.overload thy) o Code_Unit.mk_eqn thy) thms4)
-          (*FIXME*)
   end
 
 in
@@ -344,13 +343,13 @@
 definition
   int :: "nat \<Rightarrow> int"
 where
-  [code func del]: "int = of_nat"
+  [code del]: "int = of_nat"
 
-lemma int_code' [code func]:
+lemma int_code' [code]:
   "int (number_of l) = (if neg (number_of l \<Colon> int) then 0 else number_of l)"
   unfolding int_nat_number_of [folded int_def] ..
 
-lemma nat_code' [code func]:
+lemma nat_code' [code]:
   "nat (number_of l) = (if neg (number_of l \<Colon> int) then 0 else number_of l)"
   by auto
 
@@ -434,7 +433,7 @@
 
 text {* Evaluation *}
 
-lemma [code func, code func del]:
+lemma [code, code del]:
   "(Code_Eval.term_of \<Colon> nat \<Rightarrow> term) = Code_Eval.term_of" ..
 
 code_const "Code_Eval.term_of \<Colon> nat \<Rightarrow> term"