clasohm [Tue, 09 Nov 1993 13:25:07 +0100] rev 98
renamed int-prover.ML to intprover.ML,
used exact theory names for use_thy
clasohm [Tue, 09 Nov 1993 13:21:41 +0100] rev 97
renamed int-prover.ML to intprover.ML,
used exact theory names in ROOT.ML
lcp [Tue, 09 Nov 1993 11:02:01 +0100] rev 96
now forbids semicolons in the body of br, etc. No longer
requires it to end the line.
lcp [Mon, 08 Nov 1993 17:52:24 +0100] rev 95
Minor changes; addition of counit.ML
nipkow [Fri, 05 Nov 1993 18:49:22 +0100] rev 94
change of my address
lcp [Fri, 05 Nov 1993 11:48:53 +0100] rev 93
Added documenation of change_simp.
clasohm [Thu, 04 Nov 1993 14:15:46 +0100] rev 92
renamed co_inductive.ML to coinductive.ML
clasohm [Thu, 04 Nov 1993 14:12:31 +0100] rev 91
renamed twos-compl.ML to twos_compl.ML
clasohm [Thu, 04 Nov 1993 14:11:59 +0100] rev 90
renamed some files
wenzelm [Thu, 04 Nov 1993 10:34:49 +0100] rev 89
commented out install_pp for term, typ
nipkow [Fri, 29 Oct 1993 11:54:50 +0100] rev 88
added infix delsimps
nipkow [Fri, 29 Oct 1993 11:53:43 +0100] rev 87
added function del_simps
lcp [Thu, 28 Oct 1993 17:40:50 +0100] rev 86
deletion of obsolete/private files; update of README
lcp [Thu, 28 Oct 1993 11:32:37 +0100] rev 85
minor changes e.g. datatype_elims
lcp [Thu, 28 Oct 1993 11:30:35 +0100] rev 84
now uses datatype_intrs and datatype_elims
lcp [Thu, 28 Oct 1993 11:28:36 +0100] rev 83
updated version to October 93
lcp [Wed, 27 Oct 1993 13:49:35 +0100] rev 82
no longer specifies "-h 15000". Instead $ISABELLECOMP should
include any switch settings.
clasohm [Tue, 26 Oct 1993 22:24:20 +0100] rev 81
corrected some spelling mistakes;
removed a bug that made it impossible to read theories that don't have a ML
file;
extended syntax for bases in syntax.ML: a string can be used to specify a
theory that is to be read but is not merged into the base (useful for
pseudo theories used to document the dependencies of ML files)
wenzelm [Mon, 25 Oct 1993 12:42:33 +0100] rev 80
added white-space;
made ~: a fake infix;
wenzelm [Mon, 25 Oct 1993 12:32:53 +0100] rev 79
added white-space;
made ~= a fake infix;
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
lcp [Fri, 22 Oct 1993 17:39:12 +0100] rev 77
ZF/ex/tf,tf_fn: renamed the variable tf to f everywhere
clasohm [Fri, 22 Oct 1993 13:44:27 +0100] rev 76
renamed some files
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
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.
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
clasohm [Fri, 22 Oct 1993 13:35:15 +0100] rev 72
changes for new Readthy
lcp [Fri, 22 Oct 1993 11:42:02 +0100] rev 71
sample datatype defs now use datatype_intrs, datatype_elims
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 ***
wenzelm [Fri, 08 Oct 1993 14:29:55 +0100] rev 46
*** empty log message ***
wenzelm [Fri, 08 Oct 1993 14:18:51 +0100] rev 45
fixed comment;
wenzelm [Fri, 08 Oct 1993 14:16:29 +0100] rev 44
added parse rule for "<*>";
removed ndependent_tr;
wenzelm [Fri, 08 Oct 1993 14:11:12 +0100] rev 43
@List: replaced "args" by "is";
wenzelm [Fri, 08 Oct 1993 13:55:04 +0100] rev 42
*** empty log message ***
wenzelm [Fri, 08 Oct 1993 12:35:53 +0100] rev 41
added cons, rcons, last_elem, sort_strings, take_suffix;
improved tack_on;
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;
wenzelm [Fri, 08 Oct 1993 12:30:01 +0100] rev 39
"The error/exception above ...": errorneous goal now quoted;
lcp [Thu, 07 Oct 1993 11:47:50 +0100] rev 38
used ~: for "not in"
lcp [Thu, 07 Oct 1993 10:48:16 +0100] rev 37
added ~: for "not in"
lcp [Thu, 07 Oct 1993 09:49:46 +0100] rev 36
examples now use ~= for "not equals"
lcp [Thu, 07 Oct 1993 09:47:47 +0100] rev 35
ifol.thy: added ~= for "not equals"
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)
clasohm [Wed, 06 Oct 1993 14:21:36 +0100] rev 33
rename list-fn to listfn
clasohm [Wed, 06 Oct 1993 14:19:39 +0100] rev 32
changed "list-fn" to "listfn"
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
lcp [Wed, 06 Oct 1993 09:58:53 +0100] rev 30
Retrying yet again after network problems
lcp [Tue, 05 Oct 1993 17:49:23 +0100] rev 29
Modification of examples for the new operators, < and le.
lcp [Tue, 05 Oct 1993 17:27:05 +0100] rev 28
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)
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
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
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
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??
lcp [Mon, 20 Sep 1993 18:39:45 +0200] rev 9
make-all now has set +e so that New Jersey runs will continue even if some
logic fails. change_simp added to help change to new simplifier.
lcp [Mon, 20 Sep 1993 17:02:11 +0200] rev 8
Installation of new simplfier. Previously appeared to set up the old
simplifier to rewrite with the partial ordering [=, something not possible
with the new simplifier. But such rewriting appears not to have actually
been used, and there were few complications. In terms.ML setloop was used
to avoid infinite rewriting with the letrec rule. Congruence rules were
deleted, and an occasional SIMP_TAC had to become asm_simp_tac.
lcp [Fri, 17 Sep 1993 16:52:10 +0200] rev 7
Installation of new simplifier for ZF/ex. The hom_ss example in misc.ML is
particularly delicate. There is a variable renaming problem in
ramsey.ML/pigeon2_lemma. In some cases, rewriting by typechecking rules
had to be replaced by setsolver type_auto_tac... because only the solver
can instantiate variables.
lcp [Fri, 17 Sep 1993 16:16:38 +0200] rev 6
Installation of new simplifier for ZF. Deleted all congruence rules not
involving local assumptions. NB the congruence rules for Sigma and Pi
(dependent type constructions) cause difficulties and are not used by
default.
lcp [Fri, 17 Sep 1993 12:53:53 +0200] rev 5
test commit
nipkow [Thu, 16 Sep 1993 17:41:10 +0200] rev 4
added header
nipkow [Thu, 16 Sep 1993 16:55:17 +0200] rev 3
defined local addcongs
clasohm [Thu, 16 Sep 1993 16:25:32 +0200] rev 2
moved use of Thy/ROOT.ML to end of file because Thy/read.ML needs Thm
nipkow [Thu, 16 Sep 1993 14:21:44 +0200] rev 1
changed addcongs to addeqcongs in simplifier.ML
clasohm [Thu, 16 Sep 1993 12:20:38 +0200] rev 0
Initial revision