doc-src/IsarRef/Thy/HOL_Specific.thy
changeset 45701 615da8b8d758
parent 45678 1a6206f538d4
child 45758 6210c350d88b
child 45767 fe2fd2f76f48
equal deleted inserted replaced
45700:9dcbf6a1829c 45701:615da8b8d758
   691     @@{command (HOL) datatype} (spec + @'and')
   691     @@{command (HOL) datatype} (spec + @'and')
   692     ;
   692     ;
   693     @@{command (HOL) rep_datatype} ('(' (@{syntax name} +) ')')? (@{syntax term} +)
   693     @@{command (HOL) rep_datatype} ('(' (@{syntax name} +) ')')? (@{syntax term} +)
   694     ;
   694     ;
   695 
   695 
   696     spec: @{syntax parname}? @{syntax typespec} @{syntax mixfix}? '=' (cons + '|')
   696     spec: @{syntax typespec} @{syntax mixfix}? '=' (cons + '|')
   697     ;
   697     ;
   698     cons: @{syntax name} (@{syntax type} * ) @{syntax mixfix}?
   698     cons: @{syntax name} (@{syntax type} * ) @{syntax mixfix}?
   699   "}
   699   "}
   700 
   700 
   701   \begin{description}
   701   \begin{description}