wenzelm [Mon, 04 Oct 1993 15:49:49 +0100] rev 23
replaced id by idt;
added parse rules for --> and *;
removed ndependent_tr;
wenzelm [Mon, 04 Oct 1993 15:44:54 +0100] rev 22
added parse rules for -> and *;
removed ndependent_tr;
wenzelm [Mon, 04 Oct 1993 15:44:29 +0100] rev 21
replaced id by idt;
added parse rule for ->;
removed ndependent_tr;
wenzelm [Mon, 04 Oct 1993 15:38:02 +0100] rev 20
Pure/Thy/syntax.ML
removed {parse,print}_{pre,post}_proc;
removed 'val ax = ..';
wenzelm [Mon, 04 Oct 1993 15:36:31 +0100] rev 19
Pure/ROOT.ML
cleaned comments;
removed extraneous 'print_depth 1';
replaced Basic_Syntax by BasicSyntax
added 'use "install_pp.ML"';
Pure/README
fixed comments;
Pure/POLY.ML
Pure/NJ.ML
make_pp: added fbrk;
Pure/install_pp.ML
replaced "Ast" by "Syntax";
Pure/sign.ML
added 'quote' to some error msgs;
wenzelm [Mon, 04 Oct 1993 15:30:49 +0100] rev 18
lots of internal cleaning and tuning;
removed {parse,print}_{pre,post}_proc;
new lexer: now human readable due to scanner combinators;
new parser installed, but still inactive (due to grammar ambiguities);
added Syntax.test_read;
typ_of_term: sorts now made distinct and sorted;
mixfix: added forced line breaks (//);
PROP now printed before subterm of type prop with non-const head;
nipkow [Fri, 01 Oct 1993 13:26:22 +0100] rev 17
asm_full_simp_tac now fails when applied to a state w/o subgoals.
lcp [Thu, 30 Sep 1993 10:54:01 +0100] rev 16
ex/{bin.ML,comb.ML,prop.ML}: replaced NewSext by Syntax.simple_sext
ex/prop-log/hyps_thms_if: split up the fast_tac call for more speed
called expandshort
lcp [Thu, 30 Sep 1993 10:26:38 +0100] rev 15
ex/{bin.ML,comb.ML,prop.ML}: replaced NewSext by Syntax.simple_sext
domrange/image_subset,vimage_subset: deleted needless premise!
misc: This slightly simplifies two proofs in Schroeder-Bernstein Theorem
ind-syntax/rule_concl: recoded to avoid exceptions
intr-elim: now checks conclusions of introduction rules
func/fun_disjoint_Un: now uses ex_ex1I
list-fn/hd,tl,drop: new
simpdata/bquant_simps: new
list/list_case_type: restored!
bool.thy: changed 1 from a "def" to a translation
Removed occurreces of one_def in bool.ML, nat.ML, univ.ML, ex/integ.ML
nat/succ_less_induct: new induction principle
arith/add_mono: new results about monotonicity
simpdata/mem_simps: removed the ones for succ and cons; added succI1,
consI2 to ZF_ss
upair/succ_iff: new, for use with simp_tac (cons_iff already existed)
ordinal/Ord_0_in_succ: renamed from Ord_0_mem_succ
nat/nat_0_in_succ: new
ex/prop-log/hyps_thms_if: split up the fast_tac call for more speed
lcp [Thu, 30 Sep 1993 10:10:21 +0100] rev 14
ex/{bin.ML,comb.ML,prop.ML}: replaced NewSext by Syntax.simple_sext
domrange/image_subset,vimage_subset: deleted needless premise!
misc: This slightly simplifies two proofs in Schroeder-Bernstein Theorem
ind-syntax/rule_concl: recoded to avoid exceptions
intr-elim: now checks conclusions of introduction rules
func/fun_disjoint_Un: now uses ex_ex1I
list-fn/hd,tl,drop: new
simpdata/bquant_simps: new
list/list_case_type: restored!
bool.thy: changed 1 from a "def" to a translation
Removed occurreces of one_def in bool.ML, nat.ML, univ.ML, ex/integ.ML
nat/succ_less_induct: new induction principle
arith/add_mono: new results about monotonicity
simpdata/mem_simps: removed the ones for succ and cons; added succI1,
consI2 to ZF_ss
upair/succ_iff: new, for use with simp_tac (cons_iff already existed)
ordinal/Ord_0_in_succ: renamed from Ord_0_mem_succ
nat/nat_0_in_succ: new
ex/prop-log/hyps_thms_if: split up the fast_tac call for more speed
lcp [Fri, 24 Sep 1993 11:27:15 +0200] rev 13
Added example from Avron: Gentzen-Type Systems, Resolution and Tableaux, JAR 10
lcp [Fri, 24 Sep 1993 11:13:55 +0200] rev 12
Added ex_ex1I: new introduction rule for the EX! quantifier.
lcp [Fri, 24 Sep 1993 10:52:55 +0200] rev 11
Added MRS, MRL from ZF/ROOT.ML. These support forward proof, resolving a
rule's premises against a list of other proofs.
lcp [Tue, 21 Sep 1993 11:16:19 +0200] rev 10
This commit should not have been necessary. For some reason, the previous
commit did not update genrec.ML. There were still occurrences of SIMP_TAC.
Was the commit perhaps interrupted??