doc-src/IsarRef/Thy/HOL_Specific.thy
changeset 47349 803729c9fd4d
parent 46641 8801a24f9e9a
child 47802 f6cf7148d452
equal deleted inserted replaced
47348:9a82999ebbd6 47349:803729c9fd4d
  1380 
  1380 
  1381   \item @{attribute (HOL) quot_thm} declares that a certain theorem
  1381   \item @{attribute (HOL) quot_thm} declares that a certain theorem
  1382     is a quotient extension theorem. Quotient extension theorems
  1382     is a quotient extension theorem. Quotient extension theorems
  1383     allow for quotienting inside container types. Given a polymorphic
  1383     allow for quotienting inside container types. Given a polymorphic
  1384     type that serves as a container, a map function defined for this
  1384     type that serves as a container, a map function defined for this
  1385     container  using @{command (HOL) "enriched_type"} and a relation
  1385     container using @{command (HOL) "enriched_type"} and a relation
  1386     map defined for for the container type, the quotient extension
  1386     map defined for for the container type, the quotient extension
  1387     theorem should be @{term "Quotient R Abs Rep \<Longrightarrow> Quotient
  1387     theorem should be @{term "Quotient3 R Abs Rep \<Longrightarrow> Quotient3
  1388     (rel_map R) (map Abs) (map Rep)"}. Quotient extension theorems
  1388     (rel_map R) (map Abs) (map Rep)"}. Quotient extension theorems
  1389     are stored in a database and are used all the steps of lifting
  1389     are stored in a database and are used all the steps of lifting
  1390     theorems.
  1390     theorems.
  1391 
  1391 
  1392   \end{description}
  1392   \end{description}
  1737     \item[@{text iterations}] sets how many sets of assignments are
  1737     \item[@{text iterations}] sets how many sets of assignments are
  1738     generated for each particular size.
  1738     generated for each particular size.
  1739 
  1739 
  1740     \item[@{text no_assms}] specifies whether assumptions in
  1740     \item[@{text no_assms}] specifies whether assumptions in
  1741     structured proofs should be ignored.
  1741     structured proofs should be ignored.
       
  1742 
       
  1743     \item[@{text locale}] specifies how to process conjectures in
       
  1744     a locale context, i.e., they can be interpreted or expanded.
       
  1745     The option is a whitespace-separated list of the two words
       
  1746     @{text interpret} and @{text expand}. The list determines the
       
  1747     order they are employed. The default setting is to first use 
       
  1748     interpretations and then test the expanded conjecture.
       
  1749     The option is only provided as attribute declaration, but not
       
  1750     as parameter to the command. 
  1742 
  1751 
  1743     \item[@{text timeout}] sets the time limit in seconds.
  1752     \item[@{text timeout}] sets the time limit in seconds.
  1744 
  1753 
  1745     \item[@{text default_type}] sets the type(s) generally used to
  1754     \item[@{text default_type}] sets the type(s) generally used to
  1746     instantiate type variables.
  1755     instantiate type variables.