src/HOL/Import/HOL_Light_Maps.thy
changeset 82691 b69e4da2604b
parent 81935 dea6f877c225
equal deleted inserted replaced
82690:cccbfa567117 82691:b69e4da2604b
   284    replicate (Suc n) x = x # replicate n x"
   284    replicate (Suc n) x = x # replicate n x"
   285   by simp
   285   by simp
   286 
   286 
   287 lemma NULL[import_const NULL : List.null]:
   287 lemma NULL[import_const NULL : List.null]:
   288   "List.null ([]::'t18373 list) = True \<and> List.null ((h::'t18373) # t) = False"
   288   "List.null ([]::'t18373 list) = True \<and> List.null ((h::'t18373) # t) = False"
   289   unfolding null_def by simp
   289   by simp
   290 
   290 
   291 lemma ALL[import_const ALL : list_all]:
   291 lemma ALL[import_const ALL : list_all]:
   292   "list_all (P::'t18393 \<Rightarrow> bool) [] = True \<and>
   292   "list_all (P::'t18393 \<Rightarrow> bool) [] = True \<and>
   293   list_all P (h # t) = (P h \<and> list_all P t)"
   293   list_all P (h # t) = (P h \<and> list_all P t)"
   294   by simp
   294   by simp