src/HOL/Option.thy
changeset 34886 873c31d9f10d
parent 32069 6d28bbd33e2c
child 35719 99b6152aedf5
equal deleted inserted replaced
34878:d7786f56f081 34886:873c31d9f10d
   113 
   113 
   114 code_type option
   114 code_type option
   115   (SML "_ option")
   115   (SML "_ option")
   116   (OCaml "_ option")
   116   (OCaml "_ option")
   117   (Haskell "Maybe _")
   117   (Haskell "Maybe _")
       
   118   (Scala "!Option[(_)]")
   118 
   119 
   119 code_const None and Some
   120 code_const None and Some
   120   (SML "NONE" and "SOME")
   121   (SML "NONE" and "SOME")
   121   (OCaml "None" and "Some _")
   122   (OCaml "None" and "Some _")
   122   (Haskell "Nothing" and "Just")
   123   (Haskell "Nothing" and "Just")
       
   124   (Scala "None" and "!Some((_))")
   123 
   125 
   124 code_instance option :: eq
   126 code_instance option :: eq
   125   (Haskell -)
   127   (Haskell -)
   126 
   128 
   127 code_const "eq_class.eq \<Colon> 'a\<Colon>eq option \<Rightarrow> 'a option \<Rightarrow> bool"
   129 code_const "eq_class.eq \<Colon> 'a\<Colon>eq option \<Rightarrow> 'a option \<Rightarrow> bool"
   131   option NONE SOME
   133   option NONE SOME
   132 
   134 
   133 code_reserved OCaml
   135 code_reserved OCaml
   134   option None Some
   136   option None Some
   135 
   137 
       
   138 code_reserved Scala
       
   139   Option None Some
       
   140 
   136 end
   141 end