nipkow [Tue, 05 Aug 1997 16:21:45 +0200] rev 3589
Added function `replicate' and lemmas map_cong and set_replicate.
wenzelm [Tue, 05 Aug 1997 16:14:23 +0200] rev 3588
cleaned up;
added getenv;
paulson [Tue, 05 Aug 1997 10:50:24 +0200] rev 3587
Corrected a comment
nipkow [Mon, 04 Aug 1997 11:50:35 +0200] rev 3586
Added a take/dropWhile lemma.
nipkow [Fri, 01 Aug 1997 10:59:19 +0200] rev 3585
Generalized nth_drop (Conny).
nipkow [Fri, 01 Aug 1997 09:42:19 +0200] rev 3584
Corected bug in def of dropWhile (also present in Haskell lib!)
nipkow [Fri, 01 Aug 1997 09:41:38 +0200] rev 3583
Had to remove {x.x=a} = a from !simpset in one proof.
nipkow [Fri, 01 Aug 1997 09:39:28 +0200] rev 3582
Added {x.x=a} = a to !simpset.
wenzelm [Fri, 25 Jul 1997 14:31:48 +0200] rev 3581
removed split_paired_Ex;
fixed proc args;
nipkow [Fri, 25 Jul 1997 13:59:15 +0200] rev 3580
new simproc
wenzelm [Fri, 25 Jul 1997 13:20:12 +0200] rev 3579
*** empty log message ***
wenzelm [Fri, 25 Jul 1997 13:18:45 +0200] rev 3578
load simplifier.ML (again);
wenzelm [Fri, 25 Jul 1997 13:18:09 +0200] rev 3577
added prems argument to simplification procedures;
wenzelm [Fri, 25 Jul 1997 13:17:14 +0200] rev 3576
remove references to simplifier.ML;
wenzelm [Fri, 25 Jul 1997 11:47:09 +0200] rev 3575
improved rewrite_thm / rewrite_goals to handle conditional eqns;
nipkow [Thu, 24 Jul 1997 15:25:29 +0200] rev 3574
Added a few lemmas.
nipkow [Thu, 24 Jul 1997 11:20:12 +0200] rev 3573
Deleted comment.
nipkow [Thu, 24 Jul 1997 11:13:12 +0200] rev 3572
Replaced clumsy rewriting by the new function simplify on thms.
nipkow [Thu, 24 Jul 1997 11:12:18 +0200] rev 3571
List.ML: added lemmas by Stefan Merz.
simpodata.ML: removed rules about ? now subsumed by simplification proc.
paulson [Thu, 24 Jul 1997 10:46:32 +0200] rev 3570
set_of_list -> set
nipkow [Wed, 23 Jul 1997 17:44:15 +0200] rev 3569
Simplified a few proofs because of improved simplification.
nipkow [Wed, 23 Jul 1997 17:43:42 +0200] rev 3568
Prod.ML: Added split_paired_EX and lots of comments about failed attempts to
automate reasoning about products.
simpdata.ML: added simplification procedure for simplifying existential
statements of the form ? x. ... & x = t & ...
wenzelm [Wed, 23 Jul 1997 16:03:19 +0200] rev 3567
added simplification meta rules;
wenzelm [Wed, 23 Jul 1997 12:54:49 +0200] rev 3566
standard congs;
paulson [Wed, 23 Jul 1997 11:54:32 +0200] rev 3565
Now rename_params_rule merely issues warnings--and does nothing--if the
renaming cannot be performed. Previously it raised a fatal error.
paulson [Wed, 23 Jul 1997 11:52:22 +0200] rev 3564
Now Datatype.occs_in_prems prints the necessary warning ITSELF.
It is also easier to invoke and even works if the induction variable
is a parameter (rather than a free variable).
paulson [Wed, 23 Jul 1997 11:50:26 +0200] rev 3563
Uses new version of Datatype.occs_in_prems
paulson [Wed, 23 Jul 1997 11:49:20 +0200] rev 3562
auto update
paulson [Wed, 23 Jul 1997 11:48:59 +0200] rev 3561
Removal of tactical STATE
wenzelm [Wed, 23 Jul 1997 11:11:14 +0200] rev 3560
fixed polymorphic val;
wenzelm [Wed, 23 Jul 1997 11:07:36 +0200] rev 3559
tuned congs: standard;
wenzelm [Wed, 23 Jul 1997 11:04:19 +0200] rev 3558
improved simp tracing;
wenzelm [Wed, 23 Jul 1997 11:03:54 +0200] rev 3557
added simplification meta rules;
wenzelm [Wed, 23 Jul 1997 10:34:18 +0200] rev 3556
tmp fix to accomodate rep_ss changes;
wenzelm [Wed, 23 Jul 1997 10:22:48 +0200] rev 3555
added rewrite_thm;
wenzelm [Wed, 23 Jul 1997 10:22:30 +0200] rev 3554
tuned apsome;
wenzelm [Tue, 22 Jul 1997 19:33:52 +0200] rev 3553
added error_msg;
wenzelm [Tue, 22 Jul 1997 19:33:30 +0200] rev 3552
tuned error / warning;
wenzelm [Tue, 22 Jul 1997 18:46:44 +0200] rev 3551
added print_ss;
improved merge;
wenzelm [Tue, 22 Jul 1997 18:45:43 +0200] rev 3550
added dest_mss, merge_mss;
fixed matching of simproc lhss;
wenzelm [Tue, 22 Jul 1997 17:52:47 +0200] rev 3549
tuned title;
wenzelm [Tue, 22 Jul 1997 17:47:20 +0200] rev 3548
added dest and merge operations;
wenzelm [Tue, 22 Jul 1997 17:46:35 +0200] rev 3547
added pretty_cterm;
wenzelm [Tue, 22 Jul 1997 17:45:42 +0200] rev 3546
improved print_cs;
paulson [Tue, 22 Jul 1997 11:49:59 +0200] rev 3545
Cosmetic changes: margins, indentation, ...
paulson [Tue, 22 Jul 1997 11:49:44 +0200] rev 3544
Now possibility_tac is an explicit function, in order to delay
the evaluation of \!simpset
paulson [Tue, 22 Jul 1997 11:26:02 +0200] rev 3543
Cosmetic changes: margins, indentation, ...
paulson [Tue, 22 Jul 1997 11:23:03 +0200] rev 3542
Now possibility_tac and basic_possibility_tac are explicit functions, in order
to delay the evaluation of \!simpset
paulson [Tue, 22 Jul 1997 11:21:17 +0200] rev 3541
Deleted the superfluous assumption A ~= B, which must hold anyway by induction
paulson [Tue, 22 Jul 1997 11:16:57 +0200] rev 3540
Fixed the spelling of AUTH_NAMES--it could not have worked before\!
paulson [Tue, 22 Jul 1997 11:15:14 +0200] rev 3539
Option is a synonym for General because MLWorks does not yet provide
Option as a separate structure
paulson [Tue, 22 Jul 1997 11:14:18 +0200] rev 3538
Removal of the tactical STATE
paulson [Tue, 22 Jul 1997 11:12:55 +0200] rev 3537
Removal of the tactical STATE
wenzelm [Fri, 18 Jul 1997 14:06:54 +0200] rev 3536
tuned error propagation msg;
wenzelm [Fri, 18 Jul 1997 13:57:19 +0200] rev 3535
defs may now be conditional;
improved output of warnings / errors;
wenzelm [Fri, 18 Jul 1997 13:55:09 +0200] rev 3534
renamed |-> <-| <-> to Parse/PrintRule;
wenzelm [Fri, 18 Jul 1997 13:54:41 +0200] rev 3533
tuned warning;
wenzelm [Fri, 18 Jul 1997 13:52:35 +0200] rev 3532
tuned warnings;
print_current_goals_fn, result_error_fn hooks replace print_goals_ref;
wenzelm [Fri, 18 Jul 1997 13:51:28 +0200] rev 3531
considered removal of print_goals_ref;
wenzelm [Fri, 18 Jul 1997 13:37:16 +0200] rev 3530
defs: allow conditions;
wenzelm [Fri, 18 Jul 1997 13:36:43 +0200] rev 3529
tuned warning;
improved comments;
wenzelm [Fri, 18 Jul 1997 13:36:03 +0200] rev 3528
renamed |-> <-| <-> to Parse/PrintRule;
wenzelm [Fri, 18 Jul 1997 13:35:36 +0200] rev 3527
tuned warning;
wenzelm [Fri, 18 Jul 1997 13:35:15 +0200] rev 3526
tuned warning;
renamed |-> <-| <-> to Parse/PrintRule;
wenzelm [Fri, 18 Jul 1997 13:33:20 +0200] rev 3525
improved output channels: normal, warning, error;
wenzelm [Thu, 17 Jul 1997 15:03:38 +0200] rev 3524
fixed EqI meta rule;
mueller [Thu, 17 Jul 1997 12:44:58 +0200] rev 3523
changes needed for introducing fairness
mueller [Thu, 17 Jul 1997 12:44:16 +0200] rev 3522
changes neede for introducing fairness
mueller [Thu, 17 Jul 1997 12:43:32 +0200] rev 3521
changes needed for adding fairness
wenzelm [Wed, 16 Jul 1997 11:34:42 +0200] rev 3520
fixed merge of internal simprocs;
paulson [Mon, 14 Jul 1997 12:47:21 +0200] rev 3519
Changing "lost" from a parameter of protocol definitions to a constant.
Advantages: no "lost" argument everywhere; fewer Vars in subgoals;
less need for specially instantiated rules
Disadvantage: can no longer prove "Agent_not_see_encrypted_key", but this
theorem was never used, and its original proof was also broken
the introduction of the "Notes" constructor.
paulson [Mon, 14 Jul 1997 12:44:09 +0200] rev 3518
Fixed delIffs to deal correctly with the D-rule
paulson [Mon, 14 Jul 1997 12:42:28 +0200] rev 3517
Removed redundant addsimps of Un_insert_left, which is now a default simprule
paulson [Fri, 11 Jul 1997 13:32:39 +0200] rev 3516
Removal of monotonicity reasoning involving "lost" and the theorem
Agent_not_see_encrypted_key, which (a) is never used and (b) becomes harder
to prove when Notes is available.
paulson [Fri, 11 Jul 1997 13:30:01 +0200] rev 3515
Now uses the Notes constructor to distinguish the Client (who has chosen M)
from the Spy (who may have replayed her messages)
paulson [Fri, 11 Jul 1997 13:28:53 +0200] rev 3514
Moved some declarations to Message from Public and Shared
paulson [Fri, 11 Jul 1997 13:27:15 +0200] rev 3513
Now loads theory Event, which contains common declarations
paulson [Fri, 11 Jul 1997 13:26:15 +0200] rev 3512
Moving common declarations and proofs from theories "Shared"
and "Public" to "Event". NB the original "Event" theory was later renamed "Shared".
Addition of the Notes constructor to datatype "event".
wenzelm [Wed, 09 Jul 1997 17:00:34 +0200] rev 3511
removed obsolete init_pps and init_thy_reader;
wenzelm [Wed, 09 Jul 1997 16:54:17 +0200] rev 3510
improved type checking errors;
wenzelm [Wed, 09 Jul 1997 16:53:53 +0200] rev 3509
removed init_pps;
wenzelm [Wed, 09 Jul 1997 16:52:51 +0200] rev 3508
removed init_database;
nipkow [Wed, 09 Jul 1997 12:57:04 +0200] rev 3507
Improved length = size translation.
paulson [Mon, 07 Jul 1997 10:49:14 +0200] rev 3506
New proofs involving CERTIFICATE VERIFY
wenzelm [Mon, 07 Jul 1997 09:09:21 +0200] rev 3505
eliminated chmod -w;
wenzelm [Mon, 07 Jul 1997 09:07:08 +0200] rev 3504
-w option;
wenzelm [Mon, 07 Jul 1997 09:06:26 +0200] rev 3503
NOWRITE;
wenzelm [Mon, 07 Jul 1997 09:05:16 +0200] rev 3502
added -w option;
paulson [Fri, 04 Jul 1997 17:36:41 +0200] rev 3501
Changed some variables of type msg to lower case (e.g. from NB to nb
paulson [Fri, 04 Jul 1997 17:34:55 +0200] rev 3500
New constant "certificate"--just an abbreviation
nipkow [Fri, 04 Jul 1997 14:37:30 +0200] rev 3499
Reduced priority of postfix ^* etc operators such that they are the same as
application. Eg wf r^* now needs to be written wf(r^*).
paulson [Fri, 04 Jul 1997 12:36:00 +0200] rev 3498
Automatic update
paulson [Fri, 04 Jul 1997 12:32:31 +0200] rev 3497
Now catches the error of calling tgoalw when there are no goals to prove,
instead of just letting USyntax.list_mk_conj raise an exception
paulson [Fri, 04 Jul 1997 12:31:20 +0200] rev 3496
Simplified the new proofs about division
paulson [Fri, 04 Jul 1997 11:57:33 +0200] rev 3495
New comments on how to deal with unproved termination conditions
paulson [Fri, 04 Jul 1997 11:56:49 +0200] rev 3494
Fixed comments