src/HOL/Import/HOL/HOL4Base.thy
changeset 23290 c358025ad8db
parent 17727 83d64a461507
child 30952 7ab2716dd93b
equal deleted inserted replaced
23289:0cf371d943b1 23290:c358025ad8db
  5526 lemma IS_EL_FOLDL_MAP: "ALL (x::'a::type) xa::'a::type list.
  5526 lemma IS_EL_FOLDL_MAP: "ALL (x::'a::type) xa::'a::type list.
  5527    x mem xa = foldl op | False (map (op = x) xa)"
  5527    x mem xa = foldl op | False (map (op = x) xa)"
  5528   by (import rich_list IS_EL_FOLDL_MAP)
  5528   by (import rich_list IS_EL_FOLDL_MAP)
  5529 
  5529 
  5530 lemma FILTER_FILTER: "ALL (P::'a::type => bool) (Q::'a::type => bool) l::'a::type list.
  5530 lemma FILTER_FILTER: "ALL (P::'a::type => bool) (Q::'a::type => bool) l::'a::type list.
  5531    filter P (filter Q l) = [x::'a::type:l. P x & Q x]"
  5531    filter P (filter Q l) = [x::'a::type<-l. P x & Q x]"
  5532   by (import rich_list FILTER_FILTER)
  5532   by (import rich_list FILTER_FILTER)
  5533 
  5533 
  5534 lemma FCOMM_FOLDR_FLAT: "ALL (g::'a::type => 'a::type => 'a::type)
  5534 lemma FCOMM_FOLDR_FLAT: "ALL (g::'a::type => 'a::type => 'a::type)
  5535    f::'b::type => 'a::type => 'a::type.
  5535    f::'b::type => 'a::type => 'a::type.
  5536    FCOMM g f -->
  5536    FCOMM g f -->