src/HOL/Set.thy
changeset 25360 b8251517f508
parent 25287 094dab519ff5
child 25460 b80087af2274
equal deleted inserted replaced
25359:96202af17d2b 25360:b8251517f508
  2253 
  2253 
  2254 lemma Union_code [code func]:
  2254 lemma Union_code [code func]:
  2255   "Union A = UNION A (\<lambda>x. x)"
  2255   "Union A = UNION A (\<lambda>x. x)"
  2256   by auto
  2256   by auto
  2257 
  2257 
       
  2258 code_reserved SML union inter (* Avoid clashes with ML infixes *)
  2258 
  2259 
  2259 subsection {* Basic ML bindings *}
  2260 subsection {* Basic ML bindings *}
  2260 
  2261 
  2261 ML {*
  2262 ML {*
  2262 val Ball_def = @{thm Ball_def}
  2263 val Ball_def = @{thm Ball_def}