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
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
lcp [Fri, 22 Oct 1993 10:31:19 +0100] rev 68
goals/print_top,prepare_proof: now call \!print_goals_ref
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
lcp [Thu, 21 Oct 1993 17:10:15 +0100] rev 66
/NJ,POLY/delete_file: new
lcp [Thu, 21 Oct 1993 14:59:54 +0100] rev 65
simpdata/basify: now calls new fastype_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...
lcp [Thu, 21 Oct 1993 14:47:48 +0100] rev 63
now calls new fastype_of in three places
lcp [Thu, 21 Oct 1993 14:40:06 +0100] rev 62
Pure/Syntax/printer/is_prop: now calls fastype_of1
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...
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
clasohm [Sun, 17 Oct 1993 16:30:16 +0100] rev 59
renamed: terms.* to term.*, types.* to type.*, wf.* to wfd.*
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)
wenzelm [Fri, 15 Oct 1993 12:49:33 +0100] rev 57
added parser.ML, install_pp.ML
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.
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
lcp [Fri, 15 Oct 1993 10:04:30 +0100] rev 54
classical/swap_res_tac: recoded to allow backtracking
nipkow [Tue, 12 Oct 1993 13:39:35 +0100] rev 53
Added gen_all to simpdata.ML.
clasohm [Mon, 11 Oct 1993 14:03:40 +0100] rev 52
renamed ordinal.thy to ord.thy
clasohm [Mon, 11 Oct 1993 14:00:53 +0100] rev 51
renamed ordinal.ML to ord.ML
clasohm [Mon, 11 Oct 1993 13:58:22 +0100] rev 50
renamed ordinal.* to ord.*
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;
wenzelm [Mon, 11 Oct 1993 12:30:38 +0100] rev 48
removed ndependent_tr (no longer needed, use _K);
wenzelm [Mon, 11 Oct 1993 12:30:06 +0100] rev 47
*** empty log message ***