lcp [Thu, 15 Dec 1994 11:17:49 +0100] rev 791
updated comment;
renamed converse_of_Un to converse_Un
lcp [Thu, 15 Dec 1994 11:08:22 +0100] rev 790
qconverse_qconverse, qconverse_prod: renamed from
qconverse_of_qconverse, qconverse_of_prod
lcp [Wed, 14 Dec 1994 17:24:23 +0100] rev 789
well_ord_iso_predE replaces not_well_ord_iso_pred
well_ord_iso_unique: eliminated a premise using well_ord_ord_iso
Proved well_ord_iso_pred_eq, ord_iso_image_pred, ord_iso_restrict_pred,
part_ord_ord_iso, linear_ord_iso, wf_on_ord_iso, well_ord_ord_iso,
well_ord_iso_preserving, mono_map_is_fun, mono_map_is_inj, mono_map_trans,
mono_ord_isoI, well_ord_mono_ord_isoI, ord_iso_is_mono_map,
ord_iso_map_mono_map, ord_iso_map_ord_iso, domain_ord_iso_map_subset,
domain_ord_iso_map_cases, range_ord_iso_map_cases, well_ord_trichotomy
deleted bij_ss in favour of bij_inverse_ss
lcp [Wed, 14 Dec 1994 17:15:54 +0100] rev 788
Ord_iso_implies_eq_lemma: uses well_ord_iso_predE instead of
not_well_ord_iso_pred
lcp [Wed, 14 Dec 1994 16:57:55 +0100] rev 787
converse_UN, Diff_eq_0_iff: new
lcp [Wed, 14 Dec 1994 16:54:13 +0100] rev 786
added constants mono_map, ord_iso_map
lcp [Wed, 14 Dec 1994 16:51:16 +0100] rev 785
cardinal_UN_Ord_lt_csucc: added comment
le_UN_Ord_lt_csucc: tided proof by proving the lemma
inj_UN_subset
lcp [Wed, 14 Dec 1994 16:48:36 +0100] rev 784
conj_commute,disj_commute: new
clasohm [Wed, 14 Dec 1994 13:03:09 +0100] rev 783
changed get_thm to search all parent theories if the theorem is not found
in the current theory
clasohm [Wed, 14 Dec 1994 11:41:49 +0100] rev 782
added bind_thm for theorems defined by "standard ..."
wenzelm [Wed, 14 Dec 1994 10:26:30 +0100] rev 781
added any, sprop to pure_types;
wenzelm [Wed, 14 Dec 1994 10:24:54 +0100] rev 780
removed "logic1";
improved typ_to_nonterm;
clasohm [Tue, 13 Dec 1994 11:51:12 +0100] rev 779
removed FOL_Lemmas and IFOL_Lemmas; added qed_goal
wenzelm [Mon, 12 Dec 1994 10:26:05 +0100] rev 778
added print_theory that prints stored thms;
wenzelm [Fri, 09 Dec 1994 16:44:31 +0100] rev 777
minor internal changes;
wenzelm [Fri, 09 Dec 1994 16:42:09 +0100] rev 776
improved axioms_of: returns thms as the manual says;
clasohm [Fri, 09 Dec 1994 13:39:52 +0100] rev 775
removed ZF_Lemmas and added qed_goal
clasohm [Fri, 09 Dec 1994 13:05:03 +0100] rev 774
added warning for already stored theorem to store_thm
lcp [Thu, 08 Dec 1994 16:42:58 +0100] rev 773
sum_ss: moved down and added the rewrite rules for "case"
lcp [Thu, 08 Dec 1994 16:07:12 +0100] rev 772
leI: added comment
lcp [Thu, 08 Dec 1994 15:37:28 +0100] rev 771
lt_eq_pred, Ord_iso_implies_eq: new, for Kunens Theorem 7.3
lcp [Thu, 08 Dec 1994 15:07:48 +0100] rev 770
sum_ss: deleted because it conflicts with the one in Sum.ML
lcp [Thu, 08 Dec 1994 14:38:58 +0100] rev 769
not_well_ord_iso_pred: removed needless quantifier
lcp [Thu, 08 Dec 1994 14:18:31 +0100] rev 768
UN_upper_cardinal: updated to refer to Card_le_imp_lepoll
and lepoll_imp_Card_le
lcp [Thu, 08 Dec 1994 14:06:16 +0100] rev 767
sum_lepoll_self, cadd_le_self, prod_lepoll_self,
cmult_le_self, sum_lepoll_mono, cadd_le_mono, prod_lepoll_mono,
cmult_le_mono, InfCard_cmult_eq, cmult_2: new
well_ord_lepoll_imp_le: renamed to well_ord_lepoll_imp_Card_le
lcp [Thu, 08 Dec 1994 13:53:28 +0100] rev 766
le_imp_lepoll: renamed to Card_le_imp_lepoll
lepoll_imp_le: renamed to lepoll_imp_Card_le;
updated to refer to well_ord_lepoll_imp_Card_le
lcp [Thu, 08 Dec 1994 13:38:13 +0100] rev 765
Card_cardinal_le: new
clasohm [Thu, 08 Dec 1994 12:46:25 +0100] rev 764
changed Pure's grammar and the way types are converted to nonterminals
clasohm [Thu, 08 Dec 1994 12:45:28 +0100] rev 763
replaced type_syn by pure_syn in Pure signature
lcp [Thu, 08 Dec 1994 11:28:34 +0100] rev 762
test_assume_tac: now tries eq_assume_tac on exceptional cases
(formulae not of the form a:?A). Affects typechk_tac.
lcp [Thu, 08 Dec 1994 11:26:25 +0100] rev 761
res_inst_tac: added comments
clasohm [Wed, 07 Dec 1994 13:12:04 +0100] rev 760
added qed and qed_goal[w]
clasohm [Wed, 07 Dec 1994 12:34:47 +0100] rev 759
moved first call of store_theory from thy_read.ML to created .thy.ML file
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