Wed, 29 Apr 1998 11:39:52 +0200 renamed from typedef.ML;
wenzelm [Wed, 29 Apr 1998 11:39:52 +0200] rev 4866
renamed from typedef.ML;
Wed, 29 Apr 1998 11:39:28 +0200 reworked and moved to Tools/record_package.ML;
wenzelm [Wed, 29 Apr 1998 11:39:28 +0200] rev 4865
reworked and moved to Tools/record_package.ML;
Wed, 29 Apr 1998 11:38:52 +0200 removed typedef.ML, record.ML;
wenzelm [Wed, 29 Apr 1998 11:38:52 +0200] rev 4864
removed typedef.ML, record.ML; added Tools/typedef_package.ML, Tools/record_package.ML, Record.thy;
Wed, 29 Apr 1998 11:37:58 +0200 renamed to Tools/typedef_package.ML;
wenzelm [Wed, 29 Apr 1998 11:37:58 +0200] rev 4863
renamed to Tools/typedef_package.ML;
Wed, 29 Apr 1998 11:36:53 +0200 adapted to new PureThy.add_axioms_i;
wenzelm [Wed, 29 Apr 1998 11:36:53 +0200] rev 4862
adapted to new PureThy.add_axioms_i; Theory.parent_path;
Wed, 29 Apr 1998 11:36:08 +0200 adapted to new PureThy.add_tthmss;
wenzelm [Wed, 29 Apr 1998 11:36:08 +0200] rev 4861
adapted to new PureThy.add_tthmss; Theory.parent_path;
Wed, 29 Apr 1998 11:35:24 +0200 Theory.require;
wenzelm [Wed, 29 Apr 1998 11:35:24 +0200] rev 4860
Theory.require; Logic.mk_defpair; adapted to new PureThy.add_defs_i;
Wed, 29 Apr 1998 11:34:11 +0200 adapted to new PureThy.add_axioms;
wenzelm [Wed, 29 Apr 1998 11:34:11 +0200] rev 4859
adapted to new PureThy.add_axioms;
Wed, 29 Apr 1998 11:33:44 +0200 new theory section 'nonterminals';
wenzelm [Wed, 29 Apr 1998 11:33:44 +0200] rev 4858
new theory section 'nonterminals';
Wed, 29 Apr 1998 11:33:27 +0200 adapted to new PureThy.add_defs;
wenzelm [Wed, 29 Apr 1998 11:33:27 +0200] rev 4857
adapted to new PureThy.add_defs;
Wed, 29 Apr 1998 11:33:06 +0200 Theory.require;
wenzelm [Wed, 29 Apr 1998 11:33:06 +0200] rev 4856
Theory.require;
Wed, 29 Apr 1998 11:30:55 +0200 tuned setup;
wenzelm [Wed, 29 Apr 1998 11:30:55 +0200] rev 4855
tuned setup; simp_add_global, simp_del_global, simp_add_local, simp_del_local attributes;
Wed, 29 Apr 1998 11:29:39 +0200 tuned setup;
wenzelm [Wed, 29 Apr 1998 11:29:39 +0200] rev 4854
tuned setup;
Wed, 29 Apr 1998 11:29:00 +0200 tuned names of (add_)store_XXX functions;
wenzelm [Wed, 29 Apr 1998 11:29:00 +0200] rev 4853
tuned names of (add_)store_XXX functions; added attributes to add_thms, add_axioms, add_defs functions;
Wed, 29 Apr 1998 11:26:59 +0200 replaced thy_setup by 'setup' section;
wenzelm [Wed, 29 Apr 1998 11:26:59 +0200] rev 4852
replaced thy_setup by 'setup' section; adapted to new PureThy.add_axioms / PureThy.add_defs; added 'nonterminals' section;
Wed, 29 Apr 1998 11:25:26 +0200 added append;
wenzelm [Wed, 29 Apr 1998 11:25:26 +0200] rev 4851
added append;
Wed, 29 Apr 1998 11:24:58 +0200 added none: 'a -> 'a * 'b attribute list;
wenzelm [Wed, 29 Apr 1998 11:24:58 +0200] rev 4850
added none: 'a -> 'a * 'b attribute list; added no_attrs: 'a * 'b -> ('a * ('b * tag list)) * 'c attribute list; added no_attrss: 'a * 'b list -> ('a * ('b * tag list) list) * 'c attribute list; added applys: ('a * tthm list) * 'a attribute list -> ('a * tthm list);
Wed, 29 Apr 1998 11:22:52 +0200 tuned error msgs;
wenzelm [Wed, 29 Apr 1998 11:22:52 +0200] rev 4849
tuned error msgs;
Wed, 29 Apr 1998 11:22:01 +0200 moved mk_defpair to logic.ML;
wenzelm [Wed, 29 Apr 1998 11:22:01 +0200] rev 4848
moved mk_defpair to logic.ML; moved get_def to thm.ML; moved require_thy to theory.ML;
Wed, 29 Apr 1998 11:20:53 +0200 tuned get_ax (uses ancestry);
wenzelm [Wed, 29 Apr 1998 11:20:53 +0200] rev 4847
tuned get_ax (uses ancestry); added get_def: theory -> xstring -> thm;
Wed, 29 Apr 1998 11:17:14 +0200 renamed setup to apply;
wenzelm [Wed, 29 Apr 1998 11:17:14 +0200] rev 4846
renamed setup to apply; added add_nonterminals: bstring list -> theory -> theory; added parent_path: theory -> theory; added root_path: theory -> theory; added require: theory -> string -> string -> unit (from section_utils.ML);
Wed, 29 Apr 1998 11:14:34 +0200 adapted to new PureThy.add_axioms_i;
wenzelm [Wed, 29 Apr 1998 11:14:34 +0200] rev 4845
adapted to new PureThy.add_axioms_i;
Wed, 29 Apr 1998 11:13:22 +0200 added defaultS: sg -> sort;
wenzelm [Wed, 29 Apr 1998 11:13:22 +0200] rev 4844
added defaultS: sg -> sort; added full_name_path: sg -> string -> bstring -> string; added add_nonterminals: bstring list -> sg -> sg;
Wed, 29 Apr 1998 11:11:36 +0200 added thm, thms;
wenzelm [Wed, 29 Apr 1998 11:11:36 +0200] rev 4843
added thm, thms;
Wed, 29 Apr 1998 11:10:40 +0200 *** empty log message ***
wenzelm [Wed, 29 Apr 1998 11:10:40 +0200] rev 4842
*** empty log message ***
Tue, 28 Apr 1998 13:52:18 +0200 new thms, really demos of the final coalgebra theorem
paulson [Tue, 28 Apr 1998 13:52:18 +0200] rev 4841
new thms, really demos of the final coalgebra theorem
Tue, 28 Apr 1998 13:51:39 +0200 new thms image_0_left, image_Un_left, etc.
paulson [Tue, 28 Apr 1998 13:51:39 +0200] rev 4840
new thms image_0_left, image_Un_left, etc.
Tue, 28 Apr 1998 13:50:41 +0200 new thm mult_lt_mono1
paulson [Tue, 28 Apr 1998 13:50:41 +0200] rev 4839
new thm mult_lt_mono1
Mon, 27 Apr 1998 19:32:19 +0200 cleanup for split_all_tac as wrapper in claset()
oheimb [Mon, 27 Apr 1998 19:32:19 +0200] rev 4838
cleanup for split_all_tac as wrapper in claset()
Mon, 27 Apr 1998 19:30:40 +0200 removed wrong comment
oheimb [Mon, 27 Apr 1998 19:30:40 +0200] rev 4837
removed wrong comment
Mon, 27 Apr 1998 19:29:19 +0200 added option_map_eq_Some via AddIffs
oheimb [Mon, 27 Apr 1998 19:29:19 +0200] rev 4836
added option_map_eq_Some via AddIffs
Mon, 27 Apr 1998 18:06:22 +0200 *** empty log message ***
nipkow [Mon, 27 Apr 1998 18:06:22 +0200] rev 4835
*** empty log message ***
Mon, 27 Apr 1998 17:52:03 +0200 delsplits, Addsplits, Delsplits.
nipkow [Mon, 27 Apr 1998 17:52:03 +0200] rev 4834
delsplits, Addsplits, Delsplits.
Mon, 27 Apr 1998 16:47:50 +0200 Renamed expand_const -> split_const
nipkow [Mon, 27 Apr 1998 16:47:50 +0200] rev 4833
Renamed expand_const -> split_const
Mon, 27 Apr 1998 16:46:56 +0200 Added conversion of reg.expr. to automata.
nipkow [Mon, 27 Apr 1998 16:46:56 +0200] rev 4832
Added conversion of reg.expr. to automata. Renamed expand_const -> split_const.
Mon, 27 Apr 1998 16:45:27 +0200 Renamed expand_const -> split_const.
nipkow [Mon, 27 Apr 1998 16:45:27 +0200] rev 4831
Renamed expand_const -> split_const.
Mon, 27 Apr 1998 16:45:11 +0200 Added a few lemmas.
nipkow [Mon, 27 Apr 1998 16:45:11 +0200] rev 4830
Added a few lemmas. Renamed expand_const -> split_const.
Mon, 27 Apr 1998 13:47:46 +0200 New proof of apply_equality and new thm Pi_image_cons
paulson [Mon, 27 Apr 1998 13:47:46 +0200] rev 4829
New proof of apply_equality and new thm Pi_image_cons
Fri, 24 Apr 1998 16:18:39 +0200 improved split_all_tac significantly
oheimb [Fri, 24 Apr 1998 16:18:39 +0200] rev 4828
improved split_all_tac significantly
Fri, 24 Apr 1998 16:16:29 +0200 improved keyboard modifiers
oheimb [Fri, 24 Apr 1998 16:16:29 +0200] rev 4827
improved keyboard modifiers
Fri, 24 Apr 1998 16:15:34 +0200 added ASCII translation of subseteq
oheimb [Fri, 24 Apr 1998 16:15:34 +0200] rev 4826
added ASCII translation of subseteq
Fri, 24 Apr 1998 13:06:17 +0200 tidied; div & mod
paulson [Fri, 24 Apr 1998 13:06:17 +0200] rev 4825
tidied; div & mod
Fri, 24 Apr 1998 11:22:39 +0200 *** empty log message ***
oheimb [Fri, 24 Apr 1998 11:22:39 +0200] rev 4824
*** empty log message ***
Wed, 22 Apr 1998 19:09:44 +0200 added no_syn;
wenzelm [Wed, 22 Apr 1998 19:09:44 +0200] rev 4823
added no_syn;
Wed, 22 Apr 1998 19:08:49 +0200 added mk_cond_defpair, mk_defpair;
wenzelm [Wed, 22 Apr 1998 19:08:49 +0200] rev 4822
added mk_cond_defpair, mk_defpair;
Wed, 22 Apr 1998 14:06:05 +0200 Modifications due to improved simplifier.
nipkow [Wed, 22 Apr 1998 14:06:05 +0200] rev 4821
Modifications due to improved simplifier.
Wed, 22 Apr 1998 14:04:35 +0200 Tried to speed up the rewriter by eta-contracting all patterns beforehand and
nipkow [Wed, 22 Apr 1998 14:04:35 +0200] rev 4820
Tried to speed up the rewriter by eta-contracting all patterns beforehand and by classifying each pattern as to whether it allows first-order matching.
Tue, 21 Apr 1998 17:25:19 +0200 improved pair_tac to call prune_params_tac afterwards
oheimb [Tue, 21 Apr 1998 17:25:19 +0200] rev 4819
improved pair_tac to call prune_params_tac afterwards improved the (bad) efficiency of split_all_tac by about 50% split_all_tac is now added to claset() _before_ other safe tactics
Tue, 21 Apr 1998 17:23:24 +0200 split_all_tac is now added to claset() _before_ other safe tactics
oheimb [Tue, 21 Apr 1998 17:23:24 +0200] rev 4818
split_all_tac is now added to claset() _before_ other safe tactics
Tue, 21 Apr 1998 17:22:47 +0200 made proof of zmult_congruent2 more stable
oheimb [Tue, 21 Apr 1998 17:22:47 +0200] rev 4817
made proof of zmult_congruent2 more stable
Tue, 21 Apr 1998 17:22:03 +0200 simplification of explicit theory usage and merges
oheimb [Tue, 21 Apr 1998 17:22:03 +0200] rev 4816
simplification of explicit theory usage and merges
Tue, 21 Apr 1998 17:21:42 +0200 removed split_all_tac from claset() globally within IOA
oheimb [Tue, 21 Apr 1998 17:21:42 +0200] rev 4815
removed split_all_tac from claset() globally within IOA
Tue, 21 Apr 1998 17:20:54 +0200 made modifications of the simpset() local
oheimb [Tue, 21 Apr 1998 17:20:54 +0200] rev 4814
made modifications of the simpset() local significantly simplified (and stabilized) proof of is_asig_of_rename
Tue, 21 Apr 1998 17:20:28 +0200 layout improvement
oheimb [Tue, 21 Apr 1998 17:20:28 +0200] rev 4813
layout improvement
Tue, 21 Apr 1998 10:49:15 +0200 expandshort; new gcd_induct with inbuilt case analysis
paulson [Tue, 21 Apr 1998 10:49:15 +0200] rev 4812
expandshort; new gcd_induct with inbuilt case analysis
Tue, 21 Apr 1998 10:47:58 +0200 Renamed mod_XXX_cancel to mod_XXX_self
paulson [Tue, 21 Apr 1998 10:47:58 +0200] rev 4811
Renamed mod_XXX_cancel to mod_XXX_self Included their div_ equivalents
Mon, 20 Apr 1998 10:38:30 +0200 New laws for mod
paulson [Mon, 20 Apr 1998 10:38:30 +0200] rev 4810
New laws for mod
Mon, 20 Apr 1998 10:37:00 +0200 proving fib(gcd(m,n)) = gcd(fib m, fib n)
paulson [Mon, 20 Apr 1998 10:37:00 +0200] rev 4809
proving fib(gcd(m,n)) = gcd(fib m, fib n)
Sun, 19 Apr 1998 17:01:04 +0200 fixed comment;
wenzelm [Sun, 19 Apr 1998 17:01:04 +0200] rev 4808
fixed comment;
Fri, 10 Apr 1998 13:42:22 +0200 Fixed bug in inductive sections to allow disjunctive premises;
paulson [Fri, 10 Apr 1998 13:42:22 +0200] rev 4807
Fixed bug in inductive sections to allow disjunctive premises; added tracing flag trace_induct
Fri, 10 Apr 1998 13:41:04 +0200 bug fixes
paulson [Fri, 10 Apr 1998 13:41:04 +0200] rev 4806
bug fixes
Fri, 10 Apr 1998 13:40:29 +0200 can prove the empty relation to be WF
paulson [Fri, 10 Apr 1998 13:40:29 +0200] rev 4805
can prove the empty relation to be WF
Fri, 10 Apr 1998 13:15:28 +0200 Fixed bug in inductive sections to allow disjunctive premises;
paulson [Fri, 10 Apr 1998 13:15:28 +0200] rev 4804
Fixed bug in inductive sections to allow disjunctive premises; added tracing flag trace_induct
Thu, 09 Apr 1998 12:31:35 +0200 Clearer description of recdef, including use of {}
paulson [Thu, 09 Apr 1998 12:31:35 +0200] rev 4803
Clearer description of recdef, including use of {}
Thu, 09 Apr 1998 12:29:39 +0200 Simplified the syntax description; mentioned FOL vs HOL
paulson [Thu, 09 Apr 1998 12:29:39 +0200] rev 4802
Simplified the syntax description; mentioned FOL vs HOL
Tue, 07 Apr 1998 13:46:34 +0200 *** empty log message ***
oheimb [Tue, 07 Apr 1998 13:46:34 +0200] rev 4801
*** empty log message ***
Tue, 07 Apr 1998 13:46:05 +0200 replaced option_map_SomeD by option_map_eq_Some (RS iffD1)
oheimb [Tue, 07 Apr 1998 13:46:05 +0200] rev 4800
replaced option_map_SomeD by option_map_eq_Some (RS iffD1) added option_map_eq_Some to simpset(), option_map_eq_Some RS iffD1 to claset()
Tue, 07 Apr 1998 13:43:07 +0200 made split_all_tac as safe wrapper more defensive:
oheimb [Tue, 07 Apr 1998 13:43:07 +0200] rev 4799
made split_all_tac as safe wrapper more defensive: if it is added as unsafe wrapper again (as its was before), this does not break the current proofs.
Sat, 04 Apr 1998 14:30:19 +0200 no open Simplifier;
wenzelm [Sat, 04 Apr 1998 14:30:19 +0200] rev 4798
no open Simplifier;
Sat, 04 Apr 1998 14:27:11 +0200 tuned fail;
wenzelm [Sat, 04 Apr 1998 14:27:11 +0200] rev 4797
tuned fail;
Sat, 04 Apr 1998 12:31:35 +0200 type_error;
wenzelm [Sat, 04 Apr 1998 12:31:35 +0200] rev 4796
type_error; replaced thy_data by setup;
Sat, 04 Apr 1998 12:30:17 +0200 tuned comments;
wenzelm [Sat, 04 Apr 1998 12:30:17 +0200] rev 4795
tuned comments; BasicSimplifier made pervasive; added simp tags / attributes; replaced thy_data by setup;
Sat, 04 Apr 1998 12:29:07 +0200 no open Simplifier;
wenzelm [Sat, 04 Apr 1998 12:29:07 +0200] rev 4794
no open Simplifier;
Sat, 04 Apr 1998 12:28:39 +0200 replaced thy_data by thy_setup;
wenzelm [Sat, 04 Apr 1998 12:28:39 +0200] rev 4793
replaced thy_data by thy_setup;
Sat, 04 Apr 1998 12:26:47 +0200 type_error;
wenzelm [Sat, 04 Apr 1998 12:26:47 +0200] rev 4792
type_error;
Sat, 04 Apr 1998 11:44:16 +0200 replaced thy_data by setup;
wenzelm [Sat, 04 Apr 1998 11:44:16 +0200] rev 4791
replaced thy_data by setup;
Sat, 04 Apr 1998 11:43:39 +0200 removed simple;
wenzelm [Sat, 04 Apr 1998 11:43:39 +0200] rev 4790
removed simple; added fail, untag;
Sat, 04 Apr 1998 11:42:48 +0200 added triv_goal, rev_triv_goal (for Isar);
wenzelm [Sat, 04 Apr 1998 11:42:48 +0200] rev 4789
added triv_goal, rev_triv_goal (for Isar);
Sat, 04 Apr 1998 11:42:26 +0200 added Goal_def;
wenzelm [Sat, 04 Apr 1998 11:42:26 +0200] rev 4788
added Goal_def;
Sat, 04 Apr 1998 11:41:24 +0200 replaced thy_data by thy_setup;
wenzelm [Sat, 04 Apr 1998 11:41:24 +0200] rev 4787
replaced thy_data by thy_setup;
Sat, 04 Apr 1998 11:41:00 +0200 added local_theory (for Isar);
wenzelm [Sat, 04 Apr 1998 11:41:00 +0200] rev 4786
added local_theory (for Isar); added setup;
Sat, 04 Apr 1998 11:40:18 +0200 tuned trace msgs;
wenzelm [Sat, 04 Apr 1998 11:40:18 +0200] rev 4785
tuned trace msgs;
Fri, 03 Apr 1998 14:38:19 +0200 tuned names;
wenzelm [Fri, 03 Apr 1998 14:38:19 +0200] rev 4784
tuned names;
Fri, 03 Apr 1998 14:37:48 +0200 added get_tthm(s), store_tthms(s);
wenzelm [Fri, 03 Apr 1998 14:37:48 +0200] rev 4783
added get_tthm(s), store_tthms(s); tuned;
Fri, 03 Apr 1998 14:36:20 +0200 tuned comments;
wenzelm [Fri, 03 Apr 1998 14:36:20 +0200] rev 4782
tuned comments;
Fri, 03 Apr 1998 14:36:05 +0200 added attribute.ML;
wenzelm [Fri, 03 Apr 1998 14:36:05 +0200] rev 4781
added attribute.ML;
Fri, 03 Apr 1998 14:35:39 +0200 Theorem tags and attributes.
wenzelm [Fri, 03 Apr 1998 14:35:39 +0200] rev 4780
Theorem tags and attributes.
Fri, 03 Apr 1998 13:32:42 +0200 UNITY
paulson [Fri, 03 Apr 1998 13:32:42 +0200] rev 4779
UNITY
Fri, 03 Apr 1998 13:30:49 +0200 repaired incompatibility with new SML version by eta-expansion
oheimb [Fri, 03 Apr 1998 13:30:49 +0200] rev 4778
repaired incompatibility with new SML version by eta-expansion
Fri, 03 Apr 1998 12:35:27 +0200 New target HOL-UNITY
paulson [Fri, 03 Apr 1998 12:35:27 +0200] rev 4777
New target HOL-UNITY
Fri, 03 Apr 1998 12:34:33 +0200 New UNITY theory
paulson [Fri, 03 Apr 1998 12:34:33 +0200] rev 4776
New UNITY theory
Fri, 03 Apr 1998 11:22:51 +0200 Tidied proofs
paulson [Fri, 03 Apr 1998 11:22:51 +0200] rev 4775
Tidied proofs
Fri, 03 Apr 1998 11:20:41 +0200 Tidied proofs by getting rid of case_tac
paulson [Fri, 03 Apr 1998 11:20:41 +0200] rev 4774
Tidied proofs by getting rid of case_tac
Fri, 03 Apr 1998 09:54:48 +0200 improved \tt appearance of many ASCII special symbols like #
oheimb [Fri, 03 Apr 1998 09:54:48 +0200] rev 4773
improved \tt appearance of many ASCII special symbols like # isabelle theory file keywords now appear bold only when at begin of line
Thu, 02 Apr 1998 17:19:02 +0200 split_all_tac now fails if there is nothing to split
oheimb [Thu, 02 Apr 1998 17:19:02 +0200] rev 4772
split_all_tac now fails if there is nothing to split split_all_tac has moved within claset() from usafe wrappers to safe wrappers
Thu, 02 Apr 1998 13:49:04 +0200 new theorems
paulson [Thu, 02 Apr 1998 13:49:04 +0200] rev 4771
new theorems
Thu, 02 Apr 1998 13:48:48 +0200 changed if_bool_eq to if_bool_eq_conj
paulson [Thu, 02 Apr 1998 13:48:48 +0200] rev 4770
changed if_bool_eq to if_bool_eq_conj
Thu, 02 Apr 1998 13:48:28 +0200 changed if_bool_eq to if_bool_eq_conj and added if_bool_eq_disj
paulson [Thu, 02 Apr 1998 13:48:28 +0200] rev 4769
changed if_bool_eq to if_bool_eq_conj and added if_bool_eq_disj
Thu, 02 Apr 1998 13:47:03 +0200 New theorems card_Diff_le and card_insert_le; tidied
paulson [Thu, 02 Apr 1998 13:47:03 +0200] rev 4768
New theorems card_Diff_le and card_insert_le; tidied
Thu, 02 Apr 1998 12:45:47 +0200 introduced functions for updating the wrapper lists
oheimb [Thu, 02 Apr 1998 12:45:47 +0200] rev 4767
introduced functions for updating the wrapper lists merge_cs now uses merge_alists to merge wrapper lists, left cs has precedence!
Thu, 02 Apr 1998 12:39:32 +0200 *** empty log message ***
oheimb [Thu, 02 Apr 1998 12:39:32 +0200] rev 4766
*** empty log message ***
Mon, 30 Mar 1998 21:15:18 +0200 merge_cs now also merges safe and unsafe wrappers
oheimb [Mon, 30 Mar 1998 21:15:18 +0200] rev 4765
merge_cs now also merges safe and unsafe wrappers
Mon, 30 Mar 1998 21:14:04 +0200 generalized appearance of trancl_into_rtrancl and r_into_trancl
oheimb [Mon, 30 Mar 1998 21:14:04 +0200] rev 4764
generalized appearance of trancl_into_rtrancl and r_into_trancl added irrefl_tranclI, reflcl_trancl, trancl_reflcl, trancl_empty, rtrancl_empty
Mon, 30 Mar 1998 21:09:46 +0200 adapted proof of finite_converse
oheimb [Mon, 30 Mar 1998 21:09:46 +0200] rev 4763
adapted proof of finite_converse
Mon, 30 Mar 1998 21:08:05 +0200 added wf_converse_trancl, adapted proof of wfrec
oheimb [Mon, 30 Mar 1998 21:08:05 +0200] rev 4762
added wf_converse_trancl, adapted proof of wfrec
Mon, 30 Mar 1998 21:06:09 +0200 added caveat
oheimb [Mon, 30 Mar 1998 21:06:09 +0200] rev 4761
added caveat
Mon, 30 Mar 1998 21:05:25 +0200 added introduction and elimination rules for Univalent
oheimb [Mon, 30 Mar 1998 21:05:25 +0200] rev 4760
added introduction and elimination rules for Univalent
Mon, 30 Mar 1998 21:04:41 +0200 added Univalent_rel_pow
oheimb [Mon, 30 Mar 1998 21:04:41 +0200] rev 4759
added Univalent_rel_pow
Mon, 30 Mar 1998 21:04:13 +0200 removed superfluous use_thy
oheimb [Mon, 30 Mar 1998 21:04:13 +0200] rev 4758
removed superfluous use_thy
Mon, 30 Mar 1998 21:03:14 +0200 removed superfluous translations
oheimb [Mon, 30 Mar 1998 21:03:14 +0200] rev 4757
removed superfluous translations
Tue, 24 Mar 1998 16:57:40 +0100 added try, single, many;
wenzelm [Tue, 24 Mar 1998 16:57:40 +0100] rev 4756
added try, single, many; improved source: prompt;
Tue, 24 Mar 1998 15:57:18 +0100 added cproj', and therefore extended prj
oheimb [Tue, 24 Mar 1998 15:57:18 +0100] rev 4755
added cproj', and therefore extended prj tried to fix polymorphism problem for take_defs. A full solution will require significant changes.
Tue, 24 Mar 1998 15:54:42 +0100 added cproj', and therefore extended prj
oheimb [Tue, 24 Mar 1998 15:54:42 +0100] rev 4754
added cproj', and therefore extended prj
Tue, 24 Mar 1998 15:53:47 +0100 improved checks
oheimb [Tue, 24 Mar 1998 15:53:47 +0100] rev 4753
improved checks
Tue, 24 Mar 1998 15:51:37 +0100 added o2s
oheimb [Tue, 24 Mar 1998 15:51:37 +0100] rev 4752
added o2s
Tue, 24 Mar 1998 15:49:32 +0100 added finite_acyclic_wf_converse: corrected 8bit chars
oheimb [Tue, 24 Mar 1998 15:49:32 +0100] rev 4751
added finite_acyclic_wf_converse: corrected 8bit chars
Tue, 24 Mar 1998 15:46:34 +0100 added acyclicI
oheimb [Tue, 24 Mar 1998 15:46:34 +0100] rev 4750
added acyclicI
Tue, 24 Mar 1998 15:46:08 +0100 added finite_acyclic_wf_converse
oheimb [Tue, 24 Mar 1998 15:46:08 +0100] rev 4749
added finite_acyclic_wf_converse
Mon, 23 Mar 1998 13:56:53 +0100 more thms
paulson [Mon, 23 Mar 1998 13:56:53 +0100] rev 4748
more thms
Mon, 16 Mar 1998 16:54:07 +0100 inverse -> converse
paulson [Mon, 16 Mar 1998 16:54:07 +0100] rev 4747
inverse -> converse
(0) -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip