paulson [Thu, 20 Nov 1997 11:53:51 +0100] rev 4244
New, higher-level definition of \\out macro
paulson [Thu, 20 Nov 1997 11:03:53 +0100] rev 4243
Speeded up the proof of succ_lt_induct_lemma
paulson [Thu, 20 Nov 1997 11:03:26 +0100] rev 4242
Two new rewrites
paulson [Thu, 20 Nov 1997 10:55:27 +0100] rev 4241
Got rid of some slow deepen_tac calls
paulson [Thu, 20 Nov 1997 10:54:04 +0100] rev 4240
Renamed "overload" to "overloaded" for sml/nj compatibility
paulson [Thu, 20 Nov 1997 10:50:51 +0100] rev 4239
No more makeatletter/other
paulson [Tue, 18 Nov 1997 16:37:25 +0100] rev 4238
Crypt_imp_keysFor: version of Crypt_imp_invKey_keysFor for shared keys
paulson [Tue, 18 Nov 1997 16:36:33 +0100] rev 4237
The dtac was discarding information, though apparently no proofs were hurt
berghofe [Tue, 18 Nov 1997 15:30:50 +0100] rev 4236
Fixed bug in inst_split.
wenzelm [Mon, 17 Nov 1997 15:40:25 +0100] rev 4235
improved big_rec_name lookup;
paulson [Mon, 17 Nov 1997 10:50:03 +0100] rev 4234
Updated comments. A bug causes MLWorks to use much
more storage than necessary
paulson [Mon, 17 Nov 1997 10:48:07 +0100] rev 4233
Rationalized error handling: if low-level tactic (depth_tac) cannot accept the
goal then it raises exception TRANS. Top-level tactics (blast_tac)
generate warnings and then fail immediately.
berghofe [Mon, 17 Nov 1997 09:52:20 +0100] rev 4232
Tuned function mk_cntxt_splitthm.
Fixed bug which caused split_tac to fail when
(Const ("splitconst", ...) $ ...) was of function type.
nipkow [Sun, 16 Nov 1997 16:18:31 +0100] rev 4231
Removed
"(ALL x:f``A. P x) = (ALL x:A. P(f x))",
"(EX x:f``A. P x) = (EX x:A. P(f x))",
again, because they were already there and added
"(UN x:f``A. B x) = (UN a:A. B(f a))"
"(INT x:f``A. B x) = (INT a:A. B(f a))"
instead.
nipkow [Sat, 15 Nov 1997 18:41:06 +0100] rev 4230
Redesigned the decision procedures for (Abelian) groups and commutative rings.
nipkow [Sat, 15 Nov 1997 13:10:52 +0100] rev 4229
Added
> "(? x : f `` A. P x) = (? a:A. P(f a))"
> "(! x : f `` A. P x) = (! a:A. P(f a))"
wenzelm [Fri, 14 Nov 1997 15:51:09 +0100] rev 4228
merge_refs: check for different versions of theories;
wenzelm [Thu, 13 Nov 1997 17:55:27 +0100] rev 4227
export read_raw_typ;
wenzelm [Thu, 13 Nov 1997 15:14:14 +0100] rev 4226
fixed record parser;
wenzelm [Thu, 13 Nov 1997 12:43:17 +0100] rev 4225
improved record syntax;
wenzelm [Thu, 13 Nov 1997 10:31:42 +0100] rev 4224
made SML/NJ happy;
oheimb [Wed, 12 Nov 1997 18:58:50 +0100] rev 4223
added thin_refl to hyp_subst_tac
wenzelm [Wed, 12 Nov 1997 16:28:53 +0100] rev 4222
refer to $ISABELLE_HOME/src;
wenzelm [Wed, 12 Nov 1997 16:27:13 +0100] rev 4221
structure BasisLibrary;
wenzelm [Wed, 12 Nov 1997 16:26:05 +0100] rev 4220
renamed to use.ML;
wenzelm [Wed, 12 Nov 1997 16:25:45 +0100] rev 4219
Redefine 'use' command in order to support path variable expansion,
automatic suffix generation, and symbolic input filtering (if
required).
wenzelm [Wed, 12 Nov 1997 16:25:35 +0100] rev 4218
adapted to new Use, File structs;
wenzelm [Wed, 12 Nov 1997 16:23:28 +0100] rev 4217
added path variables;
wenzelm [Wed, 12 Nov 1997 16:23:11 +0100] rev 4216
File system operations.
wenzelm [Wed, 12 Nov 1997 16:22:59 +0100] rev 4215
moved old file stuff from library.ML to Thy/browser_info.ML;
subdir_of no longer infix;