src/Doc/Isar_Ref/Proof.thy
changeset 58552 66fed99e874f
parent 57979 fc136831d6ca
child 58618 782f0b662cae
equal deleted inserted replaced
58551:9986fb541c87 58552:66fed99e874f
   671   pretending to solve the pending claim without further ado.  This
   671   pretending to solve the pending claim without further ado.  This
   672   only works in interactive development, or if the @{attribute
   672   only works in interactive development, or if the @{attribute
   673   quick_and_dirty} is enabled.  Facts emerging from fake
   673   quick_and_dirty} is enabled.  Facts emerging from fake
   674   proofs are not the real thing.  Internally, the derivation object is
   674   proofs are not the real thing.  Internally, the derivation object is
   675   tainted by an oracle invocation, which may be inspected via the
   675   tainted by an oracle invocation, which may be inspected via the
   676   theorem status \cite{isabelle-implementation}.
   676   theorem status @{cite "isabelle-implementation"}.
   677   
   677   
   678   The most important application of @{command "sorry"} is to support
   678   The most important application of @{command "sorry"} is to support
   679   experimentation and top-down proof development.
   679   experimentation and top-down proof development.
   680 
   680 
   681   \end{description}
   681   \end{description}