src/Tools/Haskell/Haskell.thy
changeset 75015 eaf22c0e9ddf
parent 74871 0597884e6e91
child 75066 fe81645c0b40
equal deleted inserted replaced
75014:0778d233964d 75015:eaf22c0e9ddf
  3660   _pos :: Properties.T,
  3660   _pos :: Properties.T,
  3661   _name :: Bytes,
  3661   _name :: Bytes,
  3662   _typ :: Bytes,
  3662   _typ :: Bytes,
  3663   _value :: Bytes }
  3663   _value :: Bytes }
  3664 
  3664 
  3665 data T = Options (Map Bytes Opt)
  3665 newtype T = Options (Map Bytes Opt)
  3666 
  3666 
  3667 
  3667 
  3668 {- check -}
  3668 {- check -}
  3669 
  3669 
  3670 check_name :: T -> Bytes -> Opt
  3670 check_name :: T -> Bytes -> Opt