wenzelm [Wed, 13 May 1998 10:21:28 +0200] rev 4915
HOL/record: now includes concrete syntax for record terms;
wenzelm [Tue, 12 May 1998 18:07:03 +0200] rev 4914
added Goal, Goalw;
wenzelm [Tue, 12 May 1998 18:06:27 +0200] rev 4913
branching_level = 250;
wenzelm [Tue, 12 May 1998 18:06:01 +0200] rev 4912
fixed comment;
nipkow [Tue, 12 May 1998 08:36:07 +0200] rev 4911
Removed duplicate list_length_induct
nipkow [Mon, 11 May 1998 14:40:40 +0200] rev 4910
Reordered a few parameters.
nipkow [Mon, 11 May 1998 13:18:25 +0200] rev 4909
Lex
wenzelm [Sun, 10 May 1998 11:59:31 +0200] rev 4908
tuned comment;
nipkow [Fri, 08 May 1998 18:33:29 +0200] rev 4907
Reshuffeling, renaming and a few simple corollaries.
wenzelm [Fri, 08 May 1998 15:45:01 +0200] rev 4906
fixed translations;
wenzelm [Fri, 08 May 1998 13:54:45 +0200] rev 4905
proper thy files;
wenzelm [Fri, 08 May 1998 10:15:39 +0200] rev 4904
fixed update syntax;
wenzelm [Thu, 07 May 1998 18:34:48 +0200] rev 4903
improved source: state-based;
tuned bulk;
wenzelm [Thu, 07 May 1998 18:05:46 +0200] rev 4902
added scan_tvar;
wenzelm [Thu, 07 May 1998 18:05:08 +0200] rev 4901
added 'space';
nipkow [Thu, 07 May 1998 13:02:23 +0200] rev 4900
Got rid of NAe.delta
paulson [Wed, 06 May 1998 13:01:45 +0200] rev 4899
HOL/Update
paulson [Wed, 06 May 1998 13:01:30 +0200] rev 4898
Removed some traces of UNITY
nipkow [Wed, 06 May 1998 11:46:00 +0200] rev 4897
Changed [/] to [:=] and removed actual definition.
paulson [Tue, 05 May 1998 17:28:22 +0200] rev 4896
New syntax for function update; moved to main HOL directory
wenzelm [Tue, 05 May 1998 13:27:18 +0200] rev 4895
misc tuning;
wenzelm [Mon, 04 May 1998 21:07:57 +0200] rev 4894
'more' selector;
thms: selector_convs, update_convs;
tuned;
wenzelm [Mon, 04 May 1998 21:05:38 +0200] rev 4893
added nth_update: 'a -> int * 'a list -> 'a list;
wenzelm [Mon, 04 May 1998 21:05:14 +0200] rev 4892
tuned msg;
wenzelm [Mon, 04 May 1998 13:48:47 +0200] rev 4891
fixed constdefs syntax;
wenzelm [Mon, 04 May 1998 09:54:29 +0200] rev 4890
concrete syntax for record terms;
defs for update;
field types (just abbreviations at the moment);
some thms;
various of minor improvements;
nipkow [Mon, 04 May 1998 09:17:18 +0200] rev 4889
New behaviour of asm_full_simp_tac.
wenzelm [Sat, 02 May 1998 16:46:17 +0200] rev 4888
added CLASIMPSET(') tacticals;
wenzelm [Sat, 02 May 1998 13:27:42 +0200] rev 4887
added trfun_names;
wenzelm [Sat, 02 May 1998 13:27:06 +0200] rev 4886
added accesses: string -> string list;
oheimb [Fri, 01 May 1998 22:40:20 +0200] rev 4885
minor corrections
oheimb [Fri, 01 May 1998 22:30:42 +0200] rev 4884
Auto_tac: now uses enhanced version of asm_full_simp_tac,
Force_tac: replaced fast_tac by best_tac
oheimb [Fri, 01 May 1998 22:28:25 +0200] rev 4883
added finite_dom_map_of and ran_update
oheimb [Fri, 01 May 1998 22:27:43 +0200] rev 4882
added insert_Collect
oheimb [Fri, 01 May 1998 19:51:03 +0200] rev 4881
corrected and updated description of wrapper mechanism (including addss)
added documentation of force_tac
nipkow [Fri, 01 May 1998 11:43:38 +0200] rev 4880
*** empty log message ***
paulson [Fri, 01 May 1998 11:23:04 +0200] rev 4879
"let" is no longer restricted to FOL terms and allows any logical terms
paulson [Fri, 01 May 1998 11:22:09 +0200] rev 4878
Let.ML and Let.thy had been omitted
wenzelm [Thu, 30 Apr 1998 17:16:25 +0200] rev 4877
fixed simpset(), claset();
wenzelm [Wed, 29 Apr 1998 11:46:42 +0200] rev 4876
moved records data to Tools/record_package.ML;
tuned setup;
wenzelm [Wed, 29 Apr 1998 11:45:41 +0200] rev 4875
nontermials;
wenzelm [Wed, 29 Apr 1998 11:45:16 +0200] rev 4874
Theory.require;
adapted to new PureThy.add_defs_i, PureThy.add_axioms;
wenzelm [Wed, 29 Apr 1998 11:44:30 +0200] rev 4873
TypedefPackage.add_typedef;
RecordPackage.add_record;
wenzelm [Wed, 29 Apr 1998 11:43:53 +0200] rev 4872
Theory.require;
wenzelm [Wed, 29 Apr 1998 11:43:34 +0200] rev 4871
Logic.mk_defpair;
adapted to new PureThy.add_defs_i;
wenzelm [Wed, 29 Apr 1998 11:42:04 +0200] rev 4870
Extensible records with structural subtyping in HOL. See
Tools/record_package.ML for the actual implementation.
wenzelm [Wed, 29 Apr 1998 11:41:36 +0200] rev 4869
new theory section 'setup';
wenzelm [Wed, 29 Apr 1998 11:41:08 +0200] rev 4868
nonterminals;
tuned setup;
wenzelm [Wed, 29 Apr 1998 11:40:37 +0200] rev 4867
package extensible records with structural subtyping in HOL -- still
experimental version;
wenzelm [Wed, 29 Apr 1998 11:39:52 +0200] rev 4866
renamed from typedef.ML;
wenzelm [Wed, 29 Apr 1998 11:39:28 +0200] rev 4865
reworked and moved to Tools/record_package.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;
wenzelm [Wed, 29 Apr 1998 11:37:58 +0200] rev 4863
renamed to Tools/typedef_package.ML;
wenzelm [Wed, 29 Apr 1998 11:36:53 +0200] rev 4862
adapted to new PureThy.add_axioms_i;
Theory.parent_path;
wenzelm [Wed, 29 Apr 1998 11:36:08 +0200] rev 4861
adapted to new PureThy.add_tthmss;
Theory.parent_path;
wenzelm [Wed, 29 Apr 1998 11:35:24 +0200] rev 4860
Theory.require;
Logic.mk_defpair;
adapted to new PureThy.add_defs_i;
wenzelm [Wed, 29 Apr 1998 11:34:11 +0200] rev 4859
adapted to new PureThy.add_axioms;
wenzelm [Wed, 29 Apr 1998 11:33:44 +0200] rev 4858
new theory section 'nonterminals';
wenzelm [Wed, 29 Apr 1998 11:33:27 +0200] rev 4857
adapted to new PureThy.add_defs;
wenzelm [Wed, 29 Apr 1998 11:33:06 +0200] rev 4856
Theory.require;
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;
wenzelm [Wed, 29 Apr 1998 11:29:39 +0200] rev 4854
tuned setup;
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;
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;
wenzelm [Wed, 29 Apr 1998 11:25:26 +0200] rev 4851
added append;
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);
wenzelm [Wed, 29 Apr 1998 11:22:52 +0200] rev 4849
tuned error msgs;
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;
wenzelm [Wed, 29 Apr 1998 11:20:53 +0200] rev 4847
tuned get_ax (uses ancestry);
added get_def: theory -> xstring -> thm;
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);
wenzelm [Wed, 29 Apr 1998 11:14:34 +0200] rev 4845
adapted to new PureThy.add_axioms_i;
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;
wenzelm [Wed, 29 Apr 1998 11:11:36 +0200] rev 4843
added thm, thms;
wenzelm [Wed, 29 Apr 1998 11:10:40 +0200] rev 4842
*** empty log message ***
paulson [Tue, 28 Apr 1998 13:52:18 +0200] rev 4841
new thms, really demos of the final coalgebra theorem
paulson [Tue, 28 Apr 1998 13:51:39 +0200] rev 4840
new thms image_0_left, image_Un_left, etc.
paulson [Tue, 28 Apr 1998 13:50:41 +0200] rev 4839
new thm mult_lt_mono1
oheimb [Mon, 27 Apr 1998 19:32:19 +0200] rev 4838
cleanup for split_all_tac as wrapper in claset()
oheimb [Mon, 27 Apr 1998 19:30:40 +0200] rev 4837
removed wrong comment
oheimb [Mon, 27 Apr 1998 19:29:19 +0200] rev 4836
added option_map_eq_Some via AddIffs
nipkow [Mon, 27 Apr 1998 18:06:22 +0200] rev 4835
*** empty log message ***
nipkow [Mon, 27 Apr 1998 17:52:03 +0200] rev 4834
delsplits, Addsplits, Delsplits.
nipkow [Mon, 27 Apr 1998 16:47:50 +0200] rev 4833
Renamed expand_const -> split_const
nipkow [Mon, 27 Apr 1998 16:46:56 +0200] rev 4832
Added conversion of reg.expr. to automata.
Renamed expand_const -> split_const.
nipkow [Mon, 27 Apr 1998 16:45:27 +0200] rev 4831
Renamed expand_const -> split_const.
nipkow [Mon, 27 Apr 1998 16:45:11 +0200] rev 4830
Added a few lemmas.
Renamed expand_const -> split_const.
paulson [Mon, 27 Apr 1998 13:47:46 +0200] rev 4829
New proof of apply_equality and new thm Pi_image_cons
oheimb [Fri, 24 Apr 1998 16:18:39 +0200] rev 4828
improved split_all_tac significantly
oheimb [Fri, 24 Apr 1998 16:16:29 +0200] rev 4827
improved keyboard modifiers
oheimb [Fri, 24 Apr 1998 16:15:34 +0200] rev 4826
added ASCII translation of subseteq
paulson [Fri, 24 Apr 1998 13:06:17 +0200] rev 4825
tidied; div & mod
oheimb [Fri, 24 Apr 1998 11:22:39 +0200] rev 4824
*** empty log message ***
wenzelm [Wed, 22 Apr 1998 19:09:44 +0200] rev 4823
added no_syn;
wenzelm [Wed, 22 Apr 1998 19:08:49 +0200] rev 4822
added mk_cond_defpair, mk_defpair;
nipkow [Wed, 22 Apr 1998 14:06:05 +0200] rev 4821
Modifications due to improved simplifier.
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.
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
oheimb [Tue, 21 Apr 1998 17:23:24 +0200] rev 4818
split_all_tac is now added to claset() _before_ other safe tactics
oheimb [Tue, 21 Apr 1998 17:22:47 +0200] rev 4817
made proof of zmult_congruent2 more stable
oheimb [Tue, 21 Apr 1998 17:22:03 +0200] rev 4816
simplification of explicit theory usage and merges
oheimb [Tue, 21 Apr 1998 17:21:42 +0200] rev 4815
removed split_all_tac from claset() globally within IOA
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
oheimb [Tue, 21 Apr 1998 17:20:28 +0200] rev 4813
layout improvement
paulson [Tue, 21 Apr 1998 10:49:15 +0200] rev 4812
expandshort; new gcd_induct with inbuilt case analysis
paulson [Tue, 21 Apr 1998 10:47:58 +0200] rev 4811
Renamed mod_XXX_cancel to mod_XXX_self
Included their div_ equivalents
paulson [Mon, 20 Apr 1998 10:38:30 +0200] rev 4810
New laws for mod
paulson [Mon, 20 Apr 1998 10:37:00 +0200] rev 4809
proving fib(gcd(m,n)) = gcd(fib m, fib n)
wenzelm [Sun, 19 Apr 1998 17:01:04 +0200] rev 4808
fixed comment;
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
paulson [Fri, 10 Apr 1998 13:41:04 +0200] rev 4806
bug fixes
paulson [Fri, 10 Apr 1998 13:40:29 +0200] rev 4805
can prove the empty relation to be WF
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