equal
deleted
inserted
replaced
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 \mbox{\isa{\isacommand{undo}}}. See the Isabelle/Isar Quick Reference |
105 Note that any Isabelle/Isar command may be retracted by \hyperlink{command.undo}{\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 % |
233 |
233 |
234 \end{enumerate} |
234 \end{enumerate} |
235 |
235 |
236 The Isar proof language is embedded into the new theory format as a |
236 The Isar proof language is embedded into the new theory format as a |
237 proper sub-language. Proof mode is entered by stating some |
237 proper sub-language. Proof mode is entered by stating some |
238 \mbox{\isa{\isacommand{theorem}}} or \mbox{\isa{\isacommand{lemma}}} at the theory level, and |
238 \hyperlink{command.theorem}{\mbox{\isa{\isacommand{theorem}}}} or \hyperlink{command.lemma}{\mbox{\isa{\isacommand{lemma}}}} at the theory level, and |
239 left again with the final conclusion (e.g.\ via \mbox{\isa{\isacommand{qed}}}). |
239 left again with the final conclusion (e.g.\ via \hyperlink{command.qed}{\mbox{\isa{\isacommand{qed}}}}). |
240 A few theory specification mechanisms also require some proof, such |
240 A few theory specification mechanisms also require some proof, such |
241 as HOL's \mbox{\isa{\isacommand{typedef}}} which demands non-emptiness of the |
241 as HOL's \hyperlink{command.typedef}{\mbox{\isa{\isacommand{typedef}}}} which demands non-emptiness of the |
242 representing sets.% |
242 representing sets.% |
243 \end{isamarkuptext}% |
243 \end{isamarkuptext}% |
244 \isamarkuptrue% |
244 \isamarkuptrue% |
245 % |
245 % |
246 \isamarkupsubsection{Document preparation \label{sec:document-prep}% |
246 \isamarkupsubsection{Document preparation \label{sec:document-prep}% |