Wed, 04 Jun 1997 12:26:42 +0200 eliminated freeze_vars;
wenzelm [Wed, 04 Jun 1997 12:26:42 +0200] rev 3395
eliminated freeze_vars;
Wed, 04 Jun 1997 10:58:56 +0200 changed priority of -> from [6,5]5 to [1,0]0
mueller [Wed, 04 Jun 1997 10:58:56 +0200] rev 3394
changed priority of -> from [6,5]5 to [1,0]0
Tue, 03 Jun 1997 16:38:58 +0200 is_blank: fixed space2;
wenzelm [Tue, 03 Jun 1997 16:38:58 +0200] rev 3393
is_blank: fixed space2;
Tue, 03 Jun 1997 12:03:38 +0200 No longer refers to internal TFL structures
paulson [Tue, 03 Jun 1997 12:03:38 +0200] rev 3392
No longer refers to internal TFL structures
Tue, 03 Jun 1997 11:08:08 +0200 More de-HOLification: using Free, Const, etc. instead of mk_var, mk_const
paulson [Tue, 03 Jun 1997 11:08:08 +0200] rev 3391
More de-HOLification: using Free, Const, etc. instead of mk_var, mk_const Changed the TFL functor to a structure (currently called Prim)
Tue, 03 Jun 1997 10:56:04 +0200 New theory "Power" of exponentiation (and binomial coefficients)
paulson [Tue, 03 Jun 1997 10:56:04 +0200] rev 3390
New theory "Power" of exponentiation (and binomial coefficients)
Tue, 03 Jun 1997 10:53:58 +0200 New theorem about the cardinality of the powerset (uses exponentiation)
paulson [Tue, 03 Jun 1997 10:53:58 +0200] rev 3389
New theorem about the cardinality of the powerset (uses exponentiation)
Mon, 02 Jun 1997 12:19:01 +0200 Type inference makes a Const here, perhaps elsewhere?thry.sml
paulson [Mon, 02 Jun 1997 12:19:01 +0200] rev 3388
Type inference makes a Const here, perhaps elsewhere?thry.sml
Mon, 02 Jun 1997 12:17:19 +0200 poly_tvars allows recdefs to be made without type constraints
paulson [Mon, 02 Jun 1997 12:17:19 +0200] rev 3387
poly_tvars allows recdefs to be made without type constraints
Mon, 02 Jun 1997 12:16:24 +0200 Corrected banner: it is W0, not MiniML
paulson [Mon, 02 Jun 1997 12:16:24 +0200] rev 3386
Corrected banner: it is W0, not MiniML
Mon, 02 Jun 1997 12:15:13 +0200 New statement and proof of free_tv_subst_var in order to cope with new
paulson [Mon, 02 Jun 1997 12:15:13 +0200] rev 3385
New statement and proof of free_tv_subst_var in order to cope with new rewrite rules Un_insert_left, Un_insert_right
Mon, 02 Jun 1997 12:14:15 +0200 Now Un_insert_left, Un_insert_right are default rewrite rules
paulson [Mon, 02 Jun 1997 12:14:15 +0200] rev 3384
Now Un_insert_left, Un_insert_right are default rewrite rules
Mon, 02 Jun 1997 12:13:42 +0200 Corrected statement of filter_append; added filter_size
paulson [Mon, 02 Jun 1997 12:13:42 +0200] rev 3383
Corrected statement of filter_append; added filter_size
Mon, 02 Jun 1997 12:12:57 +0200 Simplified proof
paulson [Mon, 02 Jun 1997 12:12:57 +0200] rev 3382
Simplified proof
Mon, 02 Jun 1997 12:12:27 +0200 New theorems le_add_diff_inverse, le_add_diff_inverse2
paulson [Mon, 02 Jun 1997 12:12:27 +0200] rev 3381
New theorems le_add_diff_inverse, le_add_diff_inverse2
Fri, 30 May 1997 16:37:20 +0200 trivial changes to incorporate CTL.thy and Example.ML in html file;
mueller [Fri, 30 May 1997 16:37:20 +0200] rev 3380
trivial changes to incorporate CTL.thy and Example.ML in html file;
Fri, 30 May 1997 15:55:27 +0200 Simplified the calling sequence of CONTEXT_REWRITE_RULE
paulson [Fri, 30 May 1997 15:55:27 +0200] rev 3379
Simplified the calling sequence of CONTEXT_REWRITE_RULE Eliminated get_rhs, which was calling dest_Trueprop too many times
Fri, 30 May 1997 15:30:52 +0200 Moved "less_eq" to NatDef from Arith
paulson [Fri, 30 May 1997 15:30:52 +0200] rev 3378
Moved "less_eq" to NatDef from Arith
Fri, 30 May 1997 15:24:27 +0200 New results including the basis for unique factorization
paulson [Fri, 30 May 1997 15:24:27 +0200] rev 3377
New results including the basis for unique factorization
Fri, 30 May 1997 15:23:49 +0200 Now "primes" is a set
paulson [Fri, 30 May 1997 15:23:49 +0200] rev 3376
Now "primes" is a set
Fri, 30 May 1997 15:23:25 +0200 Now Divides must be the parent
paulson [Fri, 30 May 1997 15:23:25 +0200] rev 3375
Now Divides must be the parent
Fri, 30 May 1997 15:22:19 +0200 New proofs about cardinality. Suggested by Florian Kammueller
paulson [Fri, 30 May 1997 15:22:19 +0200] rev 3374
New proofs about cardinality. Suggested by Florian Kammueller
Fri, 30 May 1997 15:21:53 +0200 Addition of Finite as parent allows cardinality theorems
paulson [Fri, 30 May 1997 15:21:53 +0200] rev 3373
Addition of Finite as parent allows cardinality theorems
Fri, 30 May 1997 15:21:21 +0200 Replacement of "divides" by "dvd" from Divides.thy, and updating of proofs
paulson [Fri, 30 May 1997 15:21:21 +0200] rev 3372
Replacement of "divides" by "dvd" from Divides.thy, and updating of proofs
Fri, 30 May 1997 15:20:41 +0200 Overloading of "^" requires a type constraint
paulson [Fri, 30 May 1997 15:20:41 +0200] rev 3371
Overloading of "^" requires a type constraint
Fri, 30 May 1997 15:19:58 +0200 Overloading of "^" requires new type class "power", with types "nat" and
paulson [Fri, 30 May 1997 15:19:58 +0200] rev 3370
Overloading of "^" requires new type class "power", with types "nat" and "set" in that class. The operator itself is declared in Nat.thy
Fri, 30 May 1997 15:17:36 +0200 New theory Divides
paulson [Fri, 30 May 1997 15:17:36 +0200] rev 3369
New theory Divides
Fri, 30 May 1997 15:17:14 +0200 Many new theorems about cardinality
paulson [Fri, 30 May 1997 15:17:14 +0200] rev 3368
Many new theorems about cardinality
Fri, 30 May 1997 15:16:44 +0200 Now Divides must be the parent
paulson [Fri, 30 May 1997 15:16:44 +0200] rev 3367
Now Divides must be the parent
Fri, 30 May 1997 15:15:57 +0200 Moving div and mod from Arith to Divides
paulson [Fri, 30 May 1997 15:15:57 +0200] rev 3366
Moving div and mod from Arith to Divides Moving dvd from ex/Primes to Divides
Fri, 30 May 1997 15:14:59 +0200 flushOut ensures that no recent error message are lost (not certain this is
paulson [Fri, 30 May 1997 15:14:59 +0200] rev 3365
flushOut ensures that no recent error message are lost (not certain this is necessary)
Tue, 27 May 1997 17:49:52 +0200 polyml-3.1 default again (for local work);
wenzelm [Tue, 27 May 1997 17:49:52 +0200] rev 3364
polyml-3.1 default again (for local work);
Tue, 27 May 1997 16:31:26 +0200 fixed -P (checkout only);
wenzelm [Tue, 27 May 1997 16:31:26 +0200] rev 3363
fixed -P (checkout only);
Tue, 27 May 1997 15:45:07 +0200 NJ 1.09.2x as factory default! Isabelle94-8
wenzelm [Tue, 27 May 1997 15:45:07 +0200] rev 3362
NJ 1.09.2x as factory default!
Tue, 27 May 1997 15:07:02 +0200 Last changes for new release 94-8
mueller [Tue, 27 May 1997 15:07:02 +0200] rev 3361
Last changes for new release 94-8
Tue, 27 May 1997 14:38:49 +0200 added 1.09.28 note;
wenzelm [Tue, 27 May 1997 14:38:49 +0200] rev 3360
added 1.09.28 note;
Tue, 27 May 1997 13:26:42 +0200 New theorems suggested by Florian Kammueller
paulson [Tue, 27 May 1997 13:26:42 +0200] rev 3359
New theorems suggested by Florian Kammueller
Tue, 27 May 1997 13:26:11 +0200 Restoration of the two "bypassed" theorems Union_quotient and quotient_disj
paulson [Tue, 27 May 1997 13:26:11 +0200] rev 3358
Restoration of the two "bypassed" theorems Union_quotient and quotient_disj
Tue, 27 May 1997 13:25:00 +0200 Removal of card_insert_disjoint, which is now a default rewrite rule
paulson [Tue, 27 May 1997 13:25:00 +0200] rev 3357
Removal of card_insert_disjoint, which is now a default rewrite rule
Tue, 27 May 1997 13:24:15 +0200 New theorem disjoint_eq_subset_Compl
paulson [Tue, 27 May 1997 13:24:15 +0200] rev 3356
New theorem disjoint_eq_subset_Compl
Tue, 27 May 1997 13:23:53 +0200 New theorem le_Suc_eq
paulson [Tue, 27 May 1997 13:23:53 +0200] rev 3355
New theorem le_Suc_eq
Tue, 27 May 1997 13:23:27 +0200 Removal of mask.sig and mask.sml
paulson [Tue, 27 May 1997 13:23:27 +0200] rev 3354
Removal of mask.sig and mask.sml
Tue, 27 May 1997 13:22:30 +0200 Removal of module Mask and datatype binding with its constructor |->
paulson [Tue, 27 May 1997 13:22:30 +0200] rev 3353
Removal of module Mask and datatype binding with its constructor |->
Tue, 27 May 1997 13:03:41 +0200 New theorems suggested by Florian Kammueller
paulson [Tue, 27 May 1997 13:03:41 +0200] rev 3352
New theorems suggested by Florian Kammueller
Mon, 26 May 1997 14:54:24 +0200 remoded ccc1
slotosch [Mon, 26 May 1997 14:54:24 +0200] rev 3351
remoded ccc1
Mon, 26 May 1997 13:51:03 +0200 removed ccc1
slotosch [Mon, 26 May 1997 13:51:03 +0200] rev 3350
removed ccc1
Mon, 26 May 1997 13:45:39 +0200 tuned comment;
wenzelm [Mon, 26 May 1997 13:45:39 +0200] rev 3349
tuned comment;
Mon, 26 May 1997 12:54:40 +0200 Two useful facts about Powersets suggested by Florian Kammueller
paulson [Mon, 26 May 1997 12:54:40 +0200] rev 3348
Two useful facts about Powersets suggested by Florian Kammueller
Mon, 26 May 1997 12:53:45 +0200 Added a missing "result();" after problem 43.
paulson [Mon, 26 May 1997 12:53:45 +0200] rev 3347
Added a missing "result();" after problem 43.
Mon, 26 May 1997 12:44:04 +0200 Tidying using the new exhaust_tac
paulson [Mon, 26 May 1997 12:44:04 +0200] rev 3346
Tidying using the new exhaust_tac
Mon, 26 May 1997 12:42:38 +0200 Now recdef checks the name of the function being defined.
paulson [Mon, 26 May 1997 12:42:38 +0200] rev 3345
Now recdef checks the name of the function being defined. Slight tidying
Mon, 26 May 1997 12:40:51 +0200 Deleted option_case_tac because exhaust_tac performs a similar function.
paulson [Mon, 26 May 1997 12:40:51 +0200] rev 3344
Deleted option_case_tac because exhaust_tac performs a similar function. Deleted the duplicate proof of expand_option_case...
Mon, 26 May 1997 12:39:57 +0200 Renamed lessD to Suc_leI
paulson [Mon, 26 May 1997 12:39:57 +0200] rev 3343
Renamed lessD to Suc_leI
Mon, 26 May 1997 12:38:29 +0200 New operator "lists" for formalizing sets of lists
paulson [Mon, 26 May 1997 12:38:29 +0200] rev 3342
New operator "lists" for formalizing sets of lists
Mon, 26 May 1997 12:37:24 +0200 New theorem subset_inj_onto
paulson [Mon, 26 May 1997 12:37:24 +0200] rev 3341
New theorem subset_inj_onto
Mon, 26 May 1997 12:36:56 +0200 Two results suggested by Florian Kammueller
paulson [Mon, 26 May 1997 12:36:56 +0200] rev 3340
Two results suggested by Florian Kammueller
Mon, 26 May 1997 12:36:16 +0200 Tidying and a couple of useful lemmas
paulson [Mon, 26 May 1997 12:36:16 +0200] rev 3339
Tidying and a couple of useful lemmas
Mon, 26 May 1997 12:34:54 +0200 Added recdef
paulson [Mon, 26 May 1997 12:34:54 +0200] rev 3338
Added recdef
Mon, 26 May 1997 12:34:05 +0200 Primrec: New example ported from ZF
paulson [Mon, 26 May 1997 12:34:05 +0200] rev 3337
Primrec: New example ported from ZF
Mon, 26 May 1997 12:33:38 +0200 Renamed lessD to Suc_leI
paulson [Mon, 26 May 1997 12:33:38 +0200] rev 3336
Renamed lessD to Suc_leI
Mon, 26 May 1997 12:33:03 +0200 New example ported from ZF
paulson [Mon, 26 May 1997 12:33:03 +0200] rev 3335
New example ported from ZF
Mon, 26 May 1997 12:32:35 +0200 Simplified proofs using expand_option_case
paulson [Mon, 26 May 1997 12:32:35 +0200] rev 3334
Simplified proofs using expand_option_case
Mon, 26 May 1997 12:29:55 +0200 Now checks the name of the function being defined;
paulson [Mon, 26 May 1997 12:29:55 +0200] rev 3333
Now checks the name of the function being defined; More de-HOL-ification
Mon, 26 May 1997 12:29:10 +0200 More de-HOL-ification
paulson [Mon, 26 May 1997 12:29:10 +0200] rev 3332
More de-HOL-ification
Mon, 26 May 1997 12:28:30 +0200 Now checks the name of the function being defined
paulson [Mon, 26 May 1997 12:28:30 +0200] rev 3331
Now checks the name of the function being defined
Mon, 26 May 1997 12:27:58 +0200 Deleted unused functions
paulson [Mon, 26 May 1997 12:27:58 +0200] rev 3330
Deleted unused functions
Mon, 26 May 1997 12:26:35 +0200 Now a Perl script. No longer requires commands to be at the beginnings of
paulson [Mon, 26 May 1997 12:26:35 +0200] rev 3329
Now a Perl script. No longer requires commands to be at the beginnings of lines. RESTRICTION: no longer expands tabs to spaces. No longer lists the files it is altering.
Mon, 26 May 1997 12:25:15 +0200 Slight simplifications
paulson [Mon, 26 May 1997 12:25:15 +0200] rev 3328
Slight simplifications
Sun, 25 May 1997 18:45:25 +0200 Eliminated ccc1. Moved ID,oo into Cfun.
slotosch [Sun, 25 May 1997 18:45:25 +0200] rev 3327
Eliminated ccc1. Moved ID,oo into Cfun.
Sun, 25 May 1997 16:59:40 +0200 Moved the classes flat chfin from Fix to Pcpo.
slotosch [Sun, 25 May 1997 16:59:40 +0200] rev 3326
Moved the classes flat chfin from Fix to Pcpo. Corresponding theorems from Fix into Pcpo,Cont,Cfun3
Sun, 25 May 1997 16:57:19 +0200 *** empty log message ***
slotosch [Sun, 25 May 1997 16:57:19 +0200] rev 3325
*** empty log message ***
Sun, 25 May 1997 16:17:09 +0200 Eliminated the prediates flat,chfin
slotosch [Sun, 25 May 1997 16:17:09 +0200] rev 3324
Eliminated the prediates flat,chfin Changed theorems with flat(x::'a) to (x::'a::flat) Since flat<chfin theorems adm_flat,adm_flatdom are eliminated. Use adm_chain_finite and adm_chfindom instead! Examples do not use flat_flat any more
Sun, 25 May 1997 11:07:52 +0200 eliminated the constant less by the introduction of the axclass sq_ord
slotosch [Sun, 25 May 1997 11:07:52 +0200] rev 3323
eliminated the constant less by the introduction of the axclass sq_ord added explicit type ::'a::po in the following theorems: minimal2UU,antisym_less_inverse,box_less,not_less2not_eq,monofun_pair and dist_eqI (in domain-package) added instances instance fun :: (term,sq_ord)sq_ord instance "->" :: (term,sq_ord)sq_ord instance "**" :: (sq_ord,sq_ord)sq_ord instance "*" :: (sq_ord,sq_ord)sq_ord instance "++" :: (pcpo,pcpo)sq_ord instance u :: (sq_ord)sq_ord instance lift :: (term)sq_ord instance discr :: (term)sq_ord
Fri, 23 May 1997 18:55:28 +0200 tuned;
wenzelm [Fri, 23 May 1997 18:55:28 +0200] rev 3322
tuned;
Fri, 23 May 1997 18:20:20 +0200 arbitrary
nipkow [Fri, 23 May 1997 18:20:20 +0200] rev 3321
arbitrary
Fri, 23 May 1997 18:17:53 +0200 Added `arbitrary'
nipkow [Fri, 23 May 1997 18:17:53 +0200] rev 3320
Added `arbitrary'
Fri, 23 May 1997 14:52:45 +0200 fixed;
wenzelm [Fri, 23 May 1997 14:52:45 +0200] rev 3319
fixed;
Fri, 23 May 1997 14:49:39 +0200 new syntactic priority of lambda abstraction
oheimb [Fri, 23 May 1997 14:49:39 +0200] rev 3318
new syntactic priority of lambda abstraction
Fri, 23 May 1997 14:48:10 +0200 adapted entry for addss, addSss
oheimb [Fri, 23 May 1997 14:48:10 +0200] rev 3317
adapted entry for addss, addSss
Fri, 23 May 1997 14:17:40 +0200 news.
nipkow [Fri, 23 May 1997 14:17:40 +0200] rev 3316
news.
Fri, 23 May 1997 14:13:51 +0200 Documented `size' function for datatypes.
nipkow [Fri, 23 May 1997 14:13:51 +0200] rev 3315
Documented `size' function for datatypes.
Fri, 23 May 1997 13:39:22 +0200 fixed a bug
mueller [Fri, 23 May 1997 13:39:22 +0200] rev 3314
fixed a bug
Fri, 23 May 1997 13:31:59 +0200 removed TFL from test;
wenzelm [Fri, 23 May 1997 13:31:59 +0200] rev 3313
removed TFL from test;
Fri, 23 May 1997 11:28:22 +0200 remove cl.cam font server;
wenzelm [Fri, 23 May 1997 11:28:22 +0200] rev 3312
remove cl.cam font server;
Fri, 23 May 1997 10:14:16 +0200 exec the emacs;
wenzelm [Fri, 23 May 1997 10:14:16 +0200] rev 3311
exec the emacs;
Fri, 23 May 1997 09:20:35 +0200 Base theory is now Arith, not Nat. (because all datatypes now require Arith).
nipkow [Fri, 23 May 1997 09:20:35 +0200] rev 3310
Base theory is now Arith, not Nat. (because all datatypes now require Arith).
Fri, 23 May 1997 09:18:06 +0200 All datatypes now require Arith.
nipkow [Fri, 23 May 1997 09:18:06 +0200] rev 3309
All datatypes now require Arith.
Fri, 23 May 1997 09:17:26 +0200 Added overloaded function `size' for all datatypes.
nipkow [Fri, 23 May 1997 09:17:26 +0200] rev 3308
Added overloaded function `size' for all datatypes.
Thu, 22 May 1997 18:29:17 +0200 exhaust_tac can now deal with whole terms rather than just variables.
nipkow [Thu, 22 May 1997 18:29:17 +0200] rev 3307
exhaust_tac can now deal with whole terms rather than just variables.
Thu, 22 May 1997 17:20:55 +0200 added href to Isamode;
wenzelm [Thu, 22 May 1997 17:20:55 +0200] rev 3306
added href to Isamode;
Thu, 22 May 1997 16:44:47 +0200 fixed doc;
wenzelm [Thu, 22 May 1997 16:44:47 +0200] rev 3305
fixed doc;
Thu, 22 May 1997 16:37:00 +0200 adapted to Isamode 2.6;
wenzelm [Thu, 22 May 1997 16:37:00 +0200] rev 3304
adapted to Isamode 2.6;
Thu, 22 May 1997 16:04:48 +0200 tuned Isamode stuff;
wenzelm [Thu, 22 May 1997 16:04:48 +0200] rev 3303
tuned Isamode stuff;
Thu, 22 May 1997 15:13:16 +0200 New headers and other minor changes
paulson [Thu, 22 May 1997 15:13:16 +0200] rev 3302
New headers and other minor changes
Thu, 22 May 1997 15:11:56 +0200 Now the recdef induction rule variables are named u, v, ...
paulson [Thu, 22 May 1997 15:11:56 +0200] rev 3301
Now the recdef induction rule variables are named u, v, ...
Thu, 22 May 1997 15:11:23 +0200 New example of recdef and permutative rewriting
paulson [Thu, 22 May 1997 15:11:23 +0200] rev 3300
New example of recdef and permutative rewriting
(0) -3000 -1000 -300 -100 -96 +96 +100 +300 +1000 +3000 +10000 +30000 tip