src/HOL/Induct/SList.thy
changeset 39246 9e58f0499f57
parent 35247 0831bd85eee5
child 45605 a89b4bc311a5
--- a/src/HOL/Induct/SList.thy	Wed Sep 08 13:25:22 2010 +0200
+++ b/src/HOL/Induct/SList.thy	Wed Sep 08 19:21:46 2010 +0200
@@ -133,10 +133,9 @@
   map       :: "('a=>'b) => ('a list => 'b list)" where
   "map f xs = list_rec xs [] (%x l r. f(x)#r)"
 
-consts take      :: "['a list,nat] => 'a list"
-primrec
+primrec take :: "['a list,nat] => 'a list" where
   take_0:  "take xs 0 = []"
-  take_Suc: "take xs (Suc n) = list_case [] (%x l. x # take l n) xs"
+| take_Suc: "take xs (Suc n) = list_case [] (%x l. x # take l n) xs"
 
 lemma ListI: "x : list (range Leaf) ==> x : List"
 by (simp add: List_def)