ProgTutorial/Tactical.thy
changeset 556 3c214b215f7e
parent 554 638ed040e6f8
child 559 ffa5c4ec9611
equal deleted inserted replaced
555:2c34c69236ce 556:3c214b215f7e
   386   as the user would see it.  For example, processing the proof
   386   as the user would see it.  For example, processing the proof
   387 *}
   387 *}
   388  
   388  
   389 lemma 
   389 lemma 
   390   shows "False \<Longrightarrow> True"
   390   shows "False \<Longrightarrow> True"
   391 apply(tactic {* print_tac "foo message" *})
   391 apply(tactic {* print_tac @{context} "foo message" *})
   392 txt{*gives:
   392 txt{*gives:
   393      \begin{isabelle}
   393      \begin{isabelle}
   394      @{text "foo message"}\\[3mm] 
   394      @{text "foo message"}\\[3mm] 
   395      @{prop "False \<Longrightarrow> True"}\\
   395      @{prop "False \<Longrightarrow> True"}\\
   396      @{text " 1. False \<Longrightarrow> True"}\\
   396      @{text " 1. False \<Longrightarrow> True"}\\