Fri, 26 Sep 2008 14:51:27 +0200 Added some more lemmas that are useful in proof of strong induction rule.
berghofe [Fri, 26 Sep 2008 14:51:27 +0200] rev 28371
Added some more lemmas that are useful in proof of strong induction rule.
Fri, 26 Sep 2008 09:10:02 +0200 removed obsolete name convention "func"
haftmann [Fri, 26 Sep 2008 09:10:02 +0200] rev 28370
removed obsolete name convention "func"
Fri, 26 Sep 2008 09:09:53 +0200 fixed typo
haftmann [Fri, 26 Sep 2008 09:09:53 +0200] rev 28369
fixed typo
Fri, 26 Sep 2008 09:09:52 +0200 clarified function transformator interface
haftmann [Fri, 26 Sep 2008 09:09:52 +0200] rev 28368
clarified function transformator interface
Fri, 26 Sep 2008 09:09:51 +0200 op = vs. eq
haftmann [Fri, 26 Sep 2008 09:09:51 +0200] rev 28367
op = vs. eq
Thu, 25 Sep 2008 20:34:21 +0200 moved future_scheduler flag to skip_proof.ML;
wenzelm [Thu, 25 Sep 2008 20:34:21 +0200] rev 28366
moved future_scheduler flag to skip_proof.ML;
Thu, 25 Sep 2008 20:34:20 +0200 added future_scheduler (from thy_info.ML);
wenzelm [Thu, 25 Sep 2008 20:34:20 +0200] rev 28365
added future_scheduler (from thy_info.ML); prove: Goal.prove_promise if future_schedule;
Thu, 25 Sep 2008 20:34:19 +0200 simplified promise;
wenzelm [Thu, 25 Sep 2008 20:34:19 +0200] rev 28364
simplified promise; fulfill is internal only; more robust join_futures;
Thu, 25 Sep 2008 20:34:18 +0200 simplified Thm.promise;
wenzelm [Thu, 25 Sep 2008 20:34:18 +0200] rev 28363
simplified Thm.promise; prove_common: proper context for promise_result;
Thu, 25 Sep 2008 20:34:17 +0200 explicit checkpoint for low-level (global) theory operations admits concurrent SkipProof.prove;
wenzelm [Thu, 25 Sep 2008 20:34:17 +0200] rev 28362
explicit checkpoint for low-level (global) theory operations admits concurrent SkipProof.prove; tuned list operations;
Thu, 25 Sep 2008 20:34:15 +0200 explicit checkpoint for low-level (global) theory operations, admits concurrent proofs;
wenzelm [Thu, 25 Sep 2008 20:34:15 +0200] rev 28361
explicit checkpoint for low-level (global) theory operations, admits concurrent proofs;
Thu, 25 Sep 2008 19:15:50 +0200 circumvent problem with code redundancy
haftmann [Thu, 25 Sep 2008 19:15:50 +0200] rev 28360
circumvent problem with code redundancy
Thu, 25 Sep 2008 16:05:52 +0200 clarifed redundancy policy
haftmann [Thu, 25 Sep 2008 16:05:52 +0200] rev 28359
clarifed redundancy policy
Thu, 25 Sep 2008 14:37:32 +0200 tuned comments;
wenzelm [Thu, 25 Sep 2008 14:37:32 +0200] rev 28358
tuned comments;
Thu, 25 Sep 2008 14:35:03 +0200 added release_results;
wenzelm [Thu, 25 Sep 2008 14:35:03 +0200] rev 28357
added release_results; tuned comments;
Thu, 25 Sep 2008 14:35:02 +0200 abtract types: plain datatype with opaque signature matching;
wenzelm [Thu, 25 Sep 2008 14:35:02 +0200] rev 28356
abtract types: plain datatype with opaque signature matching; promise: join pending futures at end of theory;
Thu, 25 Sep 2008 14:35:01 +0200 prove: error with original thread position;
wenzelm [Thu, 25 Sep 2008 14:35:01 +0200] rev 28355
prove: error with original thread position;
Thu, 25 Sep 2008 13:21:13 +0200 explicit type OrdList.T;
wenzelm [Thu, 25 Sep 2008 13:21:13 +0200] rev 28354
explicit type OrdList.T;
Thu, 25 Sep 2008 11:14:01 +0200 (temporary workaround)
haftmann [Thu, 25 Sep 2008 11:14:01 +0200] rev 28353
(temporary workaround)
Thu, 25 Sep 2008 10:17:23 +0200 (temporal deactivation)
haftmann [Thu, 25 Sep 2008 10:17:23 +0200] rev 28352
(temporal deactivation)
Thu, 25 Sep 2008 10:17:22 +0200 non left-linear equations for nbe
haftmann [Thu, 25 Sep 2008 10:17:22 +0200] rev 28351
non left-linear equations for nbe
Thu, 25 Sep 2008 09:28:08 +0200 non left-linear equations for nbe
haftmann [Thu, 25 Sep 2008 09:28:08 +0200] rev 28350
non left-linear equations for nbe
Thu, 25 Sep 2008 09:28:07 +0200 map_force
haftmann [Thu, 25 Sep 2008 09:28:07 +0200] rev 28349
map_force
Thu, 25 Sep 2008 09:28:06 +0200 matchess
haftmann [Thu, 25 Sep 2008 09:28:06 +0200] rev 28348
matchess
Thu, 25 Sep 2008 09:28:05 +0200 burrow_fst
haftmann [Thu, 25 Sep 2008 09:28:05 +0200] rev 28347
burrow_fst
Thu, 25 Sep 2008 09:28:03 +0200 discontinued special treatment of op = vs. eq_class.eq
haftmann [Thu, 25 Sep 2008 09:28:03 +0200] rev 28346
discontinued special treatment of op = vs. eq_class.eq
Wed, 24 Sep 2008 19:39:25 +0200 report: produce individual status messages;
wenzelm [Wed, 24 Sep 2008 19:39:25 +0200] rev 28345
report: produce individual status messages;
Wed, 24 Sep 2008 19:33:14 +0200 protocol change: remapped message codes to make room for nested system messages (e.g. for protocol proxy);
wenzelm [Wed, 24 Sep 2008 19:33:14 +0200] rev 28344
protocol change: remapped message codes to make room for nested system messages (e.g. for protocol proxy); added Kind.code map;
Wed, 24 Sep 2008 19:33:13 +0200 protocol change: remapped message codes to make room for nested system messages (e.g. for protocol proxy);
wenzelm [Wed, 24 Sep 2008 19:33:13 +0200] rev 28343
protocol change: remapped message codes to make room for nested system messages (e.g. for protocol proxy);
Wed, 24 Sep 2008 18:08:42 +0200 init: OuterKeyword.report;
wenzelm [Wed, 24 Sep 2008 18:08:42 +0200] rev 28342
init: OuterKeyword.report;
Tue, 23 Sep 2008 23:07:48 +0200 prove_multi: immediate;
wenzelm [Tue, 23 Sep 2008 23:07:48 +0200] rev 28341
prove_multi: immediate;
Tue, 23 Sep 2008 22:04:30 +0200 added promise_result, prove_promise;
wenzelm [Tue, 23 Sep 2008 22:04:30 +0200] rev 28340
added promise_result, prove_promise;
Tue, 23 Sep 2008 18:31:33 +0200 Corrected call of SUBPROOF in coherent_tac that used wrong context.
berghofe [Tue, 23 Sep 2008 18:31:33 +0200] rev 28339
Corrected call of SUBPROOF in coherent_tac that used wrong context.
Tue, 23 Sep 2008 18:11:45 +0200 fixed outer syntax
haftmann [Tue, 23 Sep 2008 18:11:45 +0200] rev 28338
fixed outer syntax
Tue, 23 Sep 2008 18:11:44 +0200 case default fallback for NBE
haftmann [Tue, 23 Sep 2008 18:11:44 +0200] rev 28337
case default fallback for NBE
Tue, 23 Sep 2008 18:11:43 +0200 fixed quickcheck parameter syntax
haftmann [Tue, 23 Sep 2008 18:11:43 +0200] rev 28336
fixed quickcheck parameter syntax
Tue, 23 Sep 2008 18:11:42 +0200 renamed rtype to typerep
haftmann [Tue, 23 Sep 2008 18:11:42 +0200] rev 28335
renamed rtype to typerep
Tue, 23 Sep 2008 17:28:58 +0200 added fold_rev;
wenzelm [Tue, 23 Sep 2008 17:28:58 +0200] rev 28334
added fold_rev; tuned dest, keys;
Tue, 23 Sep 2008 15:48:55 +0200 added del_node, which is more efficient for sparse graphs;
wenzelm [Tue, 23 Sep 2008 15:48:55 +0200] rev 28333
added del_node, which is more efficient for sparse graphs;
Tue, 23 Sep 2008 15:48:54 +0200 IntGraph.del_node;
wenzelm [Tue, 23 Sep 2008 15:48:54 +0200] rev 28332
IntGraph.del_node;
Tue, 23 Sep 2008 15:48:53 +0200 join_results: special case for empty list, works without multithreading;
wenzelm [Tue, 23 Sep 2008 15:48:53 +0200] rev 28331
join_results: special case for empty list, works without multithreading;
Tue, 23 Sep 2008 15:48:52 +0200 added dest_deriv, removed external type deriv;
wenzelm [Tue, 23 Sep 2008 15:48:52 +0200] rev 28330
added dest_deriv, removed external type deriv; misc tuning of internal deriv; more substantial promise/fulfill; promise_ord: reverse order on serial numbers; removed unused is_named; get_name: unfinished proof term;
Tue, 23 Sep 2008 15:48:51 +0200 added conditional add_oracles, keep oracles_of_proof private;
wenzelm [Tue, 23 Sep 2008 15:48:51 +0200] rev 28329
added conditional add_oracles, keep oracles_of_proof private; added fulfill; removed unused is_named; tuned some table operations;
Tue, 23 Sep 2008 15:48:50 +0200 Thm.proof_of;
wenzelm [Tue, 23 Sep 2008 15:48:50 +0200] rev 28328
Thm.proof_of;
Mon, 22 Sep 2008 23:04:35 +0200 Added coherent logic prover.
berghofe [Mon, 22 Sep 2008 23:04:35 +0200] rev 28327
Added coherent logic prover.
Mon, 22 Sep 2008 23:01:54 +0200 New prover for coherent logic.
berghofe [Mon, 22 Sep 2008 23:01:54 +0200] rev 28326
New prover for coherent logic.
Mon, 22 Sep 2008 23:00:15 +0200 Added setup for coherent logic prover.
berghofe [Mon, 22 Sep 2008 23:00:15 +0200] rev 28325
Added setup for coherent logic prover.
Mon, 22 Sep 2008 22:59:35 +0200 Added examples for coherent logic prover.
berghofe [Mon, 22 Sep 2008 22:59:35 +0200] rev 28324
Added examples for coherent logic prover.
Mon, 22 Sep 2008 22:59:11 +0200 Examples for coherent logic prover.
berghofe [Mon, 22 Sep 2008 22:59:11 +0200] rev 28323
Examples for coherent logic prover.
Mon, 22 Sep 2008 19:46:24 +0200 made the perm_simp tactic to understand options such as (no_asm)
urbanc [Mon, 22 Sep 2008 19:46:24 +0200] rev 28322
made the perm_simp tactic to understand options such as (no_asm)
Mon, 22 Sep 2008 15:26:14 +0200 type thm: fully internal derivation, no longer exported;
wenzelm [Mon, 22 Sep 2008 15:26:14 +0200] rev 28321
type thm: fully internal derivation, no longer exported; incorporate former deriv.ML as internal abstract type; added rudimentary promise interface; tuned; added is_named (does not require finished derivation);
Mon, 22 Sep 2008 15:26:14 +0200 added is_finished;
wenzelm [Mon, 22 Sep 2008 15:26:14 +0200] rev 28320
added is_finished;
Mon, 22 Sep 2008 15:26:13 +0200 added Promise constructor, which is similar to Oracle but may be replaced later;
wenzelm [Mon, 22 Sep 2008 15:26:13 +0200] rev 28319
added Promise constructor, which is similar to Oracle but may be replaced later; added promise_proof; export min_proof, mk_min_proof; moved infer_derivs to thm.ML as derive_rule0/1/2; tuned oracles_of_proof; added is_named;
Mon, 22 Sep 2008 15:26:11 +0200 removed deriv.ML which is now incorporated into thm.ML;
wenzelm [Mon, 22 Sep 2008 15:26:11 +0200] rev 28318
removed deriv.ML which is now incorporated into thm.ML;
Mon, 22 Sep 2008 15:26:11 +0200 added reject_draft;
wenzelm [Mon, 22 Sep 2008 15:26:11 +0200] rev 28317
added reject_draft;
Mon, 22 Sep 2008 15:26:07 +0200 type thm: fully internal derivation, no longer exported;
wenzelm [Mon, 22 Sep 2008 15:26:07 +0200] rev 28316
type thm: fully internal derivation, no longer exported;
Mon, 22 Sep 2008 13:56:04 +0200 generic quickcheck framework
haftmann [Mon, 22 Sep 2008 13:56:04 +0200] rev 28315
generic quickcheck framework
Mon, 22 Sep 2008 13:56:03 +0200 TEMPORARY: make batch run happy
haftmann [Mon, 22 Sep 2008 13:56:03 +0200] rev 28314
TEMPORARY: make batch run happy
Mon, 22 Sep 2008 13:56:01 +0200 absolute Library path
haftmann [Mon, 22 Sep 2008 13:56:01 +0200] rev 28313
absolute Library path
Mon, 22 Sep 2008 13:55:59 +0200 different session branches for HOL-Plain vs. Plain
haftmann [Mon, 22 Sep 2008 13:55:59 +0200] rev 28312
different session branches for HOL-Plain vs. Plain
(0) -10000 -3000 -1000 -300 -100 -60 +60 +100 +300 +1000 +3000 +10000 +30000 tip