Mon, 25 Oct 1993 12:42:33 +0100 added white-space;
wenzelm [Mon, 25 Oct 1993 12:42:33 +0100] rev 80
added white-space; made ~: a fake infix;
Mon, 25 Oct 1993 12:32:53 +0100 added white-space;
wenzelm [Mon, 25 Oct 1993 12:32:53 +0100] rev 79
added white-space; made ~= a fake infix;
Fri, 22 Oct 1993 22:17:25 +0100 removed a bug that occured when a path was specified for use_thy's parameter
clasohm [Fri, 22 Oct 1993 22:17:25 +0100] rev 78
removed a bug that occured when a path was specified for use_thy's parameter and the theory was created in a .ML file
Fri, 22 Oct 1993 17:39:12 +0100 ZF/ex/tf,tf_fn: renamed the variable tf to f everywhere
lcp [Fri, 22 Oct 1993 17:39:12 +0100] rev 77
ZF/ex/tf,tf_fn: renamed the variable tf to f everywhere
Fri, 22 Oct 1993 13:44:27 +0100 renamed some files
clasohm [Fri, 22 Oct 1993 13:44:27 +0100] rev 76
renamed some files
Fri, 22 Oct 1993 13:43:45 +0100 added -h 15000 for Poly/ML in Makefile,
clasohm [Fri, 22 Oct 1993 13:43:45 +0100] rev 75
added -h 15000 for Poly/ML in Makefile, changed ROOT.ML for new Readthy
Fri, 22 Oct 1993 13:42:51 +0100 changes in Readthy:
clasohm [Fri, 22 Oct 1993 13:42:51 +0100] rev 74
changes in Readthy: - reads needed base theories automatically - keeps a time stamp for all read files - update function - checks for cycles - path list that is searched for files - reads theories that are created in .ML files - etc.
Fri, 22 Oct 1993 13:39:23 +0100 delete_file now has type string -> unit in both NJ and POLY,
clasohm [Fri, 22 Oct 1993 13:39:23 +0100] rev 73
delete_file now has type string -> unit in both NJ and POLY, use of Pure/Thy/ROOT has been moved to the end of Pure/ROOT again
Fri, 22 Oct 1993 13:35:15 +0100 changes for new Readthy
clasohm [Fri, 22 Oct 1993 13:35:15 +0100] rev 72
changes for new Readthy
Fri, 22 Oct 1993 11:42:02 +0100 sample datatype defs now use datatype_intrs, datatype_elims
lcp [Fri, 22 Oct 1993 11:42:02 +0100] rev 71
sample datatype defs now use datatype_intrs, datatype_elims
Fri, 22 Oct 1993 11:34:41 +0100 ZF/ind-syntax/fold_con_tac: deleted, since fold_tac now works
lcp [Fri, 22 Oct 1993 11:34:41 +0100] rev 70
ZF/ind-syntax/fold_con_tac: deleted, since fold_tac now works ZF/intr-elim/elim_rls: applied make_elim to succ_inject! ZF/fin: changed type_intrs in inductive def ZF/datatype/datatype_intrs, datatype_elims: renamed from data_typechecks, data_elims ZF/list: now uses datatype_intrs
Fri, 22 Oct 1993 11:25:15 +0100 tactic/fold_tac,fold_goals_tac: now handle critical pairs on the
lcp [Fri, 22 Oct 1993 11:25:15 +0100] rev 69
tactic/fold_tac,fold_goals_tac: now handle critical pairs on the right sides of the defs
Fri, 22 Oct 1993 10:31:19 +0100 goals/print_top,prepare_proof: now call \!print_goals_ref
lcp [Fri, 22 Oct 1993 10:31:19 +0100] rev 68
goals/print_top,prepare_proof: now call \!print_goals_ref
Thu, 21 Oct 1993 17:20:01 +0100 Pure/drule/print_goals_ref: new, for Centaur interface
lcp [Thu, 21 Oct 1993 17:20:01 +0100] rev 67
Pure/drule/print_goals_ref: new, for Centaur interface Pure/tctical/tracify,print_tac: now call !print_goals_ref Pure/goals/print_top,prepare_proof: now call !print_goals_ref
Thu, 21 Oct 1993 17:10:15 +0100 /NJ,POLY/delete_file: new
lcp [Thu, 21 Oct 1993 17:10:15 +0100] rev 66
/NJ,POLY/delete_file: new
Thu, 21 Oct 1993 14:59:54 +0100 simpdata/basify: now calls new fastype_of
lcp [Thu, 21 Oct 1993 14:59:54 +0100] rev 65
simpdata/basify: now calls new fastype_of
Thu, 21 Oct 1993 14:56:12 +0100 logic/mk_equals,mk_flexpair: now calls fastype_of instead of type_of.
lcp [Thu, 21 Oct 1993 14:56:12 +0100] rev 64
logic/mk_equals,mk_flexpair: now calls fastype_of instead of type_of. So it no longer checks t properly -- but it never checked u anyway, and all existing calls are derived from certified terms...
Thu, 21 Oct 1993 14:47:48 +0100 now calls new fastype_of in three places
lcp [Thu, 21 Oct 1993 14:47:48 +0100] rev 63
now calls new fastype_of in three places
Thu, 21 Oct 1993 14:40:06 +0100 Pure/Syntax/printer/is_prop: now calls fastype_of1
lcp [Thu, 21 Oct 1993 14:40:06 +0100] rev 62
Pure/Syntax/printer/is_prop: now calls fastype_of1
Thu, 21 Oct 1993 14:38:06 +0100 Pure/term/fastype_of1: renamed from fastype_of
lcp [Thu, 21 Oct 1993 14:38:06 +0100] rev 61
Pure/term/fastype_of1: renamed from fastype_of Pure/term/fastype_of: new, takes only one argument (like type_of) Pure/Syntax/printer/is_prop: now calls fastype_of1 Pure/pattern: now calls new fastype_of in three places Pure/logic/mk_equals,mk_flexpair: now calls fastype_of instead of type_of. So it no longer checks t properly -- but it never checked u anyway, and all existing calls are derived from certified terms...
Sun, 17 Oct 1993 18:03:47 +0100 renamed: S4.thy to s4.thy, S43.thy to s43.thy, T.thy to t.thy
clasohm [Sun, 17 Oct 1993 18:03:47 +0100] rev 60
renamed: S4.thy to s4.thy, S43.thy to s43.thy, T.thy to t.thy
Sun, 17 Oct 1993 16:30:16 +0100 renamed: terms.* to term.*, types.* to type.*, wf.* to wfd.*
clasohm [Sun, 17 Oct 1993 16:30:16 +0100] rev 59
renamed: terms.* to term.*, types.* to type.*, wf.* to wfd.*
Fri, 15 Oct 1993 12:51:21 +0100 file_info now returns a string that does not contain the path/filename
clasohm [Fri, 15 Oct 1993 12:51:21 +0100] rev 58
file_info now returns a string that does not contain the path/filename (so the string doesn't change when the relative path does)
Fri, 15 Oct 1993 12:49:33 +0100 added parser.ML, install_pp.ML
wenzelm [Fri, 15 Oct 1993 12:49:33 +0100] rev 57
added parser.ML, install_pp.ML
Fri, 15 Oct 1993 10:25:23 +0100 ZF/ex/tf/tree,forest_unfold: streamlined the proofs
lcp [Fri, 15 Oct 1993 10:25:23 +0100] rev 56
ZF/ex/tf/tree,forest_unfold: streamlined the proofs Updated other inductive def examples as per changes in the package.
Fri, 15 Oct 1993 10:21:01 +0100 ZF/ind-syntax/refl_thin: new
lcp [Fri, 15 Oct 1993 10:21:01 +0100] rev 55
ZF/ind-syntax/refl_thin: new ZF/intr-elim: added Pair_neq_0, succ_neq_0, refl_thin to simplify case rules ZF/sum/Inl_iff, etc.: tidied and proved using simp_tac ZF/qpair/QInl_iff, etc.: tidied and proved using simp_tac ZF/datatype,intr_elim: replaced the undirectional use of sum_univ RS subsetD by dresolve_tac InlD,InrD and etac PartE
Fri, 15 Oct 1993 10:04:30 +0100 classical/swap_res_tac: recoded to allow backtracking
lcp [Fri, 15 Oct 1993 10:04:30 +0100] rev 54
classical/swap_res_tac: recoded to allow backtracking
Tue, 12 Oct 1993 13:39:35 +0100 Added gen_all to simpdata.ML.
nipkow [Tue, 12 Oct 1993 13:39:35 +0100] rev 53
Added gen_all to simpdata.ML.
Mon, 11 Oct 1993 14:03:40 +0100 renamed ordinal.thy to ord.thy
clasohm [Mon, 11 Oct 1993 14:03:40 +0100] rev 52
renamed ordinal.thy to ord.thy
Mon, 11 Oct 1993 14:00:53 +0100 renamed ordinal.ML to ord.ML
clasohm [Mon, 11 Oct 1993 14:00:53 +0100] rev 51
renamed ordinal.ML to ord.ML
Mon, 11 Oct 1993 13:58:22 +0100 renamed ordinal.* to ord.*
clasohm [Mon, 11 Oct 1993 13:58:22 +0100] rev 50
renamed ordinal.* to ord.*
Mon, 11 Oct 1993 12:35:00 +0100 "The" now a binder, removed translation;
wenzelm [Mon, 11 Oct 1993 12:35:00 +0100] rev 49
"The" now a binder, removed translation; improved encoding and translations of tuples; added parse rules for -> and *, removed ndependent_tr;
Mon, 11 Oct 1993 12:30:38 +0100 removed ndependent_tr (no longer needed, use _K);
wenzelm [Mon, 11 Oct 1993 12:30:38 +0100] rev 48
removed ndependent_tr (no longer needed, use _K);
Mon, 11 Oct 1993 12:30:06 +0100 *** empty log message ***
wenzelm [Mon, 11 Oct 1993 12:30:06 +0100] rev 47
*** empty log message ***
Fri, 08 Oct 1993 14:29:55 +0100 *** empty log message ***
wenzelm [Fri, 08 Oct 1993 14:29:55 +0100] rev 46
*** empty log message ***
Fri, 08 Oct 1993 14:18:51 +0100 fixed comment;
wenzelm [Fri, 08 Oct 1993 14:18:51 +0100] rev 45
fixed comment;
Fri, 08 Oct 1993 14:16:29 +0100 added parse rule for "<*>";
wenzelm [Fri, 08 Oct 1993 14:16:29 +0100] rev 44
added parse rule for "<*>"; removed ndependent_tr;
Fri, 08 Oct 1993 14:11:12 +0100 @List: replaced "args" by "is";
wenzelm [Fri, 08 Oct 1993 14:11:12 +0100] rev 43
@List: replaced "args" by "is";
Fri, 08 Oct 1993 13:55:04 +0100 *** empty log message ***
wenzelm [Fri, 08 Oct 1993 13:55:04 +0100] rev 42
*** empty log message ***
Fri, 08 Oct 1993 12:35:53 +0100 added cons, rcons, last_elem, sort_strings, take_suffix;
wenzelm [Fri, 08 Oct 1993 12:35:53 +0100] rev 41
added cons, rcons, last_elem, sort_strings, take_suffix; improved tack_on;
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;
(0) -60 +60 +100 +300 +1000 +3000 +10000 +30000 tip