doc-src/IsarRef/Thy/document/intro.tex
changeset 26776 030db8c8b79d
parent 26767 cc127cc0951b
child 26842 81308d44fe0a
equal deleted inserted replaced
26775:06d6b1242dcf 26776:030db8c8b79d
   100 definition foo :: nat where "foo == 1";
   100 definition foo :: nat where "foo == 1";
   101 lemma "0 < foo" by (simp add: foo_def);
   101 lemma "0 < foo" by (simp add: foo_def);
   102 end;
   102 end;
   103 \end{ttbox}
   103 \end{ttbox}
   104 
   104 
   105   Note that any Isabelle/Isar command may be retracted by \isa{\isacommand{undo}}.  See the Isabelle/Isar Quick Reference
   105   Note that any Isabelle/Isar command may be retracted by \mbox{\isa{\isacommand{undo}}}.  See the Isabelle/Isar Quick Reference
   106   (\appref{ap:refcard}) for a comprehensive overview of available
   106   (\appref{ap:refcard}) for a comprehensive overview of available
   107   commands and other language elements.%
   107   commands and other language elements.%
   108 \end{isamarkuptext}%
   108 \end{isamarkuptext}%
   109 \isamarkuptrue%
   109 \isamarkuptrue%
   110 %
   110 %
   232 
   232 
   233   \end{enumerate}
   233   \end{enumerate}
   234 
   234 
   235   The Isar proof language is embedded into the new theory format as a
   235   The Isar proof language is embedded into the new theory format as a
   236   proper sub-language.  Proof mode is entered by stating some
   236   proper sub-language.  Proof mode is entered by stating some
   237   \isa{\isacommand{theorem}} or \isa{\isacommand{lemma}} at the theory level, and
   237   \mbox{\isa{\isacommand{theorem}}} or \mbox{\isa{\isacommand{lemma}}} at the theory level, and
   238   left again with the final conclusion (e.g.\ via \isa{\isacommand{qed}}).
   238   left again with the final conclusion (e.g.\ via \mbox{\isa{\isacommand{qed}}}).
   239   A few theory specification mechanisms also require some proof, such
   239   A few theory specification mechanisms also require some proof, such
   240   as HOL's \isa{\isacommand{typedef}} which demands non-emptiness of the
   240   as HOL's \mbox{\isa{\isacommand{typedef}}} which demands non-emptiness of the
   241   representing sets.%
   241   representing sets.%
   242 \end{isamarkuptext}%
   242 \end{isamarkuptext}%
   243 \isamarkuptrue%
   243 \isamarkuptrue%
   244 %
   244 %
   245 \isamarkupsubsection{Document preparation \label{sec:document-prep}%
   245 \isamarkupsubsection{Document preparation \label{sec:document-prep}%