src/HOL/Isar_Examples/Structured_Statements.thy
changeset 69597 ff784d5a5bfb
parent 63583 a39baba12732
equal deleted inserted replaced
69596:c8a2755bf220 69597:ff784d5a5bfb
   150   fix A :: "'a \<Rightarrow> bool"
   150   fix A :: "'a \<Rightarrow> bool"
   151   fix C
   151   fix C
   152 
   152 
   153   have C
   153   have C
   154   proof -
   154   proof -
   155     show ?thesis when "A x" (is ?A) for x :: 'a  \<comment> \<open>abstract @{term x}\<close>
   155     show ?thesis when "A x" (is ?A) for x :: 'a  \<comment> \<open>abstract \<^term>\<open>x\<close>\<close>
   156       using that \<proof>
   156       using that \<proof>
   157     show "?A a"  \<comment> \<open>concrete @{term a}\<close>
   157     show "?A a"  \<comment> \<open>concrete \<^term>\<open>a\<close>\<close>
   158       \<proof>
   158       \<proof>
   159   qed
   159   qed
   160 end
   160 end
   161 
   161 
   162 end
   162 end