src/Doc/IsarImplementation/Logic.thy
changeset 52788 da1fdbfebd39
parent 52630 fe411c1dc180
child 53015 a1119cf551e8
equal deleted inserted replaced
52787:c143ad7811fc 52788:da1fdbfebd39
   716   certified terms and theorems to produce certified terms again.
   716   certified terms and theorems to produce certified terms again.
   717 
   717 
   718   \item Type @{ML_type thm} represents proven propositions.  This is
   718   \item Type @{ML_type thm} represents proven propositions.  This is
   719   an abstract datatype that guarantees that its values have been
   719   an abstract datatype that guarantees that its values have been
   720   constructed by basic principles of the @{ML_struct Thm} module.
   720   constructed by basic principles of the @{ML_struct Thm} module.
   721   Every @{ML_type thm} value contains a sliding back-reference to the
   721   Every @{ML_type thm} value refers its background theory,
   722   enclosing theory, cf.\ \secref{sec:context-theory}.
   722   cf.\ \secref{sec:context-theory}.
   723 
   723 
   724   \item @{ML Thm.transfer}~@{text "thy thm"} transfers the given
   724   \item @{ML Thm.transfer}~@{text "thy thm"} transfers the given
   725   theorem to a \emph{larger} theory, see also \secref{sec:context}.
   725   theorem to a \emph{larger} theory, see also \secref{sec:context}.
   726   This formal adjustment of the background context has no logical
   726   This formal adjustment of the background context has no logical
   727   significance, but is occasionally required for formal reasons, e.g.\
   727   significance, but is occasionally required for formal reasons, e.g.\