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
paulson [Thu, 09 Apr 1998 12:31:35 +0200] rev 4803
Clearer description of recdef, including use of {}
paulson [Thu, 09 Apr 1998 12:29:39 +0200] rev 4802
Simplified the syntax description; mentioned FOL vs HOL
oheimb [Tue, 07 Apr 1998 13:46:34 +0200] rev 4801
*** empty log message ***
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()
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.
wenzelm [Sat, 04 Apr 1998 14:30:19 +0200] rev 4798
no open Simplifier;
wenzelm [Sat, 04 Apr 1998 14:27:11 +0200] rev 4797
tuned fail;
wenzelm [Sat, 04 Apr 1998 12:31:35 +0200] rev 4796
type_error;
replaced thy_data by setup;
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;
wenzelm [Sat, 04 Apr 1998 12:29:07 +0200] rev 4794
no open Simplifier;
wenzelm [Sat, 04 Apr 1998 12:28:39 +0200] rev 4793
replaced thy_data by thy_setup;
wenzelm [Sat, 04 Apr 1998 12:26:47 +0200] rev 4792
type_error;
wenzelm [Sat, 04 Apr 1998 11:44:16 +0200] rev 4791
replaced thy_data by setup;
wenzelm [Sat, 04 Apr 1998 11:43:39 +0200] rev 4790
removed simple;
added fail, untag;