author | krauss |
Thu, 26 May 2011 00:12:30 +0200 | |
changeset 42977 | a59db6677521 |
parent 42632 | ebec0c1a5984 |
child 42915 | f35aae36cad0 |
permissions | -rw-r--r-- |
7046 | 1 |
## targets |
2 |
||
3 |
default: dvi |
|
4 |
||
5 |
||
6 |
## dependencies |
|
7 |
||
8 |
include ../Makefile.in |
|
9 |
||
10 |
NAME = isar-ref |
|
11 |
||
27048 | 12 |
FILES = isar-ref.tex style.sty Thy/document/Generic.tex \ |
26906 | 13 |
Thy/document/HOLCF_Specific.tex Thy/document/HOL_Specific.tex \ |
14 |
Thy/document/ML_Tactic.tex Thy/document/Proof.tex \ |
|
15 |
Thy/document/Quick_Reference.tex Thy/document/Spec.tex \ |
|
28762
f5d79aeffd81
separate chapter "Inner syntax --- the term language";
wenzelm
parents:
27048
diff
changeset
|
16 |
Thy/document/ZF_Specific.tex Thy/document/Inner_Syntax.tex \ |
f5d79aeffd81
separate chapter "Inner syntax --- the term language";
wenzelm
parents:
27048
diff
changeset
|
17 |
Thy/document/Introduction.tex Thy/document/Document_Preparation.tex \ |
28838
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
28762
diff
changeset
|
18 |
Thy/document/Misc.tex Thy/document/Outer_Syntax.tex \ |
42632
ebec0c1a5984
just one railsetup.sty which is shipped with the official distribution to accompany @{rail} in Pure;
wenzelm
parents:
42618
diff
changeset
|
19 |
Thy/document/Symbols.tex ../isar.sty ../proof.sty ../iman.sty \ |
ebec0c1a5984
just one railsetup.sty which is shipped with the official distribution to accompany @{rail} in Pure;
wenzelm
parents:
42618
diff
changeset
|
20 |
../extra.sty ../ttbox.sty ../../lib/texinputs/isabelle.sty \ |
ebec0c1a5984
just one railsetup.sty which is shipped with the official distribution to accompany @{rail} in Pure;
wenzelm
parents:
42618
diff
changeset
|
21 |
../../lib/texinputs/isabellesym.sty \ |
ebec0c1a5984
just one railsetup.sty which is shipped with the official distribution to accompany @{rail} in Pure;
wenzelm
parents:
42618
diff
changeset
|
22 |
../../lib/texinputs/railsetup.sty ../pdfsetup.sty ../manual.bib |
28838
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
28762
diff
changeset
|
23 |
|
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
28762
diff
changeset
|
24 |
OUTPUT = syms.tex |
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
28762
diff
changeset
|
25 |
|
42511 | 26 |
syms.tex: showsymbols ../../lib/texinputs/isabellesym.sty |
27 |
@./showsymbols <../../lib/texinputs/isabellesym.sty >syms.tex |
|
28838
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
28762
diff
changeset
|
28 |
|
7046 | 29 |
|
30 |
dvi: $(NAME).dvi |
|
31 |
||
28838
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
28762
diff
changeset
|
32 |
$(NAME).dvi: $(FILES) isabelle_isar.eps syms.tex |
7046 | 33 |
$(LATEX) $(NAME) |
34 |
$(BIBTEX) $(NAME) |
|
35 |
$(LATEX) $(NAME) |
|
36 |
$(LATEX) $(NAME) |
|
37 |
$(SEDINDEX) $(NAME) |
|
38 |
$(LATEX) $(NAME) |
|
39 |
||
40 |
pdf: $(NAME).pdf |
|
41 |
||
28838
d5db6dfcb34a
moved table of standard Isabelle symbols to isar-ref manual;
wenzelm
parents:
28762
diff
changeset
|
42 |
$(NAME).pdf: $(FILES) isabelle_isar.pdf syms.tex |
7046 | 43 |
$(PDFLATEX) $(NAME) |
44 |
$(BIBTEX) $(NAME) |
|
45 |
$(PDFLATEX) $(NAME) |
|
46 |
$(PDFLATEX) $(NAME) |
|
47 |
$(SEDINDEX) $(NAME) |
|
48 |
$(FIXBOOKMARKS) $(NAME).out |
|
49 |
$(PDFLATEX) $(NAME) |