src/HOL/ex/Primrec.thy
changeset 21404 eb85850d3eb7
parent 19736 d8d0f8f51d69
child 22283 26140713540b
--- a/src/HOL/ex/Primrec.thy	Fri Nov 17 02:19:55 2006 +0100
+++ b/src/HOL/ex/Primrec.thy	Fri Nov 17 02:20:03 2006 +0100
@@ -43,19 +43,23 @@
 text {* The set of primitive recursive functions of type @{typ "nat list => nat"}. *}
 
 definition
-  SC :: "nat list => nat"
+  SC :: "nat list => nat" where
   "SC l = Suc (zeroHd l)"
 
-  CONSTANT :: "nat => nat list => nat"
+definition
+  CONSTANT :: "nat => nat list => nat" where
   "CONSTANT k l = k"
 
-  PROJ :: "nat => nat list => nat"
+definition
+  PROJ :: "nat => nat list => nat" where
   "PROJ i l = zeroHd (drop i l)"
 
-  COMP :: "(nat list => nat) => (nat list => nat) list => nat list => nat"
+definition
+  COMP :: "(nat list => nat) => (nat list => nat) list => nat list => nat" where
   "COMP g fs l = g (map (\<lambda>f. f l) fs)"
 
-  PREC :: "(nat list => nat) => (nat list => nat) => nat list => nat"
+definition
+  PREC :: "(nat list => nat) => (nat list => nat) => nat list => nat" where
   "PREC f g l =
     (case l of
       [] => 0