src/HOL/ex/Abstract_NAT.thy
changeset 23775 8b37b6615c52
parent 23253 b1f3f53c60b5
child 29234 60f7fb56f8cd
--- a/src/HOL/ex/Abstract_NAT.thy	Wed Jul 11 11:52:00 2007 +0200
+++ b/src/HOL/ex/Abstract_NAT.thy	Wed Jul 11 11:52:28 2007 +0200
@@ -26,7 +26,7 @@
 
 text {* \medskip Primitive recursion as a (functional) relation -- polymorphic! *}
 
-inductive2
+inductive
   Rec :: "'a \<Rightarrow> ('n \<Rightarrow> 'a \<Rightarrow> 'a) \<Rightarrow> 'n \<Rightarrow> 'a \<Rightarrow> bool"
   for e :: 'a and r :: "'n \<Rightarrow> 'a \<Rightarrow> 'a"
 where