src/HOL/NSA/HyperNat.thy
changeset 28562 4e74209f113e
parent 27468 0783dd1dc13d
child 29920 b95f5b8b93dd
--- a/src/HOL/NSA/HyperNat.thy	Fri Oct 10 06:45:50 2008 +0200
+++ b/src/HOL/NSA/HyperNat.thy	Fri Oct 10 06:45:53 2008 +0200
@@ -19,7 +19,7 @@
 
 definition
   hSuc :: "hypnat => hypnat" where
-  hSuc_def [transfer_unfold, code func del]: "hSuc = *f* Suc"
+  hSuc_def [transfer_unfold, code del]: "hSuc = *f* Suc"
 
 subsection{*Properties Transferred from Naturals*}
 
@@ -367,7 +367,7 @@
 
 definition
   of_hypnat :: "hypnat \<Rightarrow> 'a::semiring_1_cancel star" where
-  of_hypnat_def [transfer_unfold, code func del]: "of_hypnat = *f* of_nat"
+  of_hypnat_def [transfer_unfold, code del]: "of_hypnat = *f* of_nat"
 
 lemma of_hypnat_0 [simp]: "of_hypnat 0 = 0"
 by transfer (rule of_nat_0)