wenzelm [Wed, 11 Jan 1995 10:57:39 +0100] rev 843
removed print_sign, print_axioms;
wenzelm [Wed, 11 Jan 1995 10:53:22 +0100] rev 842
slightly changed OFCLASS syntax;
wenzelm [Mon, 02 Jan 1995 12:16:12 +0100] rev 841
fixed minor typos;
wenzelm [Mon, 02 Jan 1995 12:14:26 +0100] rev 840
added;
lcp [Fri, 23 Dec 1994 16:51:10 +0100] rev 839
RepFun_eq_0_iff, RepFun_0: new
lcp [Fri, 23 Dec 1994 16:50:22 +0100] rev 838
Moved Transset_includes_summands and Transset_sum_Int_subset
here from Ordinal.ML
lcp [Fri, 23 Dec 1994 16:49:48 +0100] rev 837
Re-indented declarations; declared the number 2
lcp [Fri, 23 Dec 1994 16:35:42 +0100] rev 836
Added Krzysztof's theorems irrefl_converse, trans_on_converse,
part_ord_converse, linear_converse, tot_ord_converse,
Proved rvimage_converse, ord_iso_rvimage_eq
lcp [Fri, 23 Dec 1994 16:35:08 +0100] rev 835
Added Krzysztof's theorems irrefl_rvimage, trans_on_rvimage,
part_ord_rvimage, tot_ord_rvimage, irrefl_Int_iff, trans_on_Int_iff,
part_ord_Int_iff, linear_Int_iff, tot_ord_Int_iff, wf_on_Int_iff,
well_ord_Int_iff
lcp [Fri, 23 Dec 1994 16:34:27 +0100] rev 834
singleton_iff: new
lcp [Fri, 23 Dec 1994 16:33:37 +0100] rev 833
Proved cons_lepoll_consD, succ_lepoll_succD, cons_eqpoll_consD,
succ_eqpoll_succD, cons_lepoll_cons_iff, cons_eqpoll_cons_iff. Deleted
inj_succ_succD. Streamlined proof of nat_lepoll_imp_le_lemma. Added
Krzysztof's theorems diff_sing_lepoll, lepoll_diff_sing, diff_sing_eqpoll,
lepoll_1_is_sing, inj_not_surj_succ, lesspoll_trans, lesspoll_lepoll_lesspoll,
lepoll_lesspoll_lesspoll, lepoll_imp_lesspoll_succ, lesspoll_succ_imp_lepoll,
lepoll_succ_disj, lepoll_nat_imp_Finite, lepoll_Finite,
Finite_imp_cons_Finite, Finite_imp_succ_Finite, nat_le_infinite_Ord,
nat_wf_on_converse_Memrel, nat_well_ord_converse_Memrel, well_ord_converse,
ordertype_eq_n, Finite_well_ord_converse
lcp [Fri, 23 Dec 1994 16:32:39 +0100] rev 832
Added Krzysztof's constants lesspoll and Finite
lcp [Fri, 23 Dec 1994 16:32:02 +0100] rev 831
Added Krzysztof's theorem pred_Memrel
lcp [Fri, 23 Dec 1994 16:31:23 +0100] rev 830
Moved Transset_includes_summands and Transset_sum_Int_subset to
QUniv.thy to eliminate use of merge_theories. Proved Memrel_type.
Added Krzysztof's theorems Memrel_mono, Memrel_empty, lt_Ord, succ_le_imp_le
lcp [Fri, 23 Dec 1994 16:30:35 +0100] rev 829
natE0: deleted, since unused
lcp [Fri, 23 Dec 1994 16:29:53 +0100] rev 828
Changed succ(1) to 2 in in_VLimit, two_in_univ
lcp [Fri, 23 Dec 1994 16:29:04 +0100] rev 827
csquare_rel_def: renamed k to K
lcp [Fri, 23 Dec 1994 16:28:26 +0100] rev 826
inj_apply_equality: new
lcp [Fri, 23 Dec 1994 16:27:45 +0100] rev 825
Added Krzysztof's theorems subst_elem, not_emptyI, not_emptyE
lcp [Fri, 23 Dec 1994 16:27:07 +0100] rev 824
empty_fun: generalized from -> to Pi
lcp [Fri, 23 Dec 1994 16:26:34 +0100] rev 823
Changed succ(1) to 2 in cmult_2; Simplified proof of InfCard_is_Limit
lcp [Fri, 23 Dec 1994 16:25:45 +0100] rev 822
Added Krzysztof's theorems singleton_eq_iff, fst_type, snd_type
Renamed doubleton_iff to doubleton_eq_iff
lcp [Fri, 23 Dec 1994 10:52:25 +0100] rev 821
Added Krzysztof's theorem disj_imp_disj
lcp [Wed, 21 Dec 1994 13:36:02 +0100] rev 820
Id: marker.
lcp [Wed, 21 Dec 1994 13:26:26 +0100] rev 819
Added comments and Id: marker.
lcp [Wed, 21 Dec 1994 13:10:39 +0100] rev 818
Added comments and Id: marker.
lcp [Wed, 21 Dec 1994 12:53:45 +0100] rev 817
Tools description, largely taken from ../README
lcp [Wed, 21 Dec 1994 12:46:52 +0100] rev 816
Moved description of tools to Tools/README
lcp [Tue, 20 Dec 1994 16:20:50 +0100] rev 815
ord_iso_rvimage: new
lcp [Tue, 20 Dec 1994 15:58:52 +0100] rev 814
Moved well_ord_Memrel, lt_eq_pred, Ord_iso_implies_eq_lemma,
Ord_iso_implies_eq to top of file, as they do not require the other
material. Simplified proof of ordertype_subset.
Proved ordertype_eq: a short proof using deepen_tac! Deleted
bij_ordermap_vimage and ordermap_Memrel
"bij_ordermap_vimage and ordermap_Memrelf. [| f: bij(A,B); well_ord(B,r); x:A |] ==>\
\ ordermap(A,rvimage(A,f,r)) ` x = ordermap(B,r) ` (f`x)";
"\ ordermap(A,rvimage(A,f,r)) ` x = ordermap(B,r) ` (f`x)";i. [| Ord(i); j:i |] ==> ordermap(i,Memrel(i)) ` j = j"
because ordertype_eq serves the same purpose. Proofs of bij_ordertype_vimage
and ordertype_Memrel are now trivial.
clasohm [Tue, 20 Dec 1994 13:24:04 +0100] rev 813
qed is a utility that makes ML files store the defined theories in Isabelle's
theorem database
lcp [Tue, 20 Dec 1994 10:21:32 +0100] rev 812
Simplified proof of ord_iso_image_pred using bij_inverse_ss.
Replaced not_well_ord_iso_pred_lemma by much simpler well_ord_iso_subset_lemma.
Simplifed proof of well_ord_iso_unique_lemma using well_ord_iso_subset_lemma.
lcp [Tue, 20 Dec 1994 10:19:24 +0100] rev 811
Used bind_thm to store domain_rel_subset and range_rel_subset
lcp [Mon, 19 Dec 1994 15:30:30 +0100] rev 810
removed quotes around "Datatype",
and removed needless mention of [Q]Univ
lcp [Mon, 19 Dec 1994 15:22:42 +0100] rev 809
removed quotes around "Inductive"
lcp [Mon, 19 Dec 1994 15:17:29 +0100] rev 808
ran expandshort script
lcp [Mon, 19 Dec 1994 15:11:50 +0100] rev 807
ran expandshort script
lcp [Mon, 19 Dec 1994 13:24:58 +0100] rev 806
removed quotes around "Inductive"
lcp [Mon, 19 Dec 1994 13:18:54 +0100] rev 805
added true theory dependencies
lcp [Mon, 19 Dec 1994 13:01:30 +0100] rev 804
ran expandshort script
lcp [Fri, 16 Dec 1994 18:07:12 +0100] rev 803
changed useless "qed" calls for lemmas back to uses of "result",
and/or used "bind_thm" to declare the real results.
lcp [Fri, 16 Dec 1994 17:46:02 +0100] rev 802
Defines ZF theory sections (inductive, datatype) at the start/
Moved theory section code here from Inductive.ML and
Datatype.ML
lcp [Fri, 16 Dec 1994 17:44:09 +0100] rev 801
Added Limit_csucc from CardinalArith
Moved all theorems concerning FINITE functions to Univ.ML
and deleted the declaration
val Fin_Univ_thy = merge_theories (Univ.thy,Finite.thy);
lcp [Fri, 16 Dec 1994 17:41:49 +0100] rev 800
Limit_csucc: moved to InfDatatype and proved explicitly in
theory InfDatatype.thy
lcp [Fri, 16 Dec 1994 17:39:43 +0100] rev 799
put quotation marks around constant "and" because it is a
keyword for inductive definitions!!
lcp [Fri, 16 Dec 1994 17:38:14 +0100] rev 798
added thy_syntax.ML
lcp [Fri, 16 Dec 1994 17:36:50 +0100] rev 797
Defines ZF theory sections (inductive, datatype) at the start/
Moved theory section code here from Inductive.ML and
Datatype.ML
lcp [Fri, 16 Dec 1994 17:32:14 +0100] rev 796
now also depends upon Finite.thy
lcp [Fri, 16 Dec 1994 13:44:48 +0100] rev 795
converse_converse, converse_prod: renamed from
converse_of_converse, converse_of_prod
lcp [Fri, 16 Dec 1994 13:43:01 +0100] rev 794
moved congruence rule conj_cong2 to FOL/IFOL.ML
lcp [Fri, 16 Dec 1994 13:30:34 +0100] rev 793
conj_cong2: new congruence rule
lcp [Thu, 15 Dec 1994 11:50:53 +0100] rev 792
case_ss: now built upon ZF/Order/bij_inverse_ss. Deleted
own bij_inverse_ss and replaces uses by case_ss
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