equal
deleted
inserted
replaced
88 definition foo :: nat where "foo == 1"; |
88 definition foo :: nat where "foo == 1"; |
89 lemma "0 < foo" by (simp add: foo_def); |
89 lemma "0 < foo" by (simp add: foo_def); |
90 end; |
90 end; |
91 \end{ttbox} |
91 \end{ttbox} |
92 |
92 |
93 Any Isabelle/Isar command may be retracted by @{command "undo"}. |
93 Any Isabelle/Isar command may be retracted by @{command undo}. |
94 See the Isabelle/Isar Quick Reference (\appref{ap:refcard}) for a |
94 See the Isabelle/Isar Quick Reference (\appref{ap:refcard}) for a |
95 comprehensive overview of available commands and other language |
95 comprehensive overview of available commands and other language |
96 elements. |
96 elements. |
97 *} |
97 *} |
98 |
98 |
217 |
217 |
218 \end{enumerate} |
218 \end{enumerate} |
219 |
219 |
220 The Isar proof language is embedded into the new theory format as a |
220 The Isar proof language is embedded into the new theory format as a |
221 proper sub-language. Proof mode is entered by stating some |
221 proper sub-language. Proof mode is entered by stating some |
222 @{command "theorem"} or @{command "lemma"} at the theory level, and |
222 @{command theorem} or @{command lemma} at the theory level, and |
223 left again with the final conclusion (e.g.\ via @{command "qed"}). |
223 left again with the final conclusion (e.g.\ via @{command qed}). |
224 A few theory specification mechanisms also require some proof, such |
224 A few theory specification mechanisms also require some proof, such |
225 as HOL's @{command "typedef"} which demands non-emptiness of the |
225 as HOL's @{command typedef} which demands non-emptiness of the |
226 representing sets. |
226 representing sets. |
227 *} |
227 *} |
228 |
228 |
229 |
229 |
230 section {* How to write Isar proofs anyway? \label{sec:isar-howto} *} |
230 section {* How to write Isar proofs anyway? \label{sec:isar-howto} *} |