doc-src/IsarRef/Thy/Generic.thy
changeset 46494 ea2ae63336f3
parent 46277 aea65ff733b4
child 46706 877d57975427
equal deleted inserted replaced
46493:7e69b9f3149f 46494:ea2ae63336f3
  1224 
  1224 
  1225   Generic tools may refer to the information provided by object-logic
  1225   Generic tools may refer to the information provided by object-logic
  1226   declarations internally.
  1226   declarations internally.
  1227 
  1227 
  1228   @{rail "
  1228   @{rail "
  1229     @@{command judgment} @{syntax constdecl}
  1229     @@{command judgment} @{syntax name} '::' @{syntax type} @{syntax mixfix}?
  1230     ;
  1230     ;
  1231     @@{attribute atomize} ('(' 'full' ')')?
  1231     @@{attribute atomize} ('(' 'full' ')')?
  1232     ;
  1232     ;
  1233     @@{attribute rule_format} ('(' 'noasm' ')')?
  1233     @@{attribute rule_format} ('(' 'noasm' ')')?
  1234   "}
  1234   "}