src/HOL/Import/HOL_Light_Maps.thy
changeset 55524 f41ef840f09d
parent 55466 786edc984c98
child 56266 da5f22a60cb3
--- a/src/HOL/Import/HOL_Light_Maps.thy	Sun Feb 16 21:33:28 2014 +0100
+++ b/src/HOL/Import/HOL_Light_Maps.thy	Sun Feb 16 21:33:28 2014 +0100
@@ -290,7 +290,7 @@
   foldr f (h # t) b = f h (foldr f t b)"
   by simp
 
-lemma ALL2_DEF[import_const ALL2 : List.list_all2]:
+lemma ALL2_DEF[import_const ALL2 : List.list.list_all2]:
   "list_all2 (P\<Colon>'t18495 \<Rightarrow> 't18502 \<Rightarrow> bool) [] (l2\<Colon>'t18502 list) = (l2 = []) \<and>
   list_all2 P ((h1\<Colon>'t18495) # (t1\<Colon>'t18495 list)) l2 =
   (if l2 = [] then False else P h1 (hd l2) \<and> list_all2 P t1 (tl l2))"