clasohm [Tue, 06 Dec 1994 12:50:13 +0100] rev 758
added bind_thm
clasohm [Wed, 30 Nov 1994 13:53:46 +0100] rev 757
added qed and qed_goal[w]
clasohm [Wed, 30 Nov 1994 13:18:42 +0100] rev 756
added qed_goal for meta_iffD
clasohm [Wed, 30 Nov 1994 13:13:52 +0100] rev 755
replaced "val ... = result()" by "qed ..."
lcp [Tue, 29 Nov 1994 11:51:07 +0100] rev 754
le_UN_Ord_lt_csucc: added comment
lcp [Tue, 29 Nov 1994 00:31:31 +0100] rev 753
replaced "rules" by "defs"
regensbu [Mon, 28 Nov 1994 19:48:30 +0100] rev 752
----------------------------------------------------------------------
Committing in HOLCF
Use new translation mechanism and keyword syntax, cinfix.ML no
longer needed.
Optimized proofs in Cont.ML
Modified Files:
Cfun1.ML Cfun2.thy Cont.ML Cprod3.thy Makefile README
Sprod3.thy Tr2.thy ccc1.thy
----------------------------------------------------------------------
lcp [Fri, 25 Nov 1994 11:13:55 +0100] rev 751
ZF/indrule/mutual_ind_tac: ensured that asm_full_simp_tac ignores any
equalities, by adding setmksimps K[].
ZF/indrule/mut_ss: removed Collect_cong; it is redundant.
lcp [Fri, 25 Nov 1994 11:08:12 +0100] rev 750
checks that the recursive sets are Consts before taking
them apart! Bug was introduced during the translation to theory sections.
lcp [Fri, 25 Nov 1994 11:04:44 +0100] rev 749
equiv_comp_eq: simplified proof
lcp [Fri, 25 Nov 1994 11:02:39 +0100] rev 748
moved Cantors theorem here from ZF/ex/misc
lcp [Fri, 25 Nov 1994 10:43:50 +0100] rev 747
deepen_tac: modified due to outcome of experiments. Its
choice of unsafe rule to expand is still non-deterministic.
clasohm [Fri, 25 Nov 1994 09:13:49 +0100] rev 746
added qed_goal[w]
lcp [Fri, 25 Nov 1994 00:02:37 +0100] rev 745
added blank line
lcp [Fri, 25 Nov 1994 00:01:04 +0100] rev 744
tidied proofs, using fast_tac etc. as much as possible
lcp [Fri, 25 Nov 1994 00:00:35 +0100] rev 743
prove_fun: new; no longer depends upon the version in simpdata.ML
lcp [Thu, 24 Nov 1994 10:57:24 +0100] rev 742
data_domain,Codata_domain: removed replicate; now return one
single domain
lcp [Thu, 24 Nov 1994 10:53:46 +0100] rev 741
tidied proofs, using fast_tac etc. as much as possible
lcp [Thu, 24 Nov 1994 10:47:45 +0100] rev 740
added comments on alternative uses of type_intrs/elims
lcp [Thu, 24 Nov 1994 10:38:08 +0100] rev 739
modified for new treatment of mutual recursion
lcp [Thu, 24 Nov 1994 10:31:47 +0100] rev 738
the_equality: more careful use of addSIs and addIs
lcp [Thu, 24 Nov 1994 10:23:41 +0100] rev 737
cons_fun_eq: modified strange uses of classical reasoner
lcp [Thu, 24 Nov 1994 00:33:13 +0100] rev 736
moved Cantors theorem to ZF/ZF.ML and ZF/Perm.ML
hom_tac: removed to simplify the proof of comp_homs
lcp [Thu, 24 Nov 1994 00:32:43 +0100] rev 735
moved version of Cantors theorem to ZF/Perm.ML
lcp [Thu, 24 Nov 1994 00:32:12 +0100] rev 734
ZF INDUCTIVE DEFINITIONS: Simplifying the type checking for mutually
recursive datatypes, especially with monotone operators
Inductive_Fun,CoInductive_Fun: deleted as obsolete
inductive_decl: now reads a SINGLE domain for the mutually
recursive construction. This could be a sum, perhaps not! CONCRETE SYNTAX
has changed too (but there are no examples of this to change).
lcp [Thu, 24 Nov 1994 00:31:41 +0100] rev 733
ZF/Datatype/datatype_decl: supplies a SINGLE domain for the mutually
recursive construction. This is [q]univ(A), which is closed under sum.
lcp [Thu, 24 Nov 1994 00:31:08 +0100] rev 732
updated for new deepen_tac
lcp [Thu, 24 Nov 1994 00:30:35 +0100] rev 731
trivial changes
lcp [Wed, 23 Nov 1994 11:45:56 +0100] rev 730
new reference to HO patterns
lcp [Tue, 22 Nov 1994 23:32:16 +0100] rev 729
Pure/tctical/protect_subgoal: simplified to use Sequence.hd
Pure/tctical/DEPTH_FIRST: now suppresses duplicate solutions
lcp [Tue, 22 Nov 1994 23:30:49 +0100] rev 728
Pure/term: commented typ_subst_TVars, subst_TVars, subst_Vars, subst_vars
lcp [Mon, 21 Nov 1994 18:48:03 +0100] rev 727
ZF INDUCTIVE DEFINITIONS: Simplifying the type checking for mutually
recursive datatypes, especially with monotone operators
ZF/add_ind_def/add_fp_def: deleted as obsolete
ZF/add_ind_def/add_fp_def_i: now takes dom_sum instead of domts. We no
longer automatically construct a sum of separate domains, but could use a
sum-closed set such as univ(A).
lcp [Mon, 21 Nov 1994 15:53:02 +0100] rev 726
ZF/intr_elim/elim: now "folds" definitions of the mutually recursive sets!
clasohm [Mon, 21 Nov 1994 14:11:21 +0100] rev 725
replaced 'val ... = result();' by 'qed "...";'
lcp [Mon, 21 Nov 1994 14:06:59 +0100] rev 724
ZF/indrule/mutual_ind_tac: backtracks using DEPTH_SOLVE to be certain of
solving the subgoal. Entire tactic is enclosed in DETERM to prevent
backtracking between subgoals.
lcp [Mon, 21 Nov 1994 13:47:00 +0100] rev 723
ZF/EquivClass/congruent_commuteI: uncommented and simplified proof
lcp [Mon, 21 Nov 1994 13:09:41 +0100] rev 722
ZF/ZF.ML/UN_iff, INT_iff: added to the signature
lcp [Mon, 21 Nov 1994 11:49:36 +0100] rev 721
Pure/thm/norm_term_skip: new, for skipping normalization of the context
Pure/thm/bicompose_aux: now computes nlift (number of lifted assumptions in
new subgoals) and avoids normalizing the first nlift assumptions in the
case where the proof state is not affected.
Pure/thm/norm_term_skip: now normalizes types of parameters
Pure/thm/THM: aligned colons
lcp [Mon, 21 Nov 1994 11:33:23 +0100] rev 720
Pure/sequence: added comment explaining that memoing sequences were found
to be much slower (due to overheads) than the sequences currently used.
lcp [Mon, 21 Nov 1994 11:27:10 +0100] rev 719
Pure/envir/norm_term: replaced equality test for [] by null
lcp [Mon, 21 Nov 1994 10:51:40 +0100] rev 718
page 157 erratum
lcp [Mon, 21 Nov 1994 10:39:32 +0100] rev 717
now searches all subdirectories of object-logics
whether or not they are called "ex"
nipkow [Fri, 18 Nov 1994 13:14:23 +0100] rev 716
Chnaged simplifier description (lhss)
clasohm [Fri, 18 Nov 1994 13:08:10 +0100] rev 715
added call of store_theory after thy file has been read
nipkow [Fri, 18 Nov 1994 13:04:51 +0100] rev 714
Updated description of valid lhss.
lcp [Thu, 17 Nov 1994 22:01:08 +0100] rev 713
In ZF, type i has class term, not (just) logic
clasohm [Mon, 14 Nov 1994 14:47:20 +0100] rev 712
added check for newlines not enclosed by '\' inside strings
clasohm [Mon, 14 Nov 1994 14:29:20 +0100] rev 711
updated remarks about grammar; added section about ambiguities
wenzelm [Mon, 14 Nov 1994 11:57:32 +0100] rev 710
exported 'cat';
lcp [Mon, 14 Nov 1994 10:49:39 +0100] rev 709
Pure/tctical/select: now uses cprems_of instead of prems_of and cterm_of:
new SELECT_GOAL is MUCH faster
lcp [Mon, 14 Nov 1994 10:46:50 +0100] rev 708
Pure/drule/cprems_of, cskip_flexpairs, cstrip_imp_prems: new cterm operations
lcp [Mon, 14 Nov 1994 10:41:25 +0100] rev 707
Added month for Coens thesis
lcp [Fri, 11 Nov 1994 10:53:41 +0100] rev 706
removal of FOL_dup_cs
lcp [Fri, 11 Nov 1994 10:50:49 +0100] rev 705
removal of HOL_dup_cs
rotation of arguments in split, nat_case, sum_case, list_case
lcp [Fri, 11 Nov 1994 10:42:55 +0100] rev 704
Provers/hypsubst/REPEATN: deleted; using REPEAT_DETERM_N instead.
lcp [Fri, 11 Nov 1994 10:41:09 +0100] rev 703
Pure/tctical/REPEAT_DETERM_N,REPEAT_DETERM1,REPEAT_DETERM_FIRST,
REPEAT_DETERM_SOME: new
lcp [Fri, 11 Nov 1994 10:33:05 +0100] rev 702
FOL/intprover/safe_tac: now uses REPEAT_DETERM_FIRST instead of REPEAT_DETERM
lcp [Fri, 11 Nov 1994 10:31:51 +0100] rev 701
argument swaps in HOL
lcp [Thu, 10 Nov 1994 11:36:40 +0100] rev 700
HOL,ZF/Makefile: enclosed multiple "use" calls in parentheses. This
ensures that if one dies, all die. BUT NOT Pure/Makefile, where
PolyML.use"POLY" makes the identifier "use" visible.
lcp [Thu, 10 Nov 1994 11:06:44 +0100] rev 699
updated pathnames