src/ZF/Induct/Primrec.thy
changeset 26056 6a0801279f4c
parent 24893 b8ef7afe3a6b
child 26059 b67a225b50fd
--- a/src/ZF/Induct/Primrec.thy	Mon Feb 11 15:19:17 2008 +0100
+++ b/src/ZF/Induct/Primrec.thy	Mon Feb 11 15:40:21 2008 +0100
@@ -31,7 +31,7 @@
 
 definition
   COMP :: "[i,i]=>i"  where
-  "COMP(g,fs) == \<lambda>l \<in> list(nat). g ` List.map(\<lambda>f. f`l, fs)"
+  "COMP(g,fs) == \<lambda>l \<in> list(nat). g ` List_ZF.map(\<lambda>f. f`l, fs)"
 
 definition
   PREC :: "[i,i]=>i"  where
@@ -93,7 +93,7 @@
   monos list_mono
   con_defs SC_def CONSTANT_def PROJ_def COMP_def PREC_def
   type_intros nat_typechecks list.intros
-    lam_type list_case_type drop_type List.map_type
+    lam_type list_case_type drop_type List_ZF.map_type
     apply_type rec_type