Fri, 08 Oct 1993 12:33:17 +0100 added raise_type: string -> typ list -> term list -> 'a;
wenzelm [Fri, 08 Oct 1993 12:33:17 +0100] rev 40
added raise_type: string -> typ list -> term list -> 'a; added raise_term: string -> term list -> 'a;
Fri, 08 Oct 1993 12:30:01 +0100 "The error/exception above ...": errorneous goal now quoted;
wenzelm [Fri, 08 Oct 1993 12:30:01 +0100] rev 39
"The error/exception above ...": errorneous goal now quoted;
Thu, 07 Oct 1993 11:47:50 +0100 used ~: for "not in"
lcp [Thu, 07 Oct 1993 11:47:50 +0100] rev 38
used ~: for "not in"
Thu, 07 Oct 1993 10:48:16 +0100 added ~: for "not in"
lcp [Thu, 07 Oct 1993 10:48:16 +0100] rev 37
added ~: for "not in"
Thu, 07 Oct 1993 09:49:46 +0100 examples now use ~= for "not equals"
lcp [Thu, 07 Oct 1993 09:49:46 +0100] rev 36
examples now use ~= for "not equals"
Thu, 07 Oct 1993 09:47:47 +0100 ifol.thy: added ~= for "not equals"
lcp [Thu, 07 Oct 1993 09:47:47 +0100] rev 35
ifol.thy: added ~= for "not equals"
Wed, 06 Oct 1993 14:45:04 +0100 changed filenames to lower case name of theory the file contains
clasohm [Wed, 06 Oct 1993 14:45:04 +0100] rev 34
changed filenames to lower case name of theory the file contains (only one theory per file, therefore llist.ML has been split)
Wed, 06 Oct 1993 14:21:36 +0100 rename list-fn to listfn
clasohm [Wed, 06 Oct 1993 14:21:36 +0100] rev 33
rename list-fn to listfn
Wed, 06 Oct 1993 14:19:39 +0100 changed "list-fn" to "listfn"
clasohm [Wed, 06 Oct 1993 14:19:39 +0100] rev 32
changed "list-fn" to "listfn"
Wed, 06 Oct 1993 10:33:33 +0100 tctical/dummy_quant_rl: specifies type prop to avoid the type variable
lcp [Wed, 06 Oct 1993 10:33:33 +0100] rev 31
tctical/dummy_quant_rl: specifies type prop to avoid the type variable ?'a from occurring -- which sometimes caused SELECT_GOAL to fail
Wed, 06 Oct 1993 09:58:53 +0100 Retrying yet again after network problems
lcp [Wed, 06 Oct 1993 09:58:53 +0100] rev 30
Retrying yet again after network problems
Tue, 05 Oct 1993 17:49:23 +0100 Modification of examples for the new operators, < and le.
lcp [Tue, 05 Oct 1993 17:49:23 +0100] rev 29
Modification of examples for the new operators, < and le.
Tue, 05 Oct 1993 17:27:05 +0100 Retry of the previous commit (network outage)
lcp [Tue, 05 Oct 1993 17:27:05 +0100] rev 28
Retry of the previous commit (network outage)
Tue, 05 Oct 1993 17:15:28 +0100 Retry of the previous commit (network outage)
lcp [Tue, 05 Oct 1993 17:15:28 +0100] rev 27
Retry of the previous commit (network outage)
Tue, 05 Oct 1993 15:32:29 +0100 ordinal: DEFINITION of < and le to replace : and <= on ordinals! Many
lcp [Tue, 05 Oct 1993 15:32:29 +0100] rev 26
ordinal: DEFINITION of < and le to replace : and <= on ordinals! Many changes epsilon,arith: many changes ordinal/succ_mem_succI/E: deleted; use succ_leI/E nat/nat_0_in_succ: deleted; use nat_0_le univ/Vset_rankI: deleted; use VsetI
Tue, 05 Oct 1993 15:21:29 +0100 ordinal: DEFINITION of < and le to replace : and <= on ordinals! Many
lcp [Tue, 05 Oct 1993 15:21:29 +0100] rev 25
ordinal: DEFINITION of < and le to replace : and <= on ordinals! Many changes epsilon,arith: many changes ordinal/succ_mem_succI/E: deleted; use succ_leI/E nat/nat_0_in_succ: deleted; use nat_0_le univ/Vset_rankI: deleted; use VsetI
Tue, 05 Oct 1993 13:15:01 +0100 added functions that operate on filenames: split_filename (originally located
clasohm [Tue, 05 Oct 1993 13:15:01 +0100] rev 24
added functions that operate on filenames: split_filename (originally located in Pure/read.ML), tack_on, remove_ext
Mon, 04 Oct 1993 15:49:49 +0100 replaced id by idt;
wenzelm [Mon, 04 Oct 1993 15:49:49 +0100] rev 23
replaced id by idt; added parse rules for --> and *; removed ndependent_tr;
Mon, 04 Oct 1993 15:44:54 +0100 added parse rules for -> and *;
wenzelm [Mon, 04 Oct 1993 15:44:54 +0100] rev 22
added parse rules for -> and *; removed ndependent_tr;
Mon, 04 Oct 1993 15:44:29 +0100 replaced id by idt;
wenzelm [Mon, 04 Oct 1993 15:44:29 +0100] rev 21
replaced id by idt; added parse rule for ->; removed ndependent_tr;
Mon, 04 Oct 1993 15:38:02 +0100 Pure/Thy/syntax.ML
wenzelm [Mon, 04 Oct 1993 15:38:02 +0100] rev 20
Pure/Thy/syntax.ML removed {parse,print}_{pre,post}_proc; removed 'val ax = ..';
Mon, 04 Oct 1993 15:36:31 +0100 Pure/ROOT.ML
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;
Mon, 04 Oct 1993 15:30:49 +0100 lots of internal cleaning and tuning;
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;
Fri, 01 Oct 1993 13:26:22 +0100 asm_full_simp_tac now fails when applied to a state w/o subgoals.
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.
Thu, 30 Sep 1993 10:54:01 +0100 ex/{bin.ML,comb.ML,prop.ML}: replaced NewSext by Syntax.simple_sext
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
Thu, 30 Sep 1993 10:26:38 +0100 ex/{bin.ML,comb.ML,prop.ML}: replaced NewSext by Syntax.simple_sext
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
Thu, 30 Sep 1993 10:10:21 +0100 ex/{bin.ML,comb.ML,prop.ML}: replaced NewSext by Syntax.simple_sext
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
Fri, 24 Sep 1993 11:27:15 +0200 Added example from Avron: Gentzen-Type Systems, Resolution and Tableaux, JAR 10
lcp [Fri, 24 Sep 1993 11:27:15 +0200] rev 13
Added example from Avron: Gentzen-Type Systems, Resolution and Tableaux, JAR 10
Fri, 24 Sep 1993 11:13:55 +0200 Added ex_ex1I: new introduction rule for the EX! quantifier.
lcp [Fri, 24 Sep 1993 11:13:55 +0200] rev 12
Added ex_ex1I: new introduction rule for the EX! quantifier.
Fri, 24 Sep 1993 10:52:55 +0200 Added MRS, MRL from ZF/ROOT.ML. These support forward proof, resolving a
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.
(0) -30 +30 +50 +100 +300 +1000 +3000 +10000 +30000 tip