src/HOL/Option.thy
changeset 37880 3b9ca8d2c5fb
parent 36176 3fe7e97ccca8
child 38857 97775f3e8722
equal deleted inserted replaced
37879:443909380077 37880:3b9ca8d2c5fb
   112 
   112 
   113 code_const None and Some
   113 code_const None and Some
   114   (SML "NONE" and "SOME")
   114   (SML "NONE" and "SOME")
   115   (OCaml "None" and "Some _")
   115   (OCaml "None" and "Some _")
   116   (Haskell "Nothing" and "Just")
   116   (Haskell "Nothing" and "Just")
   117   (Scala "None" and "!Some((_))")
   117   (Scala "!None" and "Some")
   118 
   118 
   119 code_instance option :: eq
   119 code_instance option :: eq
   120   (Haskell -)
   120   (Haskell -)
   121 
   121 
   122 code_const "eq_class.eq \<Colon> 'a\<Colon>eq option \<Rightarrow> 'a option \<Rightarrow> bool"
   122 code_const "eq_class.eq \<Colon> 'a\<Colon>eq option \<Rightarrow> 'a option \<Rightarrow> bool"