# HG changeset patch # User wenzelm # Date 925922141 -7200 # Node ID 5a94bd71cc41e55f343a3f1c89dc8be48f22496b # Parent dc5bf3f40ad3e025cf53b78e62d939adf6eeda9d improved Makefile; diff -r dc5bf3f40ad3 -r 5a94bd71cc41 doc-src/Ref/Makefile --- a/doc-src/Ref/Makefile Wed May 05 18:26:10 1999 +0200 +++ b/doc-src/Ref/Makefile Wed May 05 18:35:41 1999 +0200 @@ -1,35 +1,31 @@ -# $Id$ -######################################################################### -# # -# Makefile for the report "The Isabelle Reference Manual" # -# # -######################################################################### +# +# $Id$ +# + +## targets + +default: dvi +dist: dvi -FILES = ref.tex introduction.tex goals.tex tactic.tex tctical.tex\ - thm.tex theories.tex defining.tex syntax.tex substitution.tex\ - simplifier.tex classical.tex theory-syntax.tex\ - ../rail.sty ../proof.sty ../iman.sty ../extra.sty +## dependencies + +include ../Makefile.in + +NAME = ref +FILES = ref.tex introduction.tex goals.tex tactic.tex tctical.tex \ + thm.tex theories.tex defining.tex syntax.tex substitution.tex \ + simplifier.tex classical.tex theory-syntax.tex \ + ../rail.sty ../proof.sty ../iman.sty ../extra.sty -ref.dvi.gz: $(FILES) - test -r isabelle.eps || ln -s ../gfx/isabelle.eps . - -rm ref.dvi* - latex ref - rail ref - bibtex ref - latex ref - latex ref - ../sedindex ref - latex ref - gzip -f ref.dvi +dvi: $(NAME).dvi -dist: $(FILES) - test -f isabelle.eps || ln -s ../gfx/isabelle.eps . - rm -f ref.dvi* - latex ref - latex ref - ../sedindex ref - latex ref - -clean: - @rm *.aux *.log *.toc *.idx *.rai +$(NAME).dvi: $(FILES) isabelle.eps + touch $(NAME).ind + $(LATEX) $(NAME) + $(RAIL) $(NAME) + $(BIBTEX) $(NAME) + $(LATEX) $(NAME) + $(LATEX) $(NAME) + $(SEDINDEX) $(NAME) + $(LATEX) $(NAME) diff -r dc5bf3f40ad3 -r 5a94bd71cc41 doc-src/Ref/ref.bbl --- a/doc-src/Ref/ref.bbl Wed May 05 18:26:10 1999 +0200 +++ /dev/null Thu Jan 01 00:00:00 1970 +0000 @@ -1,58 +0,0 @@ -\begin{thebibliography}{10} - -\bibitem{bm88book} -Robert~S. Boyer and J~Strother Moore. -\newblock {\em A Computational Logic Handbook}. -\newblock Academic Press, 1988. - -\bibitem{charniak80} -E.~Charniak, C.~K. Riesbeck, and D.~V. McDermott. -\newblock {\em Artificial Intelligence Programming}. -\newblock Lawrence Erlbaum Associates, 1980. - -\bibitem{debruijn72} -N.~G. de~Bruijn. -\newblock Lambda calculus notation with nameless dummies, a tool for automatic - formula manipulation, with application to the {Church-Rosser Theorem}. -\newblock {\em Indagationes Mathematicae}, 34:381--392, 1972. - -\bibitem{OBJ} -K.~Futatsugi, J.A. Goguen, Jean-Pierre Jouannaud, and J.~Meseguer. -\newblock Principles of {OBJ2}. -\newblock In {\em Symposium on Principles of Programming Languages}, pages - 52--66, 1985. - -\bibitem{martin-nipkow} -Ursula Martin and Tobias Nipkow. -\newblock Ordered rewriting and confluence. -\newblock In Mark~E. Stickel, editor, {\em 10th International Conference on - Automated Deduction}, LNAI 449, pages 366--380. Springer, 1990. - -\bibitem{nipkow-patterns} -Tobias Nipkow. -\newblock Functional unification of higher-order patterns. -\newblock In M.~Vardi, editor, {\em Eighth Annual Symposium on Logic in - Computer Science}, pages 64--74. {\sc ieee} Computer Society Press, 1993. - -\bibitem{nipkow-prehofer} -Tobias Nipkow and Christian Prehofer. -\newblock Type reconstruction for type classes. -\newblock {\em Journal of Functional Programming}, 5(2):201--224, 1995. - -\bibitem{nordstrom90} -Bengt {Nordstr\"om}, Kent Petersson, and Jan Smith. -\newblock {\em Programming in {Martin-L\"of}'s Type Theory. An Introduction}. -\newblock Oxford University Press, 1990. - -\bibitem{paulson-ml2} -Lawrence~C. Paulson. -\newblock {\em {ML} for the Working Programmer}. -\newblock Cambridge University Press, 2nd edition, 1996. - -\bibitem{pelletier86} -F.~J. Pelletier. -\newblock Seventy-five problems for testing automatic theorem provers. -\newblock {\em Journal of Automated Reasoning}, 2:191--216, 1986. -\newblock Errata, JAR 4 (1988), 235--236 and JAR 18 (1997), 135. - -\end{thebibliography} diff -r dc5bf3f40ad3 -r 5a94bd71cc41 doc-src/Ref/ref.ind --- a/doc-src/Ref/ref.ind Wed May 05 18:26:10 1999 +0200 +++ /dev/null Thu Jan 01 00:00:00 1970 +0000 @@ -1,904 +0,0 @@ -\begin{theindex} - - \item {\tt !!} symbol, 71 - \item {\tt\$}, \bold{62}, 88 - \item {\tt\%} symbol, 71 - \item * SplitterFun, 129 - \item {\tt ::} symbol, 71, 72 - \item {\tt ==} symbol, 71 - \item {\tt ==>} symbol, 71 - \item {\tt =>} symbol, 71 - \item {\tt =?=} symbol, 71 - \item {\tt\at Enum} constant, 94 - \item {\tt\at Finset} constant, 94, 95 - \item {\tt [} symbol, 71 - \item {\tt [|} symbol, 71 - \item {\tt \$ISABELLE_HOME}, 3 - \item {\tt ]} symbol, 71 - \item {\tt _K} constant, 96, 98 - \item \verb'{}' symbol, 94 - \item {\tt\ttlbrace} symbol, 71 - \item {\tt\ttrbrace} symbol, 71 - \item {\tt |]} symbol, 71 - - \indexspace - - \item {\tt Abs}, \bold{62}, 88 - \item {\tt abstract_over}, \bold{63} - \item {\tt abstract_rule}, \bold{49} - \item {\tt aconv}, \bold{63} - \item {\tt add_path}, \bold{60} - \item {\tt addaltern}, \bold{137} - \item {\tt addbefore}, \bold{137} - \item {\tt Addcongs}, \bold{107} - \item {\tt addcongs}, \bold{112}, 127, 128 - \item {\tt addD2}, \bold{136} - \item {\tt AddDs}, \bold{142} - \item {\tt addDs}, \bold{135} - \item {\tt addE2}, \bold{136} - \item {\tt addeqcongs}, \bold{112}, 128 - \item {\tt AddEs}, \bold{142} - \item {\tt addEs}, \bold{135} - \item {\tt AddIs}, \bold{142} - \item {\tt addIs}, \bold{135} - \item {\tt addloop}, \bold{114} - \item {\tt addSaltern}, \bold{137} - \item {\tt addSbefore}, \bold{137} - \item {\tt addSD2}, \bold{136} - \item {\tt AddSDs}, \bold{142} - \item {\tt addSDs}, \bold{135} - \item {\tt addSE2}, \bold{136} - \item {\tt AddSEs}, \bold{142} - \item {\tt addSEs}, \bold{135} - \item {\tt Addsimprocs}, \bold{107} - \item {\tt addsimprocs}, \bold{111} - \item {\tt Addsimps}, \bold{107} - \item {\tt addsimps}, \bold{110}, 128 - \item {\tt AddSIs}, \bold{142} - \item {\tt addSIs}, \bold{135} - \item {\tt addSolver}, \bold{113} - \item {\tt Addsplits}, \bold{107} - \item {\tt addsplits}, \bold{115} - \item {\tt addss}, \bold{137}, 138 - \item {\tt addSSolver}, \bold{113} - \item {\tt addSWrapper}, \bold{137} - \item {\tt addWrapper}, \bold{137} - \item {\tt all_tac}, \bold{34} - \item {\tt ALLGOALS}, \bold{38}, 119, 122 - \item ambiguity - \subitem of parsed expressions, 81 - \item {\tt ancestors_of}, \bold{61} - \item {\tt any} nonterminal, \bold{70} - \item {\tt APPEND}, \bold{32}, 34 - \item {\tt APPEND'}, 39 - \item {\tt Appl}, 85 - \item {\tt aprop} nonterminal, \bold{72} - \item {\tt ares_tac}, \bold{23} - \item {\tt args} nonterminal, 95 - \item {\tt Arith} theory, 121 - \item arities - \subitem context conditions, 58 - \item {\tt Asm_full_simp_tac}, \bold{106} - \item {\tt asm_full_simp_tac}, 26, \bold{116}, 120 - \item {\tt asm_full_simplify}, 116 - \item {\tt asm_rl} theorem, 25 - \item {\tt Asm_simp_tac}, \bold{105}, 118 - \item {\tt asm_simp_tac}, \bold{116}, 128 - \item {\tt asm_simplify}, 116 - \item associative-commutative operators, 121 - \item {\tt assume}, \bold{48} - \item {\tt assume_ax}, 10, \bold{12} - \item {\tt assume_tac}, \bold{21}, 134 - \item {\tt assumption}, \bold{51} - \item assumptions - \subitem contradictory, 142 - \subitem deleting, 26 - \subitem in simplification, 105, 114 - \subitem inserting, 23 - \subitem negated, 132 - \subitem of main goal, 9, 10, 12, 17, 18 - \subitem reordering, 120 - \subitem rotating, 26 - \subitem substitution in, 102 - \subitem tactics for, 21 - \item ASTs, 85--90 - \subitem made from parse trees, 86 - \subitem made from terms, 88 - \item {\tt atac}, \bold{23} - \item {\tt Auto_tac}, \bold{142} - \item {\tt auto_tac} $(cs,ss)$, \bold{139} - \item {\tt axclass} section, 57 - \item axiomatic type class, 57 - \item axioms - \subitem extracting, 11 - \item {\tt axioms_of}, \bold{11} - - \indexspace - - \item {\tt ba}, \bold{14} - \item {\tt back}, \bold{13} - \item batch execution, 16 - \item {\tt bd}, \bold{14} - \item {\tt bds}, \bold{14} - \item {\tt be}, \bold{14} - \item {\tt bes}, \bold{14} - \item {\tt BEST_FIRST}, \bold{35}, 36 - \item {\tt Best_tac}, \bold{142} - \item {\tt best_tac}, \bold{140} - \item {\tt beta_conversion}, \bold{49} - \item {\tt bicompose}, \bold{52} - \item {\tt bimatch_tac}, \bold{27} - \item {\tt bind_thm}, \bold{11}, 12, 42 - \item binders, \bold{80} - \item {\tt biresolution}, \bold{51} - \item {\tt biresolve_tac}, \bold{27}, 143 - \item {\tt Blast.depth_tac}, \bold{139} - \item {\tt Blast.trace}, \bold{139} - \item {\tt Blast_tac}, \bold{142} - \item {\tt blast_tac}, \bold{138} - \item {\tt Bound}, \bold{62}, 86, 88, 89 - \item {\tt bound_hyp_subst_tac}, \bold{102} - \item {\tt br}, \bold{14} - \item {\tt BREADTH_FIRST}, \bold{35} - \item {\tt brs}, \bold{14} - \item {\tt bw}, \bold{15} - \item {\tt bws}, \bold{15} - \item {\tt by}, \bold{9}, 12--14, 18 - \item {\tt byev}, \bold{10} - - \indexspace - - \item {\tt cd}, \bold{3} - \item {\tt cert_axm}, \bold{64} - \item {\tt CHANGED}, \bold{34} - \item {\tt chop}, \bold{12}, 17 - \item {\tt choplev}, \bold{13} - \item {\tt Clarify_step_tac}, \bold{142} - \item {\tt clarify_step_tac}, \bold{139} - \item {\tt Clarify_tac}, \bold{142} - \item {\tt clarify_tac}, \bold{139} - \item {\tt Clarsimp_tac}, \bold{142} - \item {\tt clarsimp_tac}, \bold{140} - \item claset - \subitem current, 141 - \item {\tt claset} ML type, 135 - \item {\tt ClasimpFun}, 144 - \item classes - \subitem context conditions, 58 - \item classical reasoner, 130--144 - \subitem setting up, 143 - \subitem tactics, 138 - \item classical sets, 134 - \item {\tt ClassicalFun}, 143 - \item {\tt combination}, \bold{49} - \item {\tt commit}, \bold{3} - \item {\tt COMP}, \bold{51} - \item {\tt compose}, \bold{51} - \item {\tt compose_tac}, \bold{27} - \item {\tt concl_of}, \bold{45} - \item {\tt COND}, \bold{36} - \item congruence rules, 111 - \item {\tt Const}, \bold{62}, 88, 98 - \item {\tt Constant}, 85, 98 - \item constants, \bold{62} - \subitem for translations, 75 - \subitem syntactic, 90 - \item {\tt context}, \bold{4}, 105 - \item {\tt contr_tac}, \bold{142} - \item {\tt could_unify}, \bold{29} - \item {\tt cprems_of}, \bold{45} - \item {\tt cprop_of}, \bold{44} - \item {\tt CPure} theory, 55 - \item {\tt CPure.thy}, \bold{61} - \item {\tt crep_thm}, \bold{45} - \item {\tt cterm} ML type, 64 - \item {\tt cterm_instantiate}, \bold{43} - \item {\tt cterm_of}, 9, 17, \bold{64} - \item {\tt ctyp}, \bold{65} - \item {\tt ctyp_of}, \bold{66} - \item {\tt cut_facts_tac}, \bold{23}, 103 - \item {\tt cut_inst_tac}, \bold{23} - \item {\tt cut_rl} theorem, 25 - - \indexspace - - \item {\tt datatype}, 107 - \item {\tt Deepen_tac}, \bold{142} - \item {\tt deepen_tac}, \bold{140} - \item {\tt defer_tac}, \bold{24} - \item definitions, \see{rewriting, meta-level}{1}, 24, \bold{58} - \subitem unfolding, 9, 10 - \item {\tt del_path}, \bold{60} - \item {\tt Delcongs}, \bold{107} - \item {\tt delcongs}, \bold{112} - \item {\tt deleqcongs}, \bold{112} - \item {\tt delete_tmpfiles}, \bold{59} - \item delimiters, \bold{72}, 75, 76, 78 - \item {\tt delloop}, \bold{114} - \item {\tt delrules}, \bold{135} - \item {\tt Delsimprocs}, \bold{107} - \item {\tt delsimprocs}, \bold{111} - \item {\tt Delsimps}, \bold{107} - \item {\tt delsimps}, \bold{110} - \item {\tt Delsplits}, \bold{107} - \item {\tt delSWrapper}, \bold{137} - \item {\tt delWrapper}, \bold{137} - \item {\tt dependent_tr'}, 96, \bold{98} - \item {\tt DEPTH_FIRST}, \bold{35} - \item {\tt DEPTH_SOLVE}, \bold{35} - \item {\tt DEPTH_SOLVE_1}, \bold{35} - \item {\tt depth_tac}, \bold{140} - \item {\tt Deriv.drop}, \bold{53} - \item {\tt Deriv.linear}, \bold{53} - \item {\tt Deriv.size}, \bold{53} - \item {\tt Deriv.tree}, \bold{53} - \item {\tt dest_eq}, \bold{103} - \item {\tt dest_imp}, \bold{103} - \item {\tt dest_state}, \bold{45} - \item {\tt dest_Trueprop}, \bold{103} - \item destruct-resolution, 21 - \item {\tt DETERM}, \bold{36} - \item discrimination nets, \bold{28} - \item {\tt distinct_subgoals_tac}, \bold{26} - \item {\tt dmatch_tac}, \bold{21} - \item {\tt domain_type}, \bold{104} - \item {\tt dres_inst_tac}, \bold{22} - \item {\tt dresolve_tac}, \bold{21} - \item {\tt dtac}, \bold{23} - \item {\tt dummyT}, 88, 89, 99 - \item duplicate subgoals - \subitem removing, 26 - - \indexspace - - \item elim-resolution, 20 - \item {\tt ematch_tac}, \bold{21} - \item {\tt empty} constant, 94 - \item {\tt empty_cs}, \bold{135} - \item {\tt empty_ss}, \bold{109} - \item {\tt eq_assume_tac}, \bold{21}, 134 - \item {\tt eq_assumption}, \bold{51} - \item {\tt eq_mp_tac}, \bold{142} - \item {\tt eq_reflection} theorem, \bold{104}, 125 - \item {\tt eq_thm}, \bold{36} - \item {\tt eq_thy}, \bold{60} - \item {\tt equal_elim}, \bold{48} - \item {\tt equal_intr}, \bold{48} - \item equality, 101--104 - \item {\tt eres_inst_tac}, \bold{22} - \item {\tt eresolve_tac}, \bold{20} - \subitem on other than first premise, 44 - \item {\tt ERROR}, 6 - \item {\tt error}, 6 - \item error messages, 6 - \item {\tt eta_contract}, \bold{6}, 92 - \item {\tt etac}, \bold{23} - \item {\tt EVERY}, \bold{33} - \item {\tt EVERY'}, 39 - \item {\tt EVERY1}, \bold{40} - \item examples - \subitem of logic definitions, 82 - \subitem of macros, 94, 95 - \subitem of mixfix declarations, 77 - \subitem of simplification, 117 - \subitem of translations, 98 - \item exceptions - \subitem printing of, 7 - \item {\tt exit}, \bold{3} - \item {\tt extensional}, \bold{49} - - \indexspace - - \item {\tt fa}, \bold{15} - \item {\tt Fast_tac}, \bold{142} - \item {\tt fast_tac}, \bold{140} - \item {\tt fd}, \bold{15} - \item {\tt fds}, \bold{15} - \item {\tt fe}, \bold{15} - \item {\tt fes}, \bold{15} - \item files - \subitem reading, 3, 59 - \item {\tt filt_resolve_tac}, \bold{29} - \item {\tt FILTER}, \bold{34} - \item {\tt filter_goal}, \bold{19} - \item {\tt filter_thms}, \bold{29} - \item {\tt findE}, \bold{12} - \item {\tt findEs}, \bold{12} - \item {\tt findI}, \bold{12} - \item {\tt FIRST}, \bold{33} - \item {\tt FIRST'}, 39 - \item {\tt FIRST1}, \bold{40} - \item {\tt FIRSTGOAL}, \bold{38} - \item flex-flex constraints, 26, 44, 52 - \item {\tt flexflex_rule}, \bold{52} - \item {\tt flexflex_tac}, \bold{26} - \item {\tt FOL_basic_ss}, \bold{128} - \item {\tt FOL_ss}, \bold{128} - \item {\tt fold_goals_tac}, \bold{24} - \item {\tt fold_tac}, \bold{24} - \item {\tt forall_elim}, \bold{50} - \item {\tt forall_elim_list}, \bold{50} - \item {\tt forall_elim_var}, \bold{50} - \item {\tt forall_elim_vars}, \bold{50} - \item {\tt forall_intr}, \bold{49} - \item {\tt forall_intr_frees}, \bold{50} - \item {\tt forall_intr_list}, \bold{50} - \item {\tt force_strip_shyps}, \bold{45} - \item {\tt Force_tac}, \bold{142} - \item {\tt force_tac}, \bold{139} - \item {\tt forw_inst_tac}, \bold{22} - \item forward proof, 21, 42 - \item {\tt forward_tac}, \bold{21} - \item {\tt fr}, \bold{15} - \item {\tt Free}, \bold{62}, 88 - \item {\tt freezeT}, \bold{50} - \item {\tt frs}, \bold{15} - \item {\tt Full_simp_tac}, \bold{105} - \item {\tt full_simp_tac}, \bold{116} - \item {\tt full_simplify}, 116 - \item {\textit {fun}} type, 65 - \item function applications, \bold{62} - - \indexspace - - \item {\tt get_axiom}, \bold{11} - \item {\tt get_thm}, \bold{11} - \item {\tt get_thms}, \bold{11} - \item {\tt getenv}, 59 - \item {\tt getgoal}, \bold{18} - \item {\tt gethyps}, \bold{19}, 38 - \item {\tt Goal}, \bold{9}, 17 - \item {\tt goal}, \bold{9} - \item {\tt goals_limit}, \bold{13} - \item {\tt Goalw}, \bold{9} - \item {\tt goalw}, \bold{9} - \item {\tt goalw_cterm}, \bold{9} - - \indexspace - - \item {\tt has_fewer_prems}, \bold{36} - \item higher-order pattern, \bold{110} - \item {\tt HOL_basic_ss}, \bold{109} - \item {\tt hyp_subst_tac}, \bold{102} - \item {\tt hyp_subst_tacs}, \bold{144} - \item {\tt HypsubstFun}, 103, 144 - - \indexspace - - \item {\tt id} nonterminal, \bold{72}, 86, 93 - \item identifiers, 72 - \item {\tt idt} nonterminal, 92 - \item {\tt idts} nonterminal, \bold{72}, 80 - \item {\tt IF_UNSOLVED}, \bold{36} - \item {\tt iff_reflection} theorem, 125 - \item {\tt IFOL_ss}, \bold{128} - \item {\tt imp_intr} theorem, \bold{104} - \item {\tt implies_elim}, \bold{48} - \item {\tt implies_elim_list}, \bold{48} - \item {\tt implies_intr}, \bold{48} - \item {\tt implies_intr_hyps}, \bold{48} - \item {\tt implies_intr_list}, \bold{48} - \item {\tt incr_boundvars}, \bold{63}, 98 - \item {\tt indexname} ML type, 62, 73 - \item infixes, \bold{79} - \item {\tt insert} constant, 94 - \item {\tt inst_step_tac}, \bold{141} - \item {\tt instance} section, 57 - \item {\tt instantiate}, \bold{50} - \item {\tt instantiate'}, \bold{43}, 50 - \item instantiation, 22, 43, 50 - \item {\tt INTLEAVE}, \bold{32}, 34 - \item {\tt INTLEAVE'}, 39 - \item {\tt invoke_oracle}, \bold{66} - \item {\tt is} nonterminal, 94 - - \indexspace - - \item {\tt joinrules}, \bold{143} - - \indexspace - - \item {\tt keep_derivs}, \bold{53} - - \indexspace - - \item $\lambda$-abstractions, 28, \bold{62} - \item $\lambda$-calculus, 47, 49, 72 - \item {\tt lessb}, \bold{28} - \item lexer, \bold{72} - \item {\tt lift_rule}, \bold{52} - \item lifting, 52 - \item {\tt logic} class, 72, 77 - \item {\tt logic} nonterminal, \bold{72} - \item {\tt Logic.auto_rename}, \bold{26} - \item {\tt Logic.set_rename_prefix}, \bold{25} - \item {\tt long_names}, \bold{6} - \item {\tt loose_bnos}, \bold{63}, 99 - - \indexspace - - \item macros, 90--96 - \item {\tt make_elim}, \bold{44}, 136 - \item {\tt Match} exception, 97 - \item {\tt match_tac}, \bold{21}, 134 - \item {\tt max_pri}, 70, \bold{76} - \item {\tt merge_ss}, \bold{109} - \item meta-assumptions, 37, 46, 48, 51 - \subitem printing of, 5 - \item meta-equality, 47--49 - \item meta-implication, 47, 48 - \item meta-quantifiers, 47, 49 - \item meta-rewriting, 9, 15, 16, \bold{24}, - \seealso{tactics, theorems}{145} - \subitem in theorems, 43 - \item meta-rules, \see{meta-rules}{1}, 46--52 - \item {\tt METAHYPS}, 19, \bold{37} - \item mixfix declarations, 57, 75--80 - \item {\tt mk_atomize}, \bold{127} - \item {\tt mk_simproc}, \bold{123} - \item {\tt ML} section, 58, 97, 99 - \item model checkers, 81 - \item {\tt mp} theorem, \bold{143} - \item {\tt mp_tac}, \bold{142} - \item {\tt MRL}, \bold{42} - \item {\tt MRS}, \bold{42} - - \indexspace - - \item name tokens, \bold{72} - \item {\tt nat_cancel}, \bold{111} - \item {\tt net_bimatch_tac}, \bold{28} - \item {\tt net_biresolve_tac}, \bold{28} - \item {\tt net_match_tac}, \bold{28} - \item {\tt net_resolve_tac}, \bold{28} - \item {\tt no_tac}, \bold{34} - \item {\tt None}, \bold{30} - \item {\tt nonterminal} symbols, 56 - \item {\tt not_elim} theorem, \bold{143} - \item {\tt nprems_of}, \bold{45} - \item numerals, 72 - - \indexspace - - \item {\textit {o}} type, 82 - \item {\tt object}, 66 - \item {\tt op} symbol, 79 - \item {\tt option} ML type, 30 - \item oracles, 66--68 - \item {\tt ORELSE}, \bold{32}, 34, 38 - \item {\tt ORELSE'}, 39 - - \indexspace - - \item parameters - \subitem removing unused, 26 - \subitem renaming, 15, 25, 52 - \item {\tt parents_of}, \bold{61} - \item parse trees, 85 - \item {\tt parse_rules}, 92 - \item pattern, higher-order, \bold{110} - \item {\tt pause_tac}, \bold{30} - \item Poly/{\ML} compiler, 7 - \item {\tt pop_proof}, \bold{17} - \item {\tt pr}, \bold{13} - \item {\tt premises}, \bold{9}, 17 - \item {\tt prems_of}, \bold{45} - \item {\tt prems_of_ss}, \bold{113} - \item pretty printing, 76, 78--79, 95 - \item {\tt Pretty.setdepth}, \bold{5} - \item {\tt Pretty.setmargin}, \bold{5} - \item {\tt PRIMITIVE}, \bold{29} - \item {\tt primrec}, 107 - \item {\tt prin}, 7, \bold{18} - \item print mode, 56, 99 - \item print modes, 80--81 - \item {\tt print_cs}, \bold{135} - \item {\tt print_depth}, \bold{5} - \item {\tt print_exn}, \bold{7}, 41 - \item {\tt print_goals}, \bold{42} - \item {\tt print_mode}, 80 - \item {\tt print_modes}, 75 - \item {\tt print_rules}, 92 - \item {\tt print_simpset}, \bold{109} - \item {\tt print_ss}, \bold{108} - \item {\tt print_syntax}, \bold{61}, \bold{74} - \item {\tt print_tac}, \bold{30} - \item {\tt print_theory}, \bold{61} - \item {\tt print_thm}, \bold{42} - \item printing control, 4--6 - \item {\tt printyp}, \bold{18} - \item priorities, 69, \bold{76} - \item priority grammars, 69--70 - \item {\tt prlev}, \bold{13} - \item {\tt prlim}, \bold{13} - \item productions, 69, 75, 76 - \subitem copy, \bold{75}, 76, 87 - \item {\tt proof} ML type, 18 - \item proof objects, 52--54 - \item proof state, 8 - \subitem printing of, 13 - \item {\tt proof_timing}, \bold{14} - \item proofs, 8--19 - \subitem inspecting the state, 18 - \subitem managing multiple, 17 - \subitem saving and restoring, 18 - \subitem stacking, 17 - \subitem starting, 8 - \subitem timing, 14 - \item {\tt PROP} symbol, 71 - \item {\textit {prop}} type, 65, 72 - \item {\tt prop} nonterminal, \bold{70}, 82 - \item {\tt ProtoPure.thy}, \bold{61} - \item {\tt prove_goal}, 14, \bold{16} - \item {\tt prove_goalw}, \bold{16} - \item {\tt prove_goalw_cterm}, \bold{16} - \item {\tt prth}, \bold{41} - \item {\tt prthq}, \bold{42} - \item {\tt prths}, \bold{42} - \item {\tt prune_params_tac}, \bold{26} - \item {\tt pttrn} nonterminal, \bold{72} - \item {\tt pttrns} nonterminal, \bold{72} - \item {\tt Pure} theory, 55, 70, 74 - \item {\tt Pure.thy}, \bold{61} - \item {\tt push_proof}, \bold{17} - \item {\tt pwd}, \bold{3} - - \indexspace - - \item {\tt qed}, \bold{10}, 12 - \item {\tt qed_goal}, \bold{16} - \item {\tt qed_goalw}, \bold{16} - \item quantifiers, 80 - \item {\tt quit}, \bold{3} - - \indexspace - - \item {\tt read}, \bold{18} - \item {\tt read_axm}, \bold{64} - \item {\tt read_cterm}, \bold{64} - \item {\tt read_instantiate}, \bold{43} - \item {\tt read_instantiate_sg}, \bold{43} - \item reading - \subitem axioms, \see{{\tt assume_ax}}{55} - \subitem goals, \see{proofs, starting}{8} - \item {\tt reflexive}, \bold{49} - \item {\tt ren}, \bold{15} - \item {\tt rename_last_tac}, \bold{25} - \item {\tt rename_params_rule}, \bold{52} - \item {\tt rename_tac}, \bold{25} - \item {\tt rep_cs}, \bold{135} - \item {\tt rep_cterm}, \bold{64} - \item {\tt rep_ctyp}, \bold{66} - \item {\tt rep_ss}, \bold{108} - \item {\tt rep_thm}, \bold{45} - \item {\tt REPEAT}, \bold{33, 34} - \item {\tt REPEAT1}, \bold{33} - \item {\tt REPEAT_DETERM}, \bold{33} - \item {\tt REPEAT_FIRST}, \bold{39} - \item {\tt REPEAT_SOME}, \bold{38} - \item {\tt res_inst_tac}, \bold{22}, 26, 27 - \item reserved words, 72, 95 - \item {\tt reset}, 4 - \item {\tt reset_path}, \bold{60} - \item resolution, 42, 51 - \subitem tactics, 20 - \subitem without lifting, 51 - \item {\tt resolve_tac}, \bold{20}, 134 - \item {\tt restore_proof}, \bold{18} - \item {\tt result}, \bold{10}, 12, 18 - \item {\tt rev_mp} theorem, \bold{104} - \item rewrite rules, 110 - \subitem permutative, 120--123 - \item {\tt rewrite_goals_rule}, \bold{43} - \item {\tt rewrite_goals_tac}, \bold{24}, 43 - \item {\tt rewrite_rule}, \bold{43} - \item {\tt rewrite_tac}, 10, \bold{24} - \item rewriting - \subitem object-level, \see{simplification}{1} - \subitem ordered, 121 - \subitem syntactic, 90--96 - \item {\tt rewtac}, \bold{23} - \item {\tt RL}, \bold{42} - \item {\tt RLN}, \bold{42} - \item {\tt rotate_prems}, \bold{44} - \item {\tt rotate_proof}, \bold{17} - \item {\tt rotate_tac}, \bold{26} - \item {\tt RS}, \bold{42} - \item {\tt RSN}, \bold{42} - \item {\tt rtac}, \bold{23} - \item {\tt rule_by_tactic}, 26, \bold{44} - \item rules - \subitem converting destruction to elimination, 44 - - \indexspace - - \item {\tt safe_asm_full_simp_tac}, \bold{116} - \item {\tt Safe_step_tac}, \bold{142} - \item {\tt safe_step_tac}, 136, \bold{141} - \item {\tt Safe_tac}, \bold{142} - \item {\tt safe_tac}, \bold{141} - \item {\tt save_proof}, \bold{18} - \item saving your session, \bold{2} - \item search, 32 - \subitem tacticals, 34--36 - \item {\tt SELECT_GOAL}, 24, \bold{37} - \item {\tt Seq.seq} ML type, 29 - \item sequences (lazy lists), \bold{30} - \item sequent calculus, 131 - \item sessions, 1--7 - \item {\tt set}, 4 - \item {\tt setloop}, \bold{114} - \item {\tt setmksimps}, 110, \bold{126}, 128 - \item {\tt setSolver}, \bold{113}, 128 - \item {\tt setSSolver}, \bold{113}, 128 - \item {\tt setsubgoaler}, \bold{112}, 128 - \item {\tt settermless}, \bold{121} - \item {\tt setup} - \subitem simplifier, 129 - \subitem theory, 58 - \item shortcuts - \subitem for \texttt{by} commands, 14 - \subitem for tactics, 23 - \item {\tt show_brackets}, \bold{5} - \item {\tt show_consts}, \bold{6} - \item {\tt show_hyps}, \bold{5} - \item {\tt show_path}, \bold{60} - \item {\tt show_sorts}, \bold{5}, 89, 97 - \item {\tt show_tags}, \bold{5} - \item {\tt show_types}, \bold{5}, 89, 92, 99 - \item {\tt Sign.certify_term}, \bold{64} - \item {\tt Sign.certify_typ}, \bold{66} - \item {\tt Sign.sg} ML type, 55 - \item {\tt Sign.stamp_names_of}, \bold{61} - \item {\tt Sign.string_of_term}, \bold{64} - \item {\tt Sign.string_of_typ}, \bold{65} - \item {\tt sign_of}, 9, 17, \bold{61} - \item {\tt sign_of_thm}, \bold{45} - \item signatures, \bold{55}, 61, 63, 64, 66 - \item {\tt Simp_tac}, \bold{105} - \item {\tt simp_tac}, \bold{116} - \item simplification, 105--129 - \subitem conversions, 116 - \subitem forward rules, 116 - \subitem from classical reasoner, 137 - \subitem setting up, 125 - \subitem setting up the splitter, 129 - \subitem setting up the theory, 129 - \subitem tactics, 115 - \item simplification sets, 108 - \item {\tt Simplifier.asm_full_rewrite}, 116 - \item {\tt Simplifier.asm_rewrite}, 116 - \item {\tt Simplifier.full_rewrite}, 116 - \item {\tt Simplifier.rewrite}, 116 - \item {\tt Simplifier.setup}, \bold{129} - \item {\tt simplify}, 116 - \item {\tt SIMPSET}, \bold{109} - \item simpset - \subitem current, 105, 109 - \item {\tt simpset}, \bold{109} - \item {\tt SIMPSET'}, \bold{109} - \item {\tt simpset_of}, \bold{109} - \item {\tt simpset_ref}, \bold{109} - \item {\tt simpset_ref_of}, \bold{109} - \item {\tt size_of_thm}, 35, \bold{36}, 143 - \item {\tt sizef}, \bold{143} - \item {\tt slow_best_tac}, \bold{140} - \item {\tt slow_step_tac}, 136, \bold{141} - \item {\tt slow_tac}, \bold{140} - \item {\tt SOLVE}, \bold{36} - \item {\tt Some}, \bold{30} - \item {\tt SOMEGOAL}, \bold{38} - \item {\tt sort} nonterminal, \bold{72} - \item sort constraints, 71 - \item sort hypotheses, 45, 47 - \item sorts - \subitem printing of, 5 - \item {\tt ssubst} theorem, \bold{101} - \item {\tt stac}, \bold{102} - \item stamps, \bold{55}, 61 - \item {\tt standard}, \bold{44} - \item starting up, \bold{1} - \item {\tt Step_tac}, \bold{142} - \item {\tt step_tac}, 136, \bold{141} - \item {\tt store_thm}, \bold{11} - \item {\tt string_of_cterm}, \bold{64} - \item {\tt string_of_ctyp}, \bold{65} - \item {\tt string_of_thm}, \bold{42} - \item strings, 72 - \item {\tt SUBGOAL}, \bold{29} - \item subgoal module, 8--19 - \item {\tt subgoal_tac}, \bold{23} - \item {\tt subgoals_of_brl}, \bold{27} - \item {\tt subgoals_tac}, \bold{24} - \item {\tt subst} theorem, 101, \bold{104} - \item substitution - \subitem rules, 101 - \item {\tt subthy}, \bold{60} - \item {\tt swap} theorem, \bold{143} - \item {\tt swap_res_tac}, \bold{143} - \item {\tt swapify}, \bold{143} - \item {\tt sym} theorem, 102, \bold{104} - \item {\tt symmetric}, \bold{49} - \item {\tt syn_of}, \bold{74} - \item syntax - \subitem Pure, 70--75 - \subitem transformations, 85--99 - \item {\tt syntax} section, 56 - \item {\tt Syntax.ast} ML type, 85 - \item {\tt Syntax.mark_boundT}, 99 - \item {\tt Syntax.print_gram}, \bold{74} - \item {\tt Syntax.print_syntax}, \bold{74} - \item {\tt Syntax.print_trans}, \bold{74} - \item {\tt Syntax.stat_norm_ast}, 94 - \item {\tt Syntax.syntax} ML type, 74 - \item {\tt Syntax.test_read}, 78, 94 - \item {\tt Syntax.trace_norm_ast}, 94 - \item {\tt Syntax.variant_abs'}, 99 - - \indexspace - - \item {\tt tactic} ML type, 20 - \item tacticals, 32--40 - \subitem conditional, 36 - \subitem deterministic, 36 - \subitem for filtering, 34 - \subitem for restriction to a subgoal, 37 - \subitem identities for, 33 - \subitem joining a list of tactics, 33 - \subitem joining tactic functions, 39 - \subitem joining two tactics, 32 - \subitem repetition, 33 - \subitem scanning for subgoals, 38 - \subitem searching, 35 - \item tactics, 20--31 - \subitem assumption, \bold{21}, 23 - \subitem commands for applying, 9 - \subitem debugging, 18 - \subitem filtering results of, 34 - \subitem for composition, 27 - \subitem for contradiction, 142 - \subitem for inserting facts, 23 - \subitem for Modus Ponens, 142 - \subitem instantiation, 22 - \subitem matching, 21 - \subitem meta-rewriting, 23, \bold{24} - \subitem primitives for coding, 29 - \subitem resolution, \bold{20}, 23, 27, 28 - \subitem restricting to a subgoal, 37 - \subitem simplification, 115 - \subitem substitution, 101--104 - \subitem tracing, 30 - \item {\tt TERM}, 64 - \item {\tt term} ML type, 62, 88 - \item terms, \bold{62} - \subitem certified, \bold{63} - \subitem made from ASTs, 88 - \subitem printing of, 18, 64 - \subitem reading of, 18 - \item {\tt TFree}, \bold{65} - \item {\tt the_context}, \bold{4} - \item {\tt THEN}, \bold{32}, 34, 38 - \item {\tt THEN'}, 39 - \item {\tt THEN_BEST_FIRST}, \bold{35} - \item theorems, 41--54 - \subitem equality of, 36 - \subitem extracting, 11 - \subitem extracting proved, 10 - \subitem joining by resolution, 42 - \subitem of pure theory, 25 - \subitem printing of, 41 - \subitem retrieving, 12 - \subitem size of, 36 - \subitem standardizing, 44 - \subitem storing, 11 - \subitem taking apart, 44 - \item theories, 55--68 - \subitem axioms of, 11 - \subitem inspecting, \bold{61} - \subitem parent, \bold{55} - \subitem reading, 3, 59 - \subitem theorems of, 11 - \item {\tt THEORY} exception, 11, 55 - \item {\tt theory}, \bold{4} - \item {\tt theory} ML type, 55 - \item {\tt Theory.add_oracle}, \bold{66} - \item {\tt theory_of_thm}, \bold{45} - \item {\tt thin_refl} theorem, \bold{104} - \item {\tt thin_tac}, \bold{26} - \item {\tt THM} exception, 41, 42, 46, 51 - \item {\tt thm}, \bold{11} - \item {\tt thm} ML type, 41 - \item {\tt thms}, \bold{11} - \item {\tt thms_containing}, \bold{12} - \item {\tt thms_of}, \bold{11} - \item {\tt tid} nonterminal, \bold{72}, 86, 93 - \item {\tt time_use}, \bold{3} - \item {\tt time_use_thy}, \bold{4} - \item timing statistics, 14 - \item {\tt toggle}, 4 - \item token class, 99 - \item token translations, 99--100 - \item token_translation, 100 - \item {\tt token_translation}, 100 - \item {\tt topthm}, \bold{18} - \item {\tt touch_thy}, \bold{59} - \item {\tt tpairs_of}, \bold{45} - \item {\tt trace_BEST_FIRST}, \bold{35} - \item {\tt trace_DEPTH_FIRST}, \bold{35} - \item {\tt trace_goalno_tac}, \bold{39} - \item {\tt trace_REPEAT}, \bold{33} - \item {\tt trace_simp}, \bold{106}, 118 - \item tracing - \subitem of classical prover, 139 - \subitem of macros, 94 - \subitem of searching tacticals, 35 - \subitem of simplification, 107, 118--119 - \subitem of tactics, 30 - \subitem of unification, 46 - \item {\tt transfer}, \bold{60} - \item {\tt transfer_sg}, \bold{61} - \item {\tt transitive}, \bold{49} - \item translations, 96--99 - \subitem parse, 80, 88 - \subitem parse AST, \bold{86}, 87 - \subitem print, 80 - \subitem print AST, \bold{89} - \item {\tt translations} section, 91 - \item {\tt trivial}, \bold{52} - \item {\tt Trueprop} constant, 82 - \item {\tt TRY}, \bold{33, 34} - \item {\tt TRYALL}, \bold{38} - \item {\tt TVar}, \bold{65} - \item {\tt tvar} nonterminal, \bold{72, 73}, 86, 93 - \item {\tt typ} ML type, 65 - \item {\tt Type}, \bold{65} - \item {\textit {type}} type, 77 - \item {\tt type} nonterminal, \bold{72} - \item type constraints, 72, 80, 89 - \item type constructors, \bold{65} - \item type identifiers, 72 - \item type synonyms, \bold{56} - \item type unknowns, \bold{65}, 72 - \subitem freezing/thawing of, 50 - \item type variables, \bold{65} - \item types, \bold{65} - \subitem certified, \bold{65} - \subitem printing of, 5, 18, 65 - - \indexspace - - \item {\tt undo}, 8, \bold{13}, 17 - \item unknowns, \bold{62}, 72 - \item {\tt update_thy}, \bold{59} - \item {\tt uresult}, \bold{10}, 12, 18 - \item {\tt use}, \bold{3} - \item {\tt use_thy}, \bold{4} - \item {\tt use_thy_only}, \bold{59} - - \indexspace - - \item {\tt Var}, \bold{62}, 88 - \item {\tt var} nonterminal, \bold{72, 73}, 86, 93 - \item {\tt Variable}, 85 - \item variables - \subitem bound, \bold{62} - \subitem free, \bold{62} - \item {\tt variant_abs}, \bold{63} - \item {\tt varifyT}, \bold{50} - - \indexspace - - \item {\tt warning}, 6 - \item warnings, 6 - \item {\tt writeln}, 6 - - \indexspace - - \item {\tt xnum} nonterminal, \bold{72}, 86, 93 - \item {\tt xstr} nonterminal, \bold{72}, 86, 93 - - \indexspace - - \item {\tt zero_var_indexes}, \bold{44} - -\end{theindex} diff -r dc5bf3f40ad3 -r 5a94bd71cc41 doc-src/Ref/ref.rao --- a/doc-src/Ref/ref.rao Wed May 05 18:26:10 1999 +0200 +++ /dev/null Thu Jan 01 00:00:00 1970 +0000 @@ -1,449 +0,0 @@ -% This file was generated by 'rail' from 'ref.rai' -\rail@t {lbrace} -\rail@t {rbrace} -\rail@i {1}{ \par theoryDef : id '=' (name + '+') ('+' extension | ()) ; \par name : id | string ; \par extension : (section +) 'end' ( () | ml ) ; \par section : classes | default | types | arities | nonterminals | consts | syntax | trans | defs | constdefs | rules | axclass | instance | oracle | local | global | setup ; \par classes : 'classes' ( classDecl + ) ; \par classDecl : (id (() | '<' (id + ','))) ; \par default : 'default' sort ; \par sort : id | lbrace (id * ',') rbrace ; \par types : 'types' ( ( typeDecl ( () | '(' infix ')' ) ) + ) ; \par infix : ( 'infixr' | 'infixl' ) (() | string) nat ; \par typeDecl : typevarlist name ( () | '=' ( string | type ) ); \par typevarlist : () | tid | '(' ( tid + ',' ) ')'; \par type : simpleType | '(' type ')' | type '=>' type | '[' ( type + "," ) ']' '=>' type; \par simpleType: id | ( tid ( () | '::' id ) ) | '(' ( type + "," ) ')' id | simpleType id ; \par arities : 'arities' ((name + ',') '::' arity +) ; \par arity : ( () | '(' (sort + ',') ')' ) sort ; \par nonterminals : 'nonterminals' (name+) ; \par consts : 'consts' ( mixfixConstDecl + ) ; \par syntax : 'syntax' (() | mode) ( mixfixConstDecl + ); \par mode : '(' name (() | 'output') ')' ; \par mixfixConstDecl : constDecl (() | ( '(' mixfix ')' )) ; \par constDecl : ( name + ',') '::' (string | type); \par mixfix : string ( () | ( () | ('[' (nat + ',') ']')) nat ) | infix | 'binder' string nat ; \par trans : 'translations' ( pat ( '==' | '=>' | '<=' ) pat + ) ; \par pat : ( () | ( '(' id ')' ) ) string; \par rules : 'rules' (( id string ) + ) ; \par defs : 'defs' (( id string ) + ) ; \par constdefs : 'constdefs' (name '::' (string | type) (() | mixfix) string +) ; \par axclass : 'axclass' classDecl (() | ( id string ) +) ; \par instance : 'instance' ( name '<' name | name '::' arity) witness ; \par witness : (() | '(' ((string | id | longident) + ',') ')') (() | verbatim) ; \par oracle : 'oracle' name '=' name ; \par local : 'local' ; \par global : 'global' ; \par setup : 'setup' (id | longident) ; \par ml : 'ML' text ; \par } -\rail@o {1}{ -\rail@begin{2}{theoryDef} -\rail@nont{id}[] -\rail@term{=}[] -\rail@plus -\rail@nont{name}[] -\rail@nextplus{1} -\rail@cterm{+}[] -\rail@endplus -\rail@bar -\rail@term{+}[] -\rail@nont{extension}[] -\rail@nextbar{1} -\rail@endbar -\rail@end -\rail@begin{2}{name} -\rail@bar -\rail@nont{id}[] -\rail@nextbar{1} -\rail@nont{string}[] -\rail@endbar -\rail@end -\rail@begin{2}{extension} -\rail@plus -\rail@nont{section}[] -\rail@nextplus{1} -\rail@endplus -\rail@term{end}[] -\rail@bar -\rail@nextbar{1} -\rail@nont{ml}[] -\rail@endbar -\rail@end -\rail@begin{17}{section} -\rail@bar -\rail@nont{classes}[] -\rail@nextbar{1} -\rail@nont{default}[] -\rail@nextbar{2} -\rail@nont{types}[] -\rail@nextbar{3} -\rail@nont{arities}[] -\rail@nextbar{4} -\rail@nont{nonterminals}[] -\rail@nextbar{5} -\rail@nont{consts}[] -\rail@nextbar{6} -\rail@nont{syntax}[] -\rail@nextbar{7} -\rail@nont{trans}[] -\rail@nextbar{8} -\rail@nont{defs}[] -\rail@nextbar{9} -\rail@nont{constdefs}[] -\rail@nextbar{10} -\rail@nont{rules}[] -\rail@nextbar{11} -\rail@nont{axclass}[] -\rail@nextbar{12} -\rail@nont{instance}[] -\rail@nextbar{13} -\rail@nont{oracle}[] -\rail@nextbar{14} -\rail@nont{local}[] -\rail@nextbar{15} -\rail@nont{global}[] -\rail@nextbar{16} -\rail@nont{setup}[] -\rail@endbar -\rail@end -\rail@begin{2}{classes} -\rail@term{classes}[] -\rail@plus -\rail@nont{classDecl}[] -\rail@nextplus{1} -\rail@endplus -\rail@end -\rail@begin{3}{classDecl} -\rail@nont{id}[] -\rail@bar -\rail@nextbar{1} -\rail@term{<}[] -\rail@plus -\rail@nont{id}[] -\rail@nextplus{2} -\rail@cterm{,}[] -\rail@endplus -\rail@endbar -\rail@end -\rail@begin{1}{default} -\rail@term{default}[] -\rail@nont{sort}[] -\rail@end -\rail@begin{4}{sort} -\rail@bar -\rail@nont{id}[] -\rail@nextbar{1} -\rail@token{lbrace}[] -\rail@bar -\rail@nextbar{2} -\rail@plus -\rail@nont{id}[] -\rail@nextplus{3} -\rail@cterm{,}[] -\rail@endplus -\rail@endbar -\rail@token{rbrace}[] -\rail@endbar -\rail@end -\rail@begin{3}{types} -\rail@term{types}[] -\rail@plus -\rail@nont{typeDecl}[] -\rail@bar -\rail@nextbar{1} -\rail@term{(}[] -\rail@nont{infix}[] -\rail@term{)}[] -\rail@endbar -\rail@nextplus{2} -\rail@endplus -\rail@end -\rail@begin{2}{infix} -\rail@bar -\rail@term{infixr}[] -\rail@nextbar{1} -\rail@term{infixl}[] -\rail@endbar -\rail@bar -\rail@nextbar{1} -\rail@nont{string}[] -\rail@endbar -\rail@nont{nat}[] -\rail@end -\rail@begin{3}{typeDecl} -\rail@nont{typevarlist}[] -\rail@nont{name}[] -\rail@bar -\rail@nextbar{1} -\rail@term{=}[] -\rail@bar -\rail@nont{string}[] -\rail@nextbar{2} -\rail@nont{type}[] -\rail@endbar -\rail@endbar -\rail@end -\rail@begin{4}{typevarlist} -\rail@bar -\rail@nextbar{1} -\rail@nont{tid}[] -\rail@nextbar{2} -\rail@term{(}[] -\rail@plus -\rail@nont{tid}[] -\rail@nextplus{3} -\rail@cterm{,}[] -\rail@endplus -\rail@term{)}[] -\rail@endbar -\rail@end -\rail@begin{5}{type} -\rail@bar -\rail@nont{simpleType}[] -\rail@nextbar{1} -\rail@term{(}[] -\rail@nont{type}[] -\rail@term{)}[] -\rail@nextbar{2} -\rail@nont{type}[] -\rail@term{=>}[] -\rail@nont{type}[] -\rail@nextbar{3} -\rail@term{[}[] -\rail@plus -\rail@nont{type}[] -\rail@nextplus{4} -\rail@cterm{,}[] -\rail@endplus -\rail@term{]}[] -\rail@term{=>}[] -\rail@nont{type}[] -\rail@endbar -\rail@end -\rail@begin{6}{simpleType} -\rail@bar -\rail@nont{id}[] -\rail@nextbar{1} -\rail@nont{tid}[] -\rail@bar -\rail@nextbar{2} -\rail@term{::}[] -\rail@nont{id}[] -\rail@endbar -\rail@nextbar{3} -\rail@term{(}[] -\rail@plus -\rail@nont{type}[] -\rail@nextplus{4} -\rail@cterm{,}[] -\rail@endplus -\rail@term{)}[] -\rail@nont{id}[] -\rail@nextbar{5} -\rail@nont{simpleType}[] -\rail@nont{id}[] -\rail@endbar -\rail@end -\rail@begin{3}{arities} -\rail@term{arities}[] -\rail@plus -\rail@plus -\rail@nont{name}[] -\rail@nextplus{1} -\rail@cterm{,}[] -\rail@endplus -\rail@term{::}[] -\rail@nont{arity}[] -\rail@nextplus{2} -\rail@endplus -\rail@end -\rail@begin{3}{arity} -\rail@bar -\rail@nextbar{1} -\rail@term{(}[] -\rail@plus -\rail@nont{sort}[] -\rail@nextplus{2} -\rail@cterm{,}[] -\rail@endplus -\rail@term{)}[] -\rail@endbar -\rail@nont{sort}[] -\rail@end -\rail@begin{2}{nonterminals} -\rail@term{nonterminals}[] -\rail@plus -\rail@nont{name}[] -\rail@nextplus{1} -\rail@endplus -\rail@end -\rail@begin{2}{consts} -\rail@term{consts}[] -\rail@plus -\rail@nont{mixfixConstDecl}[] -\rail@nextplus{1} -\rail@endplus -\rail@end -\rail@begin{2}{syntax} -\rail@term{syntax}[] -\rail@bar -\rail@nextbar{1} -\rail@nont{mode}[] -\rail@endbar -\rail@plus -\rail@nont{mixfixConstDecl}[] -\rail@nextplus{1} -\rail@endplus -\rail@end -\rail@begin{2}{mode} -\rail@term{(}[] -\rail@nont{name}[] -\rail@bar -\rail@nextbar{1} -\rail@term{output}[] -\rail@endbar -\rail@term{)}[] -\rail@end -\rail@begin{2}{mixfixConstDecl} -\rail@nont{constDecl}[] -\rail@bar -\rail@nextbar{1} -\rail@term{(}[] -\rail@nont{mixfix}[] -\rail@term{)}[] -\rail@endbar -\rail@end -\rail@begin{2}{constDecl} -\rail@plus -\rail@nont{name}[] -\rail@nextplus{1} -\rail@cterm{,}[] -\rail@endplus -\rail@term{::}[] -\rail@bar -\rail@nont{string}[] -\rail@nextbar{1} -\rail@nont{type}[] -\rail@endbar -\rail@end -\rail@begin{6}{mixfix} -\rail@bar -\rail@nont{string}[] -\rail@bar -\rail@nextbar{1} -\rail@bar -\rail@nextbar{2} -\rail@term{[}[] -\rail@plus -\rail@nont{nat}[] -\rail@nextplus{3} -\rail@cterm{,}[] -\rail@endplus -\rail@term{]}[] -\rail@endbar -\rail@nont{nat}[] -\rail@endbar -\rail@nextbar{4} -\rail@nont{infix}[] -\rail@nextbar{5} -\rail@term{binder}[] -\rail@nont{string}[] -\rail@nont{nat}[] -\rail@endbar -\rail@end -\rail@begin{4}{trans} -\rail@term{translations}[] -\rail@plus -\rail@nont{pat}[] -\rail@bar -\rail@term{==}[] -\rail@nextbar{1} -\rail@term{=>}[] -\rail@nextbar{2} -\rail@term{<=}[] -\rail@endbar -\rail@nont{pat}[] -\rail@nextplus{3} -\rail@endplus -\rail@end -\rail@begin{2}{pat} -\rail@bar -\rail@nextbar{1} -\rail@term{(}[] -\rail@nont{id}[] -\rail@term{)}[] -\rail@endbar -\rail@nont{string}[] -\rail@end -\rail@begin{2}{rules} -\rail@term{rules}[] -\rail@plus -\rail@nont{id}[] -\rail@nont{string}[] -\rail@nextplus{1} -\rail@endplus -\rail@end -\rail@begin{2}{defs} -\rail@term{defs}[] -\rail@plus -\rail@nont{id}[] -\rail@nont{string}[] -\rail@nextplus{1} -\rail@endplus -\rail@end -\rail@begin{3}{constdefs} -\rail@term{constdefs}[] -\rail@plus -\rail@nont{name}[] -\rail@term{::}[] -\rail@bar -\rail@nont{string}[] -\rail@nextbar{1} -\rail@nont{type}[] -\rail@endbar -\rail@bar -\rail@nextbar{1} -\rail@nont{mixfix}[] -\rail@endbar -\rail@nont{string}[] -\rail@nextplus{2} -\rail@endplus -\rail@end -\rail@begin{3}{axclass} -\rail@term{axclass}[] -\rail@nont{classDecl}[] -\rail@bar -\rail@nextbar{1} -\rail@plus -\rail@nont{id}[] -\rail@nont{string}[] -\rail@nextplus{2} -\rail@endplus -\rail@endbar -\rail@end -\rail@begin{2}{instance} -\rail@term{instance}[] -\rail@bar -\rail@nont{name}[] -\rail@term{<}[] -\rail@nont{name}[] -\rail@nextbar{1} -\rail@nont{name}[] -\rail@term{::}[] -\rail@nont{arity}[] -\rail@endbar -\rail@nont{witness}[] -\rail@end -\rail@begin{5}{witness} -\rail@bar -\rail@nextbar{1} -\rail@term{(}[] -\rail@plus -\rail@bar -\rail@nont{string}[] -\rail@nextbar{2} -\rail@nont{id}[] -\rail@nextbar{3} -\rail@nont{longident}[] -\rail@endbar -\rail@nextplus{4} -\rail@cterm{,}[] -\rail@endplus -\rail@term{)}[] -\rail@endbar -\rail@bar -\rail@nextbar{1} -\rail@nont{verbatim}[] -\rail@endbar -\rail@end -\rail@begin{1}{oracle} -\rail@term{oracle}[] -\rail@nont{name}[] -\rail@term{=}[] -\rail@nont{name}[] -\rail@end -\rail@begin{1}{local} -\rail@term{local}[] -\rail@end -\rail@begin{1}{global} -\rail@term{global}[] -\rail@end -\rail@begin{2}{setup} -\rail@term{setup}[] -\rail@bar -\rail@nont{id}[] -\rail@nextbar{1} -\rail@nont{longident}[] -\rail@endbar -\rail@end -\rail@begin{1}{ml} -\rail@term{ML}[] -\rail@nont{text}[] -\rail@end -} diff -r dc5bf3f40ad3 -r 5a94bd71cc41 doc-src/System/Makefile --- a/doc-src/System/Makefile Wed May 05 18:26:10 1999 +0200 +++ b/doc-src/System/Makefile Wed May 05 18:35:41 1999 +0200 @@ -1,30 +1,25 @@ -# $Id$ -######################################################################### -# # -# Makefile for the report "The Isabelle System Manual" # -# # -######################################################################### +# +# $Id$ +# + +## targets + +default: dvi +dist: dvi -FILES = system.tex \ - ../iman.sty ../extra.sty +## dependencies + +include ../Makefile.in + +NAME = system +FILES = system.tex ../iman.sty ../extra.sty -system.dvi.gz: $(FILES) - test -r isabelle.eps || ln -s ../gfx/isabelle.eps . - -rm system.dvi* - latex system - latex system - ../sedindex system - latex system - gzip -f system.dvi +dvi: $(NAME).dvi -dist: $(FILES) - test -r isabelle.eps || ln -s ../gfx/isabelle.eps . - -rm system.dvi* - latex system - latex system - ../sedindex system - latex system - -clean: - @rm *.aux *.log *.toc *.idx +$(NAME).dvi: $(FILES) isabelle.eps + touch $(NAME).ind + $(LATEX) $(NAME) + $(LATEX) $(NAME) + $(SEDINDEX) $(NAME) + $(LATEX) $(NAME) diff -r dc5bf3f40ad3 -r 5a94bd71cc41 doc-src/System/system.ind --- a/doc-src/System/system.ind Wed May 05 18:26:10 1999 +0200 +++ /dev/null Thu Jan 01 00:00:00 1970 +0000 @@ -1,85 +0,0 @@ -\begin{theindex} - - \item {\tt browser} tool, 19 - - \indexspace - - \item {\tt doc} tool, 8 - \item {\tt DVI_VIEWER} setting, 4 - - \indexspace - - \item {\tt expandshort} tool, 8 - - \indexspace - - \item {\tt findlogics} tool, 9 - - \indexspace - - \item {\tt getenv} tool, 9 - - \indexspace - - \item HTML, 12 - - \indexspace - - \item {\tt INSTALL}, 1 - \item {\tt install} tool, 10 - \item {\tt installfonts} tool, 14 - \item {\tt ISABELLE} setting, 3 - \item {\tt Isabelle}, 1, 7 - \item {\tt isabelle}, 1, 4 - \item {\tt ISABELLE_BROWSER_INFO} setting, 4, 17 - \item {\tt ISABELLE_DOCS} setting, 4 - \item {\tt ISABELLE_HOME} setting, 2, 3 - \item {\tt ISABELLE_HOME_USER} setting, 3 - \item {\tt ISABELLE_INSTALL_FONTS} setting, 4 - \item {\tt ISABELLE_INSTALLFONTS} setting, 14 - \item {\tt ISABELLE_INTERFACE} setting, 4, 7 - \item {\tt ISABELLE_LOGIC} setting, 4 - \item {\tt ISABELLE_OUTPUT} setting, 3, 4 - \item {\tt ISABELLE_PATH} setting, 3, 4 - \item {\tt ISABELLE_TMP_PREFIX} setting, 4 - \item {\tt ISABELLE_TOOLS} setting, 4 - \item {\tt ISABELLE_USEDIR_OPTIONS} setting, 4, 12, 17 - \item {\tt IsaMakefile}, 11, 12 - \item {\tt ISATOOL} setting, 3 - \item {\tt isatool}, 1, 7 - - \indexspace - - \item {\tt logo} tool, 11 - - \indexspace - - \item {\tt make} tool, 11 - \item {\tt makeall} tool, 12 - \item {\tt ML_HOME} setting, 3 - \item {\tt ML_IDENTIFIER} setting, 3 - \item {\tt ML_OPTIONS} setting, 3 - \item {\tt ML_PLATFORM} setting, 3 - \item {\tt ML_SYSTEM} setting, 3 - - \indexspace - - \item {\tt nonascii} tool, 15 - - \indexspace - - \item settings, \bold{1} - \item {\tt symbolinput} tool, 16 - \item {\tt symbols}, 14 - - \indexspace - - \item theory browsing information, \bold{17} - \item theory graph browser, \bold{18} - - \indexspace - - \item {\tt use_dir}, 18 - \item {\tt usedir} tool, 12 - -\end{theindex} diff -r dc5bf3f40ad3 -r 5a94bd71cc41 doc-src/Tutorial/Makefile --- a/doc-src/Tutorial/Makefile Wed May 05 18:26:10 1999 +0200 +++ b/doc-src/Tutorial/Makefile Wed May 05 18:35:41 1999 +0200 @@ -1,34 +1,29 @@ -# $Id$ -######################################################################### -# # -# Makefile for the report "Isabelle/HOL. The Tutorial" # -# # -######################################################################### +# +# $Id$ +# + +## targets + +default: dvi +dist: dvi -FILES = tutorial.tex basics.tex fp.tex appendix.tex \ - ../iman.sty ttbox.sty extra.sty +## dependencies + +include ../Makefile.in + +NAME = tutorial +FILES = tutorial.tex basics.tex fp.tex appendix.tex \ + ../iman.sty ttbox.sty extra.sty + +dvi: $(NAME).dvi -tutorial.ps.gz: $(FILES) - isatool make - test -r isabelle_hol.eps || ln -s ../gfx/isabelle_hol.eps . - -rm tutorial.dvi* - latex tutorial - bibtex tutorial - latex tutorial - latex tutorial - ../sedindex tutorial - latex tutorial - dvips tutorial.dvi -o tutorial.ps - gzip tutorial.ps - -dist: $(FILES) - test -r isabelle_hol.eps || ln -s ../gfx/isabelle_hol.eps . - -rm tutorial.dvi* - latex tutorial - latex tutorial - ../sedindex tutorial - latex tutorial - -clean: - @rm *.aux *.log *.toc *.idx +$(NAME).dvi: $(FILES) isabelle_hol.eps + touch $(NAME).ind + $(LATEX) $(NAME) + $(RAIL) $(NAME) + $(BIBTEX) $(NAME) + $(LATEX) $(NAME) + $(LATEX) $(NAME) + $(SEDINDEX) $(NAME) + $(LATEX) $(NAME) diff -r dc5bf3f40ad3 -r 5a94bd71cc41 doc-src/Tutorial/tutorial.bbl --- a/doc-src/Tutorial/tutorial.bbl Wed May 05 18:26:10 1999 +0200 +++ /dev/null Thu Jan 01 00:00:00 1970 +0000 @@ -1,49 +0,0 @@ -\begin{thebibliography}{1} - -\bibitem{Bird-Wadler} -Richard Bird and Philip Wadler. -\newblock {\em Introduction to Functional Programming}. -\newblock Prentice-Hall, 1988. - -\bibitem{Gunter-HOL92} -Elsa~L. Gunter. -\newblock Why we can't have {SML} style datatype declarations in {HOL}. -\newblock In L.J.M. Claesen and M.J.C. Gordon, editors, {\em Higher Order Logic - Theorem Proving and its Applications: Proc.\ IFIP TC10/WG10.2 Intl. Workshop, - 1992}, pages 561--568. North-Holland, 1993. - -\bibitem{Knuth3-75} -Donald~E. Knuth. -\newblock {\em The Art of Computer Programming, Volume 3: Sorting and - Searching}. -\newblock Addison-Wesley, 1975. - -\bibitem{MuellerNvOS98} -Olaf M\"uller, Tobias Nipkow, David~von Oheimb, and Oskar Slotosch. -\newblock {HOLCF = HOL + LCF}. -\newblock {\em J. Functional Programming}, 1999. -\newblock To appear. - -\bibitem{Isa-Ref-Man} -Lawrence~C. Paulson. -\newblock {\em The Isabelle Reference Manual}. -\newblock University of Cambridge, Computer Laboratory. -\newblock \verb$http://www.in.tum.de/~isabelle/dist/$. - -\bibitem{Isa-Logics-Man} -Lawrence~C. Paulson. -\newblock {\em Isabelle's Object-Logics}. -\newblock University of Cambridge, Computer Laboratory. -\newblock \verb$http://www.in.tum.de/~isabelle/dist/$. - -\bibitem{Paulson-LCF} -Lawrence~C. Paulson. -\newblock {\em Logic and Computation}. -\newblock Cambridge University Press, 1987. - -\bibitem{Paulson-ML} -Lawrence~C. Paulson. -\newblock {\em ML for the Working Programmer}. -\newblock Cambridge University Press, 2nd edition, 1996. - -\end{thebibliography} diff -r dc5bf3f40ad3 -r 5a94bd71cc41 doc-src/Tutorial/tutorial.ind --- a/doc-src/Tutorial/tutorial.ind Wed May 05 18:26:10 1999 +0200 +++ /dev/null Thu Jan 01 00:00:00 1970 +0000 @@ -1,148 +0,0 @@ -\begin{theindex} - - \item {\tt[]}, \bold{7} - \item {\tt\#}, \bold{7} - \item {\ttnot}, \bold{3} - \item {\tt-->}, \bold{3} - \item {\tt\&}, \bold{3} - \item {\ttor}, \bold{3} - \item {\tt?}, \bold{3}, 4 - \item {\ttall}, \bold{3} - \item {\ttuniquex}, \bold{3} - \item {\tt *}, \bold{17} - \item {\tt +}, \bold{17} - \item {\tt -}, \bold{17, 18} - \item {\tt <}, \bold{17} - \item {\tt <=}, \bold{17} - \item \ttlbr, \bold{9} - \item \ttrbr, \bold{9} - \item {\tt==>}, \bold{9} - \item {\tt==}, \bold{19} - \item {\tt\%}, \bold{3} - \item {\tt =>}, \bold{2} - - \indexspace - - \item {\tt addsimps}, \bold{22} - \item {\tt Addsplits}, \bold{24} - \item {\tt addsplits}, \bold{24} - \item {\tt and}, \bold{29} - \item {\tt arith_tac}, \bold{17} - \item arithmetic, 17--18, 24 - \item {\tt Asm_full_simp_tac}, \bold{21} - \item {\tt asm_full_simp_tac}, \bold{22} - \item {\tt Asm_simp_tac}, \bold{21} - \item {\tt asm_simp_tac}, \bold{22} - - \indexspace - - \item {\tt bool}, 2 - - \indexspace - - \item {\tt case}, \bold{3}, 4, \bold{13}, 24 - \item {\tt constdefs}, \bold{19} - \item {\tt consts}, \bold{7} - \item {\tt context}, \bold{11} - \item current theory, \bold{11} - - \indexspace - - \item {\tt datatype}, \bold{7}, 29--33 - \item {\tt defs}, \bold{19} - \item {\tt delsimps}, \bold{22} - \item {\tt Delsplits}, \bold{24} - \item {\tt delsplits}, \bold{24} - \item {\tt div}, \bold{17} - - \indexspace - - \item {\tt exhaust_tac}, \bold{14} - - \indexspace - - \item {\tt False}, \bold{3} - \item formula, \bold{3} - \item {\tt Full_simp_tac}, \bold{21} - \item {\tt full_simp_tac}, \bold{22} - - \indexspace - - \item {\tt hd}, \bold{12} - - \indexspace - - \item {\tt if}, \bold{3}, 4, 24 - \item {\tt infixr}, \bold{7} - \item inner syntax, \bold{8} - - \indexspace - - \item {\tt LEAST}, \bold{17} - \item {\tt let}, \bold{3}, 4, 23 - \item {\tt list}, 2 - \item loading theories, 12 - - \indexspace - - \item {\tt Main}, \bold{2} - \item {\tt max}, \bold{17, 18} - \item measure function, \bold{36} - \item {\tt min}, \bold{17, 18} - \item {\tt mod}, \bold{17} - \item {\tt mutual_induct_tac}, \bold{30} - - \indexspace - - \item {\tt nat}, 2, \bold{17} - \item {\tt None}, \bold{33} - - \indexspace - - \item {\tt option}, \bold{33} - - \indexspace - - \item parent theory, \bold{1} - \item primitive recursion, \bold{13} - \item {\tt primrec}, 7, \bold{13}, 29--33 - \item proof scripts, \bold{2} - - \indexspace - - \item {\tt recdef}, 35--38 - \item reloading theories, 12 - - \indexspace - - \item schematic variable, \bold{4} - \item {\tt set}, 2 - \item {\tt show_brackets}, \bold{4} - \item {\tt show_types}, \bold{3}, 11 - \item {\tt Simp_tac}, \bold{21} - \item {\tt simp_tac}, \bold{22} - \item simplifier, \bold{20} - \item simpset, \bold{21} - \item {\tt Some}, \bold{33} - - \indexspace - - \item tactic, \bold{11} - \item term, \bold{3} - \item theory, \bold{1} - \item {\tt tl}, \bold{12} - \item total, \bold{7} - \item tracing the simplifier, \bold{25} - \item {\tt True}, \bold{3} - \item type constraints, \bold{3} - \item type inference, \bold{3} - \item type synonyms, \bold{18} - \item {\tt types}, \bold{18} - - \indexspace - - \item unknown, \bold{4} - \item {\tt update_thy}, \bold{12} - \item {\tt use_thy}, \bold{2}, 12 - -\end{theindex}