author | wenzelm |
Thu, 07 Aug 2025 22:42:21 +0200 | |
changeset 82968 | b2b88d5b01b6 |
parent 80914 | d97fdabd9e2b |
permissions | -rw-r--r-- |
47269 | 1 |
(* Title: HOL/Library/LaTeXsugar.thy |
55116 | 2 |
Author: Gerwin Klein, Tobias Nipkow, Norbert Schirmer |
47269 | 3 |
Copyright 2005 NICTA and TUM |
4 |
*) |
|
5 |
||
6 |
(*<*) |
|
7 |
theory LaTeXsugar |
|
8 |
imports Main |
|
9 |
begin |
|
10 |
||
11 |
(* DUMMY *) |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
74563
diff
changeset
|
12 |
consts DUMMY :: 'a (\<open>\<^latex>\<open>\_\<close>\<close>) |
47269 | 13 |
|
14 |
(* THEOREMS *) |
|
15 |
notation (Rule output) |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
74563
diff
changeset
|
16 |
Pure.imp (\<open>\<^latex>\<open>\mbox{}\inferrule{\mbox{\<close>_\<^latex>\<open>}}\<close>\<^latex>\<open>{\mbox{\<close>_\<^latex>\<open>}}\<close>\<close>) |
47269 | 17 |
|
18 |
syntax (Rule output) |
|
19 |
"_bigimpl" :: "asms \<Rightarrow> prop \<Rightarrow> prop" |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
74563
diff
changeset
|
20 |
(\<open>\<^latex>\<open>\mbox{}\inferrule{\<close>_\<^latex>\<open>}\<close>\<^latex>\<open>{\mbox{\<close>_\<^latex>\<open>}}\<close>\<close>) |
47269 | 21 |
|
22 |
"_asms" :: "prop \<Rightarrow> asms \<Rightarrow> asms" |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
74563
diff
changeset
|
23 |
(\<open>\<^latex>\<open>\mbox{\<close>_\<^latex>\<open>}\\\<close>/ _\<close>) |
47269 | 24 |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
74563
diff
changeset
|
25 |
"_asm" :: "prop \<Rightarrow> asms" (\<open>\<^latex>\<open>\mbox{\<close>_\<^latex>\<open>}\<close>\<close>) |
47269 | 26 |
|
27 |
notation (Axiom output) |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
74563
diff
changeset
|
28 |
"Trueprop" (\<open>\<^latex>\<open>\mbox{}\inferrule{\mbox{}}{\mbox{\<close>_\<^latex>\<open>}}\<close>\<close>) |
47269 | 29 |
|
30 |
notation (IfThen output) |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
74563
diff
changeset
|
31 |
Pure.imp (\<open>\<^latex>\<open>{\normalsize{}\<close>If\<^latex>\<open>\,}\<close> _/ \<^latex>\<open>{\normalsize \,\<close>then\<^latex>\<open>\,}\<close>/ _.\<close>) |
47269 | 32 |
syntax (IfThen output) |
33 |
"_bigimpl" :: "asms \<Rightarrow> prop \<Rightarrow> prop" |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
74563
diff
changeset
|
34 |
(\<open>\<^latex>\<open>{\normalsize{}\<close>If\<^latex>\<open>\,}\<close> _ /\<^latex>\<open>{\normalsize \,\<close>then\<^latex>\<open>\,}\<close>/ _.\<close>) |
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
74563
diff
changeset
|
35 |
"_asms" :: "prop \<Rightarrow> asms \<Rightarrow> asms" (\<open>\<^latex>\<open>\mbox{\<close>_\<^latex>\<open>}\<close> /\<^latex>\<open>{\normalsize \,\<close>and\<^latex>\<open>\,}\<close>/ _\<close>) |
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
74563
diff
changeset
|
36 |
"_asm" :: "prop \<Rightarrow> asms" (\<open>\<^latex>\<open>\mbox{\<close>_\<^latex>\<open>}\<close>\<close>) |
47269 | 37 |
|
38 |
notation (IfThenNoBox output) |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
74563
diff
changeset
|
39 |
Pure.imp (\<open>\<^latex>\<open>{\normalsize{}\<close>If\<^latex>\<open>\,}\<close> _/ \<^latex>\<open>{\normalsize \,\<close>then\<^latex>\<open>\,}\<close>/ _.\<close>) |
47269 | 40 |
syntax (IfThenNoBox output) |
41 |
"_bigimpl" :: "asms \<Rightarrow> prop \<Rightarrow> prop" |
|
80914
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
74563
diff
changeset
|
42 |
(\<open>\<^latex>\<open>{\normalsize{}\<close>If\<^latex>\<open>\,}\<close> _ /\<^latex>\<open>{\normalsize \,\<close>then\<^latex>\<open>\,}\<close>/ _.\<close>) |
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
74563
diff
changeset
|
43 |
"_asms" :: "prop \<Rightarrow> asms \<Rightarrow> asms" (\<open>_ /\<^latex>\<open>{\normalsize \,\<close>and\<^latex>\<open>\,}\<close>/ _\<close>) |
d97fdabd9e2b
standardize mixfix annotations via "isabelle update -a -u mixfix_cartouches" --- to simplify systematic editing;
wenzelm
parents:
74563
diff
changeset
|
44 |
"_asm" :: "prop \<Rightarrow> asms" (\<open>_\<close>) |
47269 | 45 |
|
67463 | 46 |
setup \<open> |
73761 | 47 |
Document_Output.antiquotation_pretty_source \<^binding>\<open>const_typ\<close> |
74563 | 48 |
(Scan.lift Parse.embedded_inner_syntax) |
67463 | 49 |
(fn ctxt => fn c => |
69082 | 50 |
let val tc = Proof_Context.read_const {proper = false, strict = false} ctxt c in |
73761 | 51 |
Pretty.block [Document_Output.pretty_term ctxt tc, Pretty.str " ::", |
67505
ceb324e34c14
clarified signature: items with \isasep are special;
wenzelm
parents:
67463
diff
changeset
|
52 |
Pretty.brk 1, Syntax.pretty_typ ctxt (fastype_of tc)] |
67463 | 53 |
end) |
67406 | 54 |
\<close> |
49629 | 55 |
|
47269 | 56 |
end |
67399 | 57 |
(*>*) |