ProgTutorial/FirstSteps.thy
changeset 412 73f716b9201a
parent 401 36d61044f9bf
child 413 95461cf6fd07
equal deleted inserted replaced
411:24fc00319c4a 412:73f716b9201a
   840   It is also possible to prove lemmas with the antiquotation @{text "@{lemma \<dots> by \<dots>}"}
   840   It is also possible to prove lemmas with the antiquotation @{text "@{lemma \<dots> by \<dots>}"}
   841   whose first argument is a statement (possibly many of them separated by @{text "and"})
   841   whose first argument is a statement (possibly many of them separated by @{text "and"})
   842   and the second is a proof. For example
   842   and the second is a proof. For example
   843 *}
   843 *}
   844 
   844 
   845 ML{*val foo_thm = @{lemma "True" and "True" by simp simp} *}
   845 ML{*val foo_thm = @{lemma "True" and "False \<Longrightarrow> P" by simp_all} *}
   846 
   846 
   847 text {*
   847 text {*
   848   The result can be printed out as follows.
   848   The result can be printed out as follows.
   849 
   849 
   850   @{ML_response_fake [gray,display]
   850   @{ML_response_fake [gray,display]