doc-src/IsarRef/Thy/HOL_Specific.thy
changeset 36139 0c2538afe8e8
parent 35841 94f901e4969a
child 36158 d2ad76e374d3
equal deleted inserted replaced
36138:1faa0fc34174 36139:0c2538afe8e8
   469   equations take precedence over later ones.  This allows to give the
   469   equations take precedence over later ones.  This allows to give the
   470   specification in a format very similar to functional programming.
   470   specification in a format very similar to functional programming.
   471   Note that the resulting simplification and induction rules
   471   Note that the resulting simplification and induction rules
   472   correspond to the transformed specification, not the one given
   472   correspond to the transformed specification, not the one given
   473   originally. This usually means that each equation given by the user
   473   originally. This usually means that each equation given by the user
   474   may result in several theroems.  Also note that this automatic
   474   may result in several theorems.  Also note that this automatic
   475   transformation only works for ML-style datatype patterns.
   475   transformation only works for ML-style datatype patterns.
   476 
   476 
   477   \item @{text domintros} enables the automated generation of
   477   \item @{text domintros} enables the automated generation of
   478   introduction rules for the domain predicate. While mostly not
   478   introduction rules for the domain predicate. While mostly not
   479   needed, they can be helpful in some proofs about partial functions.
   479   needed, they can be helpful in some proofs about partial functions.