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