src/Doc/Datatypes/Datatypes.thy
changeset 55398 67e9fdd9ae9e
parent 55355 b5b64d9d1002
child 55410 54b09e82b9e1
equal deleted inserted replaced
55397:c2506f61fd26 55398:67e9fdd9ae9e
   769 
   769 
   770 \item[@{text "t."}\hthm{case} @{text "[simp, code]"}\rm:] ~ \\
   770 \item[@{text "t."}\hthm{case} @{text "[simp, code]"}\rm:] ~ \\
   771 @{thm list.case(1)[no_vars]} \\
   771 @{thm list.case(1)[no_vars]} \\
   772 @{thm list.case(2)[no_vars]}
   772 @{thm list.case(2)[no_vars]}
   773 
   773 
   774 \item[@{text "t."}\hthm{case\_cong}\rm:] ~ \\
   774 \item[@{text "t."}\hthm{case\_cong} @{text "[fundef_cong]"}\rm:] ~ \\
   775 @{thm list.case_cong[no_vars]}
   775 @{thm list.case_cong[no_vars]}
   776 
   776 
   777 \item[@{text "t."}\hthm{weak\_case\_cong} @{text "[cong]"}\rm:] ~ \\
   777 \item[@{text "t."}\hthm{weak\_case\_cong} @{text "[cong]"}\rm:] ~ \\
   778 @{thm list.weak_case_cong[no_vars]}
   778 @{thm list.weak_case_cong[no_vars]}
   779 
   779 
  2603 
  2603 
  2604 % options: no_discs_sels no_code rep_compat
  2604 % options: no_discs_sels no_code rep_compat
  2605 
  2605 
  2606 \noindent
  2606 \noindent
  2607 Section~\ref{ssec:datatype-generated-theorems} lists the generated theorems.
  2607 Section~\ref{ssec:datatype-generated-theorems} lists the generated theorems.
       
  2608 For technical reasons, the @{text "[fundef_cong]"} attribute is not set on the
       
  2609 generated @{text case_cong} theorem. It can be added manually using
       
  2610 \keyw{declare}.
  2608 *}
  2611 *}
  2609 
  2612 
  2610 
  2613 
  2611 (*
  2614 (*
  2612 section {* Standard ML Interface
  2615 section {* Standard ML Interface