diff -r d505274da801 -r 4566bac4517d src/HOL/IMP/ACom.thy --- a/src/HOL/IMP/ACom.thy Mon Aug 20 20:54:40 2018 +0200 +++ b/src/HOL/IMP/ACom.thy Tue Aug 21 17:29:46 2018 +0200 @@ -1,11 +1,11 @@ (* Author: Tobias Nipkow *) +subsection "Annotated Commands" + theory ACom imports Com begin -subsection "Annotated Commands" - datatype 'a acom = SKIP 'a ("SKIP {_}" 61) | Assign vname aexp 'a ("(_ ::= _/ {_})" [1000, 61, 0] 61) |