src/HOL/ex/Cartouche_Examples.thy
changeset 56500 90f17a04567d
parent 56499 7e0178c84994
child 58889 5b7a9633cfa8
equal deleted inserted replaced
56499:7e0178c84994 56500:90f17a04567d
    25   from \<open>x = y\<close> have "x = y" .
    25   from \<open>x = y\<close> have "x = y" .
    26 
    26 
    27   txt \<open>Of course, this can be nested inside formal comments and
    27   txt \<open>Of course, this can be nested inside formal comments and
    28     antiquotations, e.g. like this @{thm \<open>x = y\<close>} or this @{thm sym
    28     antiquotations, e.g. like this @{thm \<open>x = y\<close>} or this @{thm sym
    29     [OF \<open>x = y\<close>]}.\<close>
    29     [OF \<open>x = y\<close>]}.\<close>
       
    30 
       
    31   have "x = y"
       
    32     by (tactic \<open>rtac @{thm \<open>x = y\<close>} 1\<close>)  -- \<open>more cartouches involving ML\<close>
    30 end
    33 end
    31 
    34 
    32 
    35 
    33 subsection {* Outer syntax: cartouche within command syntax *}
    36 subsection {* Outer syntax: cartouche within command syntax *}
    34 
    37