src/HOL/Product_Type.thy
changeset 34900 9b12b0824bfe
parent 34886 873c31d9f10d
child 35115 446c5063e4fd
equal deleted inserted replaced
34899:8674bb6f727b 34900:9b12b0824bfe
   998 
   998 
   999 code_type *
   999 code_type *
  1000   (SML infix 2 "*")
  1000   (SML infix 2 "*")
  1001   (OCaml infix 2 "*")
  1001   (OCaml infix 2 "*")
  1002   (Haskell "!((_),/ (_))")
  1002   (Haskell "!((_),/ (_))")
  1003   (Scala "!((_),/ (_))")
  1003   (Scala "((_),/ (_))")
  1004 
  1004 
  1005 code_instance * :: eq
  1005 code_instance * :: eq
  1006   (Haskell -)
  1006   (Haskell -)
  1007 
  1007 
  1008 code_const "eq_class.eq \<Colon> 'a\<Colon>eq \<times> 'b\<Colon>eq \<Rightarrow> 'a \<times> 'b \<Rightarrow> bool"
  1008 code_const "eq_class.eq \<Colon> 'a\<Colon>eq \<times> 'b\<Colon>eq \<Rightarrow> 'a \<times> 'b \<Rightarrow> bool"