src/HOL/ex/Primrec.thy
changeset 55415 05f5fdb8d093
parent 46546 42298c5d33b1
child 58889 5b7a9633cfa8
--- a/src/HOL/ex/Primrec.thy	Wed Feb 12 08:35:57 2014 +0100
+++ b/src/HOL/ex/Primrec.thy	Wed Feb 12 08:35:57 2014 +0100
@@ -191,7 +191,7 @@
   "PREC f g l =
     (case l of
       [] => 0
-    | x # l' => nat_rec (f l') (\<lambda>y r. g (r # y # l')) x)"
+    | x # l' => rec_nat (f l') (\<lambda>y r. g (r # y # l')) x)"
   -- {* Note that @{term g} is applied first to @{term "PREC f g y"} and then to @{term y}! *}
 
 inductive PRIMREC :: "(nat list => nat) => bool" where