doc-src/IsarRef/Thy/HOL_Specific.thy
changeset 37420 1cf6f134e7f2
parent 36453 2f383885d8f8
child 37422 6d19e4e6ebf5
equal deleted inserted replaced
37409:6c9f23863808 37420:1cf6f134e7f2
  1064     ;
  1064     ;
  1065 
  1065 
  1066     target: 'OCaml' | 'SML' | 'Haskell'
  1066     target: 'OCaml' | 'SML' | 'Haskell'
  1067     ;
  1067     ;
  1068 
  1068 
  1069     'code\_datatype' const +
  1069     'code\_datatype' ( const + )
  1070     ;
  1070     ;
  1071 
  1071 
  1072     'code\_const' (const + 'and') \\
  1072     'code\_const' (const + 'and') \\
  1073       ( ( '(' target ( syntax ? + 'and' ) ')' ) + )
  1073       ( ( '(' target ( syntax ? + 'and' ) ')' ) + )
  1074     ;
  1074     ;