Wed, 21 Dec 1994 13:10:39 +0100 Added comments and Id: marker.
lcp [Wed, 21 Dec 1994 13:10:39 +0100] rev 818
Added comments and Id: marker.
Wed, 21 Dec 1994 12:53:45 +0100 Tools description, largely taken from ../README
lcp [Wed, 21 Dec 1994 12:53:45 +0100] rev 817
Tools description, largely taken from ../README
Wed, 21 Dec 1994 12:46:52 +0100 Moved description of tools to Tools/README
lcp [Wed, 21 Dec 1994 12:46:52 +0100] rev 816
Moved description of tools to Tools/README
Tue, 20 Dec 1994 16:20:50 +0100 ord_iso_rvimage: new
lcp [Tue, 20 Dec 1994 16:20:50 +0100] rev 815
ord_iso_rvimage: new
Tue, 20 Dec 1994 15:58:52 +0100 Moved well_ord_Memrel, lt_eq_pred, Ord_iso_implies_eq_lemma,
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.
Tue, 20 Dec 1994 13:24:04 +0100 qed is a utility that makes ML files store the defined theories in Isabelle's
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
Tue, 20 Dec 1994 10:21:32 +0100 Simplified proof of ord_iso_image_pred using bij_inverse_ss.
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.
Tue, 20 Dec 1994 10:19:24 +0100 Used bind_thm to store domain_rel_subset and range_rel_subset
lcp [Tue, 20 Dec 1994 10:19:24 +0100] rev 811
Used bind_thm to store domain_rel_subset and range_rel_subset
Mon, 19 Dec 1994 15:30:30 +0100 removed quotes around "Datatype",
lcp [Mon, 19 Dec 1994 15:30:30 +0100] rev 810
removed quotes around "Datatype", and removed needless mention of [Q]Univ
Mon, 19 Dec 1994 15:22:42 +0100 removed quotes around "Inductive"
lcp [Mon, 19 Dec 1994 15:22:42 +0100] rev 809
removed quotes around "Inductive"
Mon, 19 Dec 1994 15:17:29 +0100 ran expandshort script
lcp [Mon, 19 Dec 1994 15:17:29 +0100] rev 808
ran expandshort script
Mon, 19 Dec 1994 15:11:50 +0100 ran expandshort script
lcp [Mon, 19 Dec 1994 15:11:50 +0100] rev 807
ran expandshort script
Mon, 19 Dec 1994 13:24:58 +0100 removed quotes around "Inductive"
lcp [Mon, 19 Dec 1994 13:24:58 +0100] rev 806
removed quotes around "Inductive"
Mon, 19 Dec 1994 13:18:54 +0100 added true theory dependencies
lcp [Mon, 19 Dec 1994 13:18:54 +0100] rev 805
added true theory dependencies
Mon, 19 Dec 1994 13:01:30 +0100 ran expandshort script
lcp [Mon, 19 Dec 1994 13:01:30 +0100] rev 804
ran expandshort script
Fri, 16 Dec 1994 18:07:12 +0100 changed useless "qed" calls for lemmas back to uses of "result",
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.
Fri, 16 Dec 1994 17:46:02 +0100 Defines ZF theory sections (inductive, datatype) at the start/
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
Fri, 16 Dec 1994 17:44:09 +0100 Added Limit_csucc from CardinalArith
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);
Fri, 16 Dec 1994 17:41:49 +0100 Limit_csucc: moved to InfDatatype and proved explicitly in
lcp [Fri, 16 Dec 1994 17:41:49 +0100] rev 800
Limit_csucc: moved to InfDatatype and proved explicitly in theory InfDatatype.thy
Fri, 16 Dec 1994 17:39:43 +0100 put quotation marks around constant "and" because it is a
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!!
Fri, 16 Dec 1994 17:38:14 +0100 added thy_syntax.ML
lcp [Fri, 16 Dec 1994 17:38:14 +0100] rev 798
added thy_syntax.ML
Fri, 16 Dec 1994 17:36:50 +0100 Defines ZF theory sections (inductive, datatype) at the start/
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
Fri, 16 Dec 1994 17:32:14 +0100 now also depends upon Finite.thy
lcp [Fri, 16 Dec 1994 17:32:14 +0100] rev 796
now also depends upon Finite.thy
Fri, 16 Dec 1994 13:44:48 +0100 converse_converse, converse_prod: renamed from
lcp [Fri, 16 Dec 1994 13:44:48 +0100] rev 795
converse_converse, converse_prod: renamed from converse_of_converse, converse_of_prod
Fri, 16 Dec 1994 13:43:01 +0100 moved congruence rule conj_cong2 to FOL/IFOL.ML
lcp [Fri, 16 Dec 1994 13:43:01 +0100] rev 794
moved congruence rule conj_cong2 to FOL/IFOL.ML
Fri, 16 Dec 1994 13:30:34 +0100 conj_cong2: new congruence rule
lcp [Fri, 16 Dec 1994 13:30:34 +0100] rev 793
conj_cong2: new congruence rule
Thu, 15 Dec 1994 11:50:53 +0100 case_ss: now built upon ZF/Order/bij_inverse_ss. Deleted
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
Thu, 15 Dec 1994 11:17:49 +0100 updated comment;
lcp [Thu, 15 Dec 1994 11:17:49 +0100] rev 791
updated comment; renamed converse_of_Un to converse_Un
Thu, 15 Dec 1994 11:08:22 +0100 qconverse_qconverse, qconverse_prod: renamed from
lcp [Thu, 15 Dec 1994 11:08:22 +0100] rev 790
qconverse_qconverse, qconverse_prod: renamed from qconverse_of_qconverse, qconverse_of_prod
Wed, 14 Dec 1994 17:24:23 +0100 well_ord_iso_predE replaces not_well_ord_iso_pred
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
Wed, 14 Dec 1994 17:15:54 +0100 Ord_iso_implies_eq_lemma: uses well_ord_iso_predE instead of
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
Wed, 14 Dec 1994 16:57:55 +0100 converse_UN, Diff_eq_0_iff: new
lcp [Wed, 14 Dec 1994 16:57:55 +0100] rev 787
converse_UN, Diff_eq_0_iff: new
Wed, 14 Dec 1994 16:54:13 +0100 added constants mono_map, ord_iso_map
lcp [Wed, 14 Dec 1994 16:54:13 +0100] rev 786
added constants mono_map, ord_iso_map
Wed, 14 Dec 1994 16:51:16 +0100 cardinal_UN_Ord_lt_csucc: added comment
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
Wed, 14 Dec 1994 16:48:36 +0100 conj_commute,disj_commute: new
lcp [Wed, 14 Dec 1994 16:48:36 +0100] rev 784
conj_commute,disj_commute: new
Wed, 14 Dec 1994 13:03:09 +0100 changed get_thm to search all parent theories if the theorem is not found
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
Wed, 14 Dec 1994 11:41:49 +0100 added bind_thm for theorems defined by "standard ..."
clasohm [Wed, 14 Dec 1994 11:41:49 +0100] rev 782
added bind_thm for theorems defined by "standard ..."
Wed, 14 Dec 1994 10:26:30 +0100 added any, sprop to pure_types;
wenzelm [Wed, 14 Dec 1994 10:26:30 +0100] rev 781
added any, sprop to pure_types;
Wed, 14 Dec 1994 10:24:54 +0100 removed "logic1";
wenzelm [Wed, 14 Dec 1994 10:24:54 +0100] rev 780
removed "logic1"; improved typ_to_nonterm;
Tue, 13 Dec 1994 11:51:12 +0100 removed FOL_Lemmas and IFOL_Lemmas; added qed_goal
clasohm [Tue, 13 Dec 1994 11:51:12 +0100] rev 779
removed FOL_Lemmas and IFOL_Lemmas; added qed_goal
Mon, 12 Dec 1994 10:26:05 +0100 added print_theory that prints stored thms;
wenzelm [Mon, 12 Dec 1994 10:26:05 +0100] rev 778
added print_theory that prints stored thms;
Fri, 09 Dec 1994 16:44:31 +0100 minor internal changes;
wenzelm [Fri, 09 Dec 1994 16:44:31 +0100] rev 777
minor internal changes;
Fri, 09 Dec 1994 16:42:09 +0100 improved axioms_of: returns thms as the manual says;
wenzelm [Fri, 09 Dec 1994 16:42:09 +0100] rev 776
improved axioms_of: returns thms as the manual says;
Fri, 09 Dec 1994 13:39:52 +0100 removed ZF_Lemmas and added qed_goal
clasohm [Fri, 09 Dec 1994 13:39:52 +0100] rev 775
removed ZF_Lemmas and added qed_goal
Fri, 09 Dec 1994 13:05:03 +0100 added warning for already stored theorem to store_thm
clasohm [Fri, 09 Dec 1994 13:05:03 +0100] rev 774
added warning for already stored theorem to store_thm
Thu, 08 Dec 1994 16:42:58 +0100 sum_ss: moved down and added the rewrite rules for "case"
lcp [Thu, 08 Dec 1994 16:42:58 +0100] rev 773
sum_ss: moved down and added the rewrite rules for "case"
Thu, 08 Dec 1994 16:07:12 +0100 leI: added comment
lcp [Thu, 08 Dec 1994 16:07:12 +0100] rev 772
leI: added comment
Thu, 08 Dec 1994 15:37:28 +0100 lt_eq_pred, Ord_iso_implies_eq: new, for Kunens Theorem 7.3
lcp [Thu, 08 Dec 1994 15:37:28 +0100] rev 771
lt_eq_pred, Ord_iso_implies_eq: new, for Kunens Theorem 7.3
(0) -300 -100 -48 +48 +100 +300 +1000 +3000 +10000 +30000 tip