src/HOL/Int.thy
changeset 53572 6646bb548c6b
parent 53131 82cc2aeb7d13
child 54202 de1816a7293e
equal deleted inserted replaced
53571:cbb94074682b 53572:6646bb548c6b
  1612   by simp_all
  1612   by simp_all
  1613 
  1613 
  1614 
  1614 
  1615 text {* Serializer setup *}
  1615 text {* Serializer setup *}
  1616 
  1616 
  1617 code_modulename SML
  1617 code_identifier
  1618   Int Arith
  1618   code_module Int \<rightharpoonup> (SML) Arith and (OCaml) Arith and (Haskell) Arith
  1619 
       
  1620 code_modulename OCaml
       
  1621   Int Arith
       
  1622 
       
  1623 code_modulename Haskell
       
  1624   Int Arith
       
  1625 
  1619 
  1626 quickcheck_params [default_type = int]
  1620 quickcheck_params [default_type = int]
  1627 
  1621 
  1628 hide_const (open) Pos Neg sub dup
  1622 hide_const (open) Pos Neg sub dup
  1629 
  1623