doc-src/IsarRef/Thy/HOL_Specific.thy
changeset 41505 6d19301074cf
parent 41396 5379e4a85a66
child 41506 4c717333b0cc
equal deleted inserted replaced
41503:a7462e442e35 41505:6d19301074cf
   386 
   386 
   387 section {* Functorial structure of types *}
   387 section {* Functorial structure of types *}
   388 
   388 
   389 text {*
   389 text {*
   390   \begin{matharray}{rcl}
   390   \begin{matharray}{rcl}
   391     @{command_def (HOL) "type_lifting"} & : & @{text "local_theory \<rightarrow> proof(prove)"}
   391     @{command_def (HOL) "enriched_type"} & : & @{text "local_theory \<rightarrow> proof(prove)"}
   392   \end{matharray}
   392   \end{matharray}
   393 
   393 
   394   \begin{rail}
   394   \begin{rail}
   395     'type_lifting' (prefix ':')? term
   395     'enriched_type' (prefix ':')? term
   396     ;
   396     ;
   397   \end{rail}
   397   \end{rail}
   398 
   398 
   399   \begin{description}
   399   \begin{description}
   400 
   400 
   401   \item @{command (HOL) "type_lifting"} allows to prove and register
   401   \item @{command (HOL) "enriched_type"} allows to prove and register
   402   properties about type constructors which refer to their functorial
   402   properties about type constructors which refer to their functorial
   403   structure; these properties then can be used by other packages to
   403   structure; these properties then can be used by other packages to
   404   deal with those type constructors in certain type constructions.
   404   deal with those type constructors in certain type constructions.
   405   Characteristic theorems are noted in the current local theory; by
   405   Characteristic theorems are noted in the current local theory; by
   406   default, they are prefixed with base name of the type constructor,
   406   default, they are prefixed with base name of the type constructor,