src/Doc/Prog_Prove/LaTeXsugar.thy
changeset 73761 ef1a18e20ace
parent 69082 0405d06f08f3
child 74563 042041c0ebeb
equal deleted inserted replaced
73760:f4be1b0d7a51 73761:ef1a18e20ace
    42   ("\<^latex>\<open>{\\normalsize{}\<close>If\<^latex>\<open>\\,}\<close> _ /\<^latex>\<open>{\\normalsize \\,\<close>then\<^latex>\<open>\\,}\<close>/ _.")
    42   ("\<^latex>\<open>{\\normalsize{}\<close>If\<^latex>\<open>\\,}\<close> _ /\<^latex>\<open>{\\normalsize \\,\<close>then\<^latex>\<open>\\,}\<close>/ _.")
    43   "_asms" :: "prop \<Rightarrow> asms \<Rightarrow> asms" ("_ /\<^latex>\<open>{\\normalsize \\,\<close>and\<^latex>\<open>\\,}\<close>/ _")
    43   "_asms" :: "prop \<Rightarrow> asms \<Rightarrow> asms" ("_ /\<^latex>\<open>{\\normalsize \\,\<close>and\<^latex>\<open>\\,}\<close>/ _")
    44   "_asm" :: "prop \<Rightarrow> asms" ("_")
    44   "_asm" :: "prop \<Rightarrow> asms" ("_")
    45 
    45 
    46 setup \<open>
    46 setup \<open>
    47   Thy_Output.antiquotation_pretty_source \<^binding>\<open>const_typ\<close> (Scan.lift Args.embedded_inner_syntax)
    47   Document_Output.antiquotation_pretty_source \<^binding>\<open>const_typ\<close>
       
    48     (Scan.lift Args.embedded_inner_syntax)
    48     (fn ctxt => fn c =>
    49     (fn ctxt => fn c =>
    49       let val tc = Proof_Context.read_const {proper = false, strict = false} ctxt c in
    50       let val tc = Proof_Context.read_const {proper = false, strict = false} ctxt c in
    50         Pretty.block [Thy_Output.pretty_term ctxt tc, Pretty.str " ::",
    51         Pretty.block [Document_Output.pretty_term ctxt tc, Pretty.str " ::",
    51           Pretty.brk 1, Syntax.pretty_typ ctxt (fastype_of tc)]
    52           Pretty.brk 1, Syntax.pretty_typ ctxt (fastype_of tc)]
    52       end)
    53       end)
    53 \<close>
    54 \<close>
    54 
    55 
    55 end
    56 end