src/HOL/Library/ExecutableSet.thy
changeset 21911 e29bcab0c81c
parent 21875 5df10a17644e
child 22177 515021e98684
equal deleted inserted replaced
21910:5b553ed23251 21911:e29bcab0c81c
   273 nonfix union;
   273 nonfix union;
   274 nonfix subset;
   274 nonfix subset;
   275 *}
   275 *}
   276 
   276 
   277 code_modulename SML
   277 code_modulename SML
       
   278   ExecutableSet List
       
   279   Set List
       
   280 
       
   281 code_modulename OCaml
   278   ExecutableSet List
   282   ExecutableSet List
   279   Set List
   283   Set List
   280 
   284 
   281 code_modulename Haskell
   285 code_modulename Haskell
   282   ExecutableSet List
   286   ExecutableSet List