ProgTutorial/Essential.thy
changeset 481 32323727af96
parent 469 7a558c5119b2
child 482 9699ad581dc2
equal deleted inserted replaced
480:ae49c5e8868e 481:32323727af96
  2223   can use @{ML_ind declaration_attribute in Thm}. To illustrate this function,
  2223   can use @{ML_ind declaration_attribute in Thm}. To illustrate this function,
  2224   let us introduce a theorem list.
  2224   let us introduce a theorem list.
  2225 *}
  2225 *}
  2226 
  2226 
  2227 ML{*structure MyThms = Named_Thms
  2227 ML{*structure MyThms = Named_Thms
  2228   (val name = "attr_thms" 
  2228   (val name = @{binding "attr_thms"} 
  2229    val description = "Theorems for an Attribute") *}
  2229    val description = "Theorems for an Attribute") *}
  2230 
  2230 
  2231 text {* 
  2231 text {* 
  2232   We are going to modify this list by adding and deleting theorems.
  2232   We are going to modify this list by adding and deleting theorems.
  2233   For this we use the two functions @{ML MyThms.add_thm} and
  2233   For this we use the two functions @{ML MyThms.add_thm} and