Mon, 22 Aug 2011 17:22:49 -0700 avoid warnings
huffman [Mon, 22 Aug 2011 17:22:49 -0700] rev 44454
avoid warnings
Mon, 22 Aug 2011 16:49:45 -0700 comment out dead code to avoid compiler warnings
huffman [Mon, 22 Aug 2011 16:49:45 -0700] rev 44453
comment out dead code to avoid compiler warnings
Mon, 22 Aug 2011 10:43:10 -0700 legacy theorem names
huffman [Mon, 22 Aug 2011 10:43:10 -0700] rev 44452
legacy theorem names
Mon, 22 Aug 2011 10:19:39 -0700 remove duplicate lemma
huffman [Mon, 22 Aug 2011 10:19:39 -0700] rev 44451
remove duplicate lemma
Tue, 23 Aug 2011 23:18:13 +0200 fixed "hBOOL" of existential variables, and generate more helpers
blanchet [Tue, 23 Aug 2011 23:18:13 +0200] rev 44450
fixed "hBOOL" of existential variables, and generate more helpers
Tue, 23 Aug 2011 22:44:08 +0200 don't select facts when using sledgehammer_tac for reconstruction
blanchet [Tue, 23 Aug 2011 22:44:08 +0200] rev 44449
don't select facts when using sledgehammer_tac for reconstruction
Tue, 23 Aug 2011 20:35:41 +0200 don't perform a triviality check if the goal is skipped anyway
blanchet [Tue, 23 Aug 2011 20:35:41 +0200] rev 44448
don't perform a triviality check if the goal is skipped anyway
Tue, 23 Aug 2011 19:50:25 +0200 optional reconstructor
blanchet [Tue, 23 Aug 2011 19:50:25 +0200] rev 44447
optional reconstructor
Wed, 24 Aug 2011 17:25:45 +0200 misc tuning and simplification;
wenzelm [Wed, 24 Aug 2011 17:25:45 +0200] rev 44446
misc tuning and simplification;
Wed, 24 Aug 2011 17:16:48 +0200 tuned pri: prefer purging of canceled execution;
wenzelm [Wed, 24 Aug 2011 17:16:48 +0200] rev 44445
tuned pri: prefer purging of canceled execution;
Wed, 24 Aug 2011 17:14:31 +0200 tuned Document.node: maintain "touched" flag to indicate changes in entries etc.;
wenzelm [Wed, 24 Aug 2011 17:14:31 +0200] rev 44444
tuned Document.node: maintain "touched" flag to indicate changes in entries etc.;
Wed, 24 Aug 2011 16:49:48 +0200 clarified Document.Node.clear -- retain header (cf. ML version);
wenzelm [Wed, 24 Aug 2011 16:49:48 +0200] rev 44443
clarified Document.Node.clear -- retain header (cf. ML version);
Wed, 24 Aug 2011 16:27:27 +0200 clarified norm_header/header_edit -- disallow update of loaded theories;
wenzelm [Wed, 24 Aug 2011 16:27:27 +0200] rev 44442
clarified norm_header/header_edit -- disallow update of loaded theories;
Wed, 24 Aug 2011 15:55:43 +0200 misc tuning and simplification;
wenzelm [Wed, 24 Aug 2011 15:55:43 +0200] rev 44441
misc tuning and simplification;
Wed, 24 Aug 2011 15:30:43 +0200 ignore irrelevant timings;
wenzelm [Wed, 24 Aug 2011 15:30:43 +0200] rev 44440
ignore irrelevant timings;
Wed, 24 Aug 2011 13:40:10 +0200 print state only for visible command, to avoid wasting resources for the larger part of the text;
wenzelm [Wed, 24 Aug 2011 13:40:10 +0200] rev 44439
print state only for visible command, to avoid wasting resources for the larger part of the text;
Wed, 24 Aug 2011 13:38:07 +0200 early filtering of unchanged perspective;
wenzelm [Wed, 24 Aug 2011 13:38:07 +0200] rev 44438
early filtering of unchanged perspective;
Wed, 24 Aug 2011 13:37:43 +0200 more reliable update_perspective handler based on actual text visibility (e.g. on startup or when resizing without scrolling);
wenzelm [Wed, 24 Aug 2011 13:37:43 +0200] rev 44437
more reliable update_perspective handler based on actual text visibility (e.g. on startup or when resizing without scrolling);
Wed, 24 Aug 2011 13:03:39 +0200 update_perspective without actual edits, bypassing the full state assignment protocol;
wenzelm [Wed, 24 Aug 2011 13:03:39 +0200] rev 44436
update_perspective without actual edits, bypassing the full state assignment protocol; edit_nodes/Perspective: do not touch_descendants here; propagate editor scroll events via update_perspective; misc tuning;
Tue, 23 Aug 2011 21:19:24 +0200 tuned;
wenzelm [Tue, 23 Aug 2011 21:19:24 +0200] rev 44435
tuned;
Tue, 23 Aug 2011 21:14:59 +0200 handle potentially more approriate BufferUpdate.LOADED event;
wenzelm [Tue, 23 Aug 2011 21:14:59 +0200] rev 44434
handle potentially more approriate BufferUpdate.LOADED event;
Mon, 22 Aug 2011 23:39:05 +0200 special treatment of structure index 1 in Pure, including legacy warning;
wenzelm [Mon, 22 Aug 2011 23:39:05 +0200] rev 44433
special treatment of structure index 1 in Pure, including legacy warning;
Tue, 23 Aug 2011 19:49:21 +0200 compile
blanchet [Tue, 23 Aug 2011 19:49:21 +0200] rev 44432
compile
Tue, 23 Aug 2011 19:00:48 +0200 added "max_calls" option to get a fixed number of Sledgehammer calls per theory
blanchet [Tue, 23 Aug 2011 19:00:48 +0200] rev 44431
added "max_calls" option to get a fixed number of Sledgehammer calls per theory
Tue, 23 Aug 2011 18:42:05 +0200 beef up "sledgehammer_tac" reconstructor
blanchet [Tue, 23 Aug 2011 18:42:05 +0200] rev 44430
beef up "sledgehammer_tac" reconstructor
Tue, 23 Aug 2011 18:42:05 +0200 clean up Sledgehammer tactic
blanchet [Tue, 23 Aug 2011 18:42:05 +0200] rev 44429
clean up Sledgehammer tactic
Tue, 23 Aug 2011 17:44:31 +0200 fixed document;
wenzelm [Tue, 23 Aug 2011 17:44:31 +0200] rev 44428
fixed document;
Tue, 23 Aug 2011 17:43:06 +0200 tuned signature;
wenzelm [Tue, 23 Aug 2011 17:43:06 +0200] rev 44427
tuned signature;
Tue, 23 Aug 2011 17:12:54 +0200 merged
wenzelm [Tue, 23 Aug 2011 17:12:54 +0200] rev 44426
merged
Tue, 23 Aug 2011 16:37:23 +0200 always use TFF if possible
blanchet [Tue, 23 Aug 2011 16:37:23 +0200] rev 44425
always use TFF if possible
Tue, 23 Aug 2011 16:14:19 +0200 clearer separator in generated file names
blanchet [Tue, 23 Aug 2011 16:14:19 +0200] rev 44424
clearer separator in generated file names
Tue, 23 Aug 2011 16:07:01 +0200 exploit TFF format in Z3 used as ATP, and renamed it "z3_tptp"
blanchet [Tue, 23 Aug 2011 16:07:01 +0200] rev 44423
exploit TFF format in Z3 used as ATP, and renamed it "z3_tptp"
Tue, 23 Aug 2011 15:50:27 +0200 updated known failures for Z3 3.0 TPTP
blanchet [Tue, 23 Aug 2011 15:50:27 +0200] rev 44422
updated known failures for Z3 3.0 TPTP
Tue, 23 Aug 2011 15:18:46 +0200 updated Z3 docs
blanchet [Tue, 23 Aug 2011 15:18:46 +0200] rev 44421
updated Z3 docs
Tue, 23 Aug 2011 15:15:43 +0200 avoid TFF format with older Vampire versions
blanchet [Tue, 23 Aug 2011 15:15:43 +0200] rev 44420
avoid TFF format with older Vampire versions
Tue, 23 Aug 2011 14:57:16 +0200 update the Vampire related parts of the documentation
blanchet [Tue, 23 Aug 2011 14:57:16 +0200] rev 44419
update the Vampire related parts of the documentation
Tue, 23 Aug 2011 14:44:19 +0200 fixed TFF slicing
blanchet [Tue, 23 Aug 2011 14:44:19 +0200] rev 44418
fixed TFF slicing
Tue, 23 Aug 2011 14:44:19 +0200 kindly ask Vampire to output axiom names
blanchet [Tue, 23 Aug 2011 14:44:19 +0200] rev 44417
kindly ask Vampire to output axiom names
Tue, 23 Aug 2011 14:44:19 +0200 added formats to the slice and use TFF for remote Vampire
blanchet [Tue, 23 Aug 2011 14:44:19 +0200] rev 44416
added formats to the slice and use TFF for remote Vampire
Tue, 23 Aug 2011 07:14:09 +0200 tuned specifications, syntax and proofs
haftmann [Tue, 23 Aug 2011 07:14:09 +0200] rev 44415
tuned specifications, syntax and proofs
Mon, 22 Aug 2011 22:00:36 +0200 tuned specifications and syntax
haftmann [Mon, 22 Aug 2011 22:00:36 +0200] rev 44414
tuned specifications and syntax
Tue, 23 Aug 2011 03:34:17 +0900 Quotient Package: some infrastructure for lifting inside sets
Cezary Kaliszyk <kaliszyk@in.tum.de> [Tue, 23 Aug 2011 03:34:17 +0900] rev 44413
Quotient Package: some infrastructure for lifting inside sets
Mon, 22 Aug 2011 15:02:45 +0200 include all encodings in tests, now that the incompleteness of some encodings has been addressed
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44412
include all encodings in tests, now that the incompleteness of some encodings has been addressed
Mon, 22 Aug 2011 15:02:45 +0200 change Metis's default settings if type information axioms are generated
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44411
change Metis's default settings if type information axioms are generated
Mon, 22 Aug 2011 15:02:45 +0200 we must tag any type whose ground types intersect a nonmonotonic type
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44410
we must tag any type whose ground types intersect a nonmonotonic type
Mon, 22 Aug 2011 15:02:45 +0200 prefer the lighter, slightly unsound monotonicity-based encodings for Metis
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44409
prefer the lighter, slightly unsound monotonicity-based encodings for Metis
Mon, 22 Aug 2011 15:02:45 +0200 made reconstruction of type tag equalities "\?x = \?x" reliable
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44408
made reconstruction of type tag equalities "\?x = \?x" reliable
Mon, 22 Aug 2011 15:02:45 +0200 tuning ATP problem output
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44407
tuning ATP problem output
Mon, 22 Aug 2011 15:02:45 +0200 revert guard logic -- make sure that typing information is generated for existentials
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44406
revert guard logic -- make sure that typing information is generated for existentials
Mon, 22 Aug 2011 15:02:45 +0200 generate tag equations for existential variables
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44405
generate tag equations for existential variables
Mon, 22 Aug 2011 15:02:45 +0200 tuning, plus started implementing tag equation generation for existential variables
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44404
tuning, plus started implementing tag equation generation for existential variables
Mon, 22 Aug 2011 15:02:45 +0200 precisely distinguish between universal and existential quantifiers, instead of assuming the worst (universal), for monotonicity analysis
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44403
precisely distinguish between universal and existential quantifiers, instead of assuming the worst (universal), for monotonicity analysis
Mon, 22 Aug 2011 15:02:45 +0200 clearer terminology
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44402
clearer terminology
Mon, 22 Aug 2011 15:02:45 +0200 renamed "heavy" to "uniform", based on discussion with Nick Smallbone
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44401
renamed "heavy" to "uniform", based on discussion with Nick Smallbone
Mon, 22 Aug 2011 15:02:45 +0200 removed unused configuration option
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44400
removed unused configuration option
Mon, 22 Aug 2011 15:02:45 +0200 added caching for (in)finiteness checks
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44399
added caching for (in)finiteness checks
Mon, 22 Aug 2011 15:02:45 +0200 remove needless typing information
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44398
remove needless typing information
Mon, 22 Aug 2011 15:02:45 +0200 cleaner handling of polymorphic monotonicity inference
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44397
cleaner handling of polymorphic monotonicity inference
Mon, 22 Aug 2011 15:02:45 +0200 started cleaning up polymorphic monotonicity-based encodings, based on discussions with Nick Smallbone
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44396
started cleaning up polymorphic monotonicity-based encodings, based on discussions with Nick Smallbone
Mon, 22 Aug 2011 15:02:45 +0200 more precise warning
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44395
more precise warning
Mon, 22 Aug 2011 15:02:45 +0200 added option to control soundness of encodings more precisely, for evaluation purposes
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44394
added option to control soundness of encodings more precisely, for evaluation purposes
Mon, 22 Aug 2011 15:02:45 +0200 make sound mode more sound (and clean up code)
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44393
make sound mode more sound (and clean up code)
Mon, 22 Aug 2011 15:02:45 +0200 reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44392
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
Mon, 22 Aug 2011 15:02:45 +0200 gracefully handle empty SPASS problems
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44391
gracefully handle empty SPASS problems
Mon, 22 Aug 2011 15:02:45 +0200 pass sound option to Sledgehammer tactic
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44390
pass sound option to Sledgehammer tactic
Tue, 23 Aug 2011 16:53:05 +0200 tuned signature -- contrast physical output primitives versus Output.raw_message;
wenzelm [Tue, 23 Aug 2011 16:53:05 +0200] rev 44389
tuned signature -- contrast physical output primitives versus Output.raw_message;
Tue, 23 Aug 2011 16:41:16 +0200 tuned signature;
wenzelm [Tue, 23 Aug 2011 16:41:16 +0200] rev 44388
tuned signature;
Tue, 23 Aug 2011 16:39:21 +0200 discontinued slightly odd Future/Lazy.get_finished, which do not really fit into the execution model of Future.cancel/join_tasks (canceled tasks need to be dequeued and terminated explicitly);
wenzelm [Tue, 23 Aug 2011 16:39:21 +0200] rev 44387
discontinued slightly odd Future/Lazy.get_finished, which do not really fit into the execution model of Future.cancel/join_tasks (canceled tasks need to be dequeued and terminated explicitly);
Tue, 23 Aug 2011 15:48:41 +0200 some support for toplevel printing wrt. editor perspective (still inactive);
wenzelm [Tue, 23 Aug 2011 15:48:41 +0200] rev 44386
some support for toplevel printing wrt. editor perspective (still inactive);
Tue, 23 Aug 2011 12:20:12 +0200 propagate editor perspective through document model;
wenzelm [Tue, 23 Aug 2011 12:20:12 +0200] rev 44385
propagate editor perspective through document model;
Mon, 22 Aug 2011 21:42:02 +0200 some support for editor perspective;
wenzelm [Mon, 22 Aug 2011 21:42:02 +0200] rev 44384
some support for editor perspective;
Mon, 22 Aug 2011 21:09:26 +0200 discontinued redundant Edit_Command_ID;
wenzelm [Mon, 22 Aug 2011 21:09:26 +0200] rev 44383
discontinued redundant Edit_Command_ID;
Mon, 22 Aug 2011 20:11:44 +0200 reduced warnings;
wenzelm [Mon, 22 Aug 2011 20:11:44 +0200] rev 44382
reduced warnings;
Mon, 22 Aug 2011 20:00:04 +0200 tuned message;
wenzelm [Mon, 22 Aug 2011 20:00:04 +0200] rev 44381
tuned message;
Mon, 22 Aug 2011 17:10:22 +0200 old-style numbered structure index is legacy feature (hardly ever used now);
wenzelm [Mon, 22 Aug 2011 17:10:22 +0200] rev 44380
old-style numbered structure index is legacy feature (hardly ever used now);
Mon, 22 Aug 2011 16:12:23 +0200 added official Text.Range.Ordering;
wenzelm [Mon, 22 Aug 2011 16:12:23 +0200] rev 44379
added official Text.Range.Ordering; some support for text perspective;
Mon, 22 Aug 2011 14:15:52 +0200 tuned signature;
wenzelm [Mon, 22 Aug 2011 14:15:52 +0200] rev 44378
tuned signature;
Mon, 22 Aug 2011 12:17:22 +0200 reverted some odd changes to HOL/Import (cf. 74c08021ab2e);
wenzelm [Mon, 22 Aug 2011 12:17:22 +0200] rev 44377
reverted some odd changes to HOL/Import (cf. 74c08021ab2e);
Mon, 22 Aug 2011 10:57:33 +0200 merged
krauss [Mon, 22 Aug 2011 10:57:33 +0200] rev 44376
merged
Sun, 21 Aug 2011 22:13:04 +0200 modernized specifications
krauss [Sun, 21 Aug 2011 22:13:04 +0200] rev 44375
modernized specifications
Sun, 21 Aug 2011 22:13:04 +0200 removed session HOL/Subst -- now subsumed my more modern HOL/ex/Unification.thy
krauss [Sun, 21 Aug 2011 22:13:04 +0200] rev 44374
removed session HOL/Subst -- now subsumed my more modern HOL/ex/Unification.thy
Sun, 21 Aug 2011 22:13:04 +0200 removed technical or trivial unused facts
krauss [Sun, 21 Aug 2011 22:13:04 +0200] rev 44373
removed technical or trivial unused facts
Sun, 21 Aug 2011 22:13:04 +0200 more precise authors and comments;
krauss [Sun, 21 Aug 2011 22:13:04 +0200] rev 44372
more precise authors and comments; tuned order and headers
Sun, 21 Aug 2011 22:13:04 +0200 added proof of idempotence, roughly after HOL/Subst/Unify.thy
krauss [Sun, 21 Aug 2011 22:13:04 +0200] rev 44371
added proof of idempotence, roughly after HOL/Subst/Unify.thy
Sun, 21 Aug 2011 22:13:04 +0200 tuned proofs, sledgehammering overly verbose parts
krauss [Sun, 21 Aug 2011 22:13:04 +0200] rev 44370
tuned proofs, sledgehammering overly verbose parts
Sun, 21 Aug 2011 22:13:04 +0200 tuned notation
krauss [Sun, 21 Aug 2011 22:13:04 +0200] rev 44369
tuned notation
Sun, 21 Aug 2011 22:13:04 +0200 ported some lemmas from HOL/Subst/*;
krauss [Sun, 21 Aug 2011 22:13:04 +0200] rev 44368
ported some lemmas from HOL/Subst/*; tuned order
Sun, 21 Aug 2011 22:13:04 +0200 changed constant names and notation to match HOL/Subst/*.thy, from which this theory is a clone.
krauss [Sun, 21 Aug 2011 22:13:04 +0200] rev 44367
changed constant names and notation to match HOL/Subst/*.thy, from which this theory is a clone.
Sun, 21 Aug 2011 21:18:59 -0700 merged
huffman [Sun, 21 Aug 2011 21:18:59 -0700] rev 44366
merged
Sun, 21 Aug 2011 12:22:31 -0700 add lemmas interior_Times and closure_Times
huffman [Sun, 21 Aug 2011 12:22:31 -0700] rev 44365
add lemmas interior_Times and closure_Times
Sun, 21 Aug 2011 22:56:55 +0200 avoid pred/set mixture
haftmann [Sun, 21 Aug 2011 22:56:55 +0200] rev 44364
avoid pred/set mixture
Sun, 21 Aug 2011 19:47:52 +0200 avoid pred/set mixture
haftmann [Sun, 21 Aug 2011 19:47:52 +0200] rev 44363
avoid pred/set mixture
Sun, 21 Aug 2011 22:04:01 +0200 merged
wenzelm [Sun, 21 Aug 2011 22:04:01 +0200] rev 44362
merged
Sun, 21 Aug 2011 11:03:15 -0700 remove unnecessary euclidean_space class constraints
huffman [Sun, 21 Aug 2011 11:03:15 -0700] rev 44361
remove unnecessary euclidean_space class constraints
Sun, 21 Aug 2011 09:46:20 -0700 section -> subsection
huffman [Sun, 21 Aug 2011 09:46:20 -0700] rev 44360
section -> subsection
Sun, 21 Aug 2011 09:38:31 -0700 scale dependency graph to fit on page
huffman [Sun, 21 Aug 2011 09:38:31 -0700] rev 44359
scale dependency graph to fit on page
Sun, 21 Aug 2011 21:24:42 +0200 more robust initialization of token marker and line context wrt. session startup;
wenzelm [Sun, 21 Aug 2011 21:24:42 +0200] rev 44358
more robust initialization of token marker and line context wrt. session startup;
Sun, 21 Aug 2011 20:42:26 +0200 tuned Parse.group: delayed failure message;
wenzelm [Sun, 21 Aug 2011 20:42:26 +0200] rev 44357
tuned Parse.group: delayed failure message;
Sun, 21 Aug 2011 20:25:49 +0200 avoid actual Color.white, which would be turned into Color.black by org.gjt.sp.jedit.print.BufferPrintable;
wenzelm [Sun, 21 Aug 2011 20:25:49 +0200] rev 44356
avoid actual Color.white, which would be turned into Color.black by org.gjt.sp.jedit.print.BufferPrintable;
Sun, 21 Aug 2011 20:04:02 +0200 default style for user fonts -- to prevent org.gjt.sp.jedit.print.BufferPrintable from choking on null;
wenzelm [Sun, 21 Aug 2011 20:04:02 +0200] rev 44355
default style for user fonts -- to prevent org.gjt.sp.jedit.print.BufferPrintable from choking on null;
Sun, 21 Aug 2011 19:32:20 +0200 tuned;
wenzelm [Sun, 21 Aug 2011 19:32:20 +0200] rev 44354
tuned;
Sun, 21 Aug 2011 14:16:44 +0200 discontinued somewhat pointless Par_List.map_name -- most of the time is spent in tokenization;
wenzelm [Sun, 21 Aug 2011 14:16:44 +0200] rev 44353
discontinued somewhat pointless Par_List.map_name -- most of the time is spent in tokenization;
Sun, 21 Aug 2011 13:42:55 +0200 discontinued obsolete Thy_Syntax.report_span -- information can be reproduced in Isabelle/Scala;
wenzelm [Sun, 21 Aug 2011 13:42:55 +0200] rev 44352
discontinued obsolete Thy_Syntax.report_span -- information can be reproduced in Isabelle/Scala;
Sun, 21 Aug 2011 13:36:23 +0200 merged
wenzelm [Sun, 21 Aug 2011 13:36:23 +0200] rev 44351
merged
Sat, 20 Aug 2011 15:19:35 -0700 replace lemma realpow_two_diff with new lemma square_diff_square_factored
huffman [Sat, 20 Aug 2011 15:19:35 -0700] rev 44350
replace lemma realpow_two_diff with new lemma square_diff_square_factored
Sat, 20 Aug 2011 15:54:26 -0700 remove redundant lemma real_0_le_divide_iff in favor or zero_le_divide_iff
huffman [Sat, 20 Aug 2011 15:54:26 -0700] rev 44349
remove redundant lemma real_0_le_divide_iff in favor or zero_le_divide_iff
Sat, 20 Aug 2011 13:07:00 -0700 move lemma add_eq_0_iff to Groups.thy
huffman [Sat, 20 Aug 2011 13:07:00 -0700] rev 44348
move lemma add_eq_0_iff to Groups.thy
Sat, 20 Aug 2011 12:51:15 -0700 remove redundant lemma realpow_two_disj, use square_eq_iff or power2_eq_iff instead
huffman [Sat, 20 Aug 2011 12:51:15 -0700] rev 44347
remove redundant lemma realpow_two_disj, use square_eq_iff or power2_eq_iff instead
Sat, 20 Aug 2011 10:08:47 -0700 rename real_squared_diff_one_factored to square_diff_one_factored and move to Rings.thy
huffman [Sat, 20 Aug 2011 10:08:47 -0700] rev 44346
rename real_squared_diff_one_factored to square_diff_one_factored and move to Rings.thy
Sat, 20 Aug 2011 09:59:28 -0700 add lemma power2_eq_iff
huffman [Sat, 20 Aug 2011 09:59:28 -0700] rev 44345
add lemma power2_eq_iff
Sat, 20 Aug 2011 07:09:44 -0700 remove some over-specific rules from the simpset
huffman [Sat, 20 Aug 2011 07:09:44 -0700] rev 44344
remove some over-specific rules from the simpset
Sat, 20 Aug 2011 06:35:43 -0700 merged
huffman [Sat, 20 Aug 2011 06:35:43 -0700] rev 44343
merged
Sat, 20 Aug 2011 06:34:51 -0700 redefine constant 'trivial_limit' as an abbreviation
huffman [Sat, 20 Aug 2011 06:34:51 -0700] rev 44342
redefine constant 'trivial_limit' as an abbreviation
Sun, 21 Aug 2011 13:23:29 +0200 purely functional task_queue.ML -- moved actual interrupt_unsynchronized to future.ML;
wenzelm [Sun, 21 Aug 2011 13:23:29 +0200] rev 44341
purely functional task_queue.ML -- moved actual interrupt_unsynchronized to future.ML;
Sun, 21 Aug 2011 13:10:48 +0200 refined Task_Queue.cancel: passive tasks are considered running due to pending abort operation;
wenzelm [Sun, 21 Aug 2011 13:10:48 +0200] rev 44340
refined Task_Queue.cancel: passive tasks are considered running due to pending abort operation;
Sat, 20 Aug 2011 23:36:18 +0200 odd workaround for odd problem of load order in HOL/ex/ROOT.ML (!??);
wenzelm [Sat, 20 Aug 2011 23:36:18 +0200] rev 44339
odd workaround for odd problem of load order in HOL/ex/ROOT.ML (!??);
Sat, 20 Aug 2011 23:35:30 +0200 refined Graph implementation: more abstract/scalable Graph.Keys instead of plain lists -- order of adjacency is now standardized wrt. Key.ord;
wenzelm [Sat, 20 Aug 2011 23:35:30 +0200] rev 44338
refined Graph implementation: more abstract/scalable Graph.Keys instead of plain lists -- order of adjacency is now standardized wrt. Key.ord;
Sat, 20 Aug 2011 22:46:19 +0200 clarified get_imports -- should not rely on accidental order within graph;
wenzelm [Sat, 20 Aug 2011 22:46:19 +0200] rev 44337
clarified get_imports -- should not rely on accidental order within graph;
Sat, 20 Aug 2011 22:28:53 +0200 tuned Table.delete_safe: avoid potentially expensive attempt of delete;
wenzelm [Sat, 20 Aug 2011 22:28:53 +0200] rev 44336
tuned Table.delete_safe: avoid potentially expensive attempt of delete;
Sat, 20 Aug 2011 20:24:12 +0200 discontinued "Interrupt", which could disturb administrative tasks of the document model;
wenzelm [Sat, 20 Aug 2011 20:24:12 +0200] rev 44335
discontinued "Interrupt", which could disturb administrative tasks of the document model;
Sat, 20 Aug 2011 20:00:55 +0200 more direct balanced version Ord_List.unions;
wenzelm [Sat, 20 Aug 2011 20:00:55 +0200] rev 44334
more direct balanced version Ord_List.unions;
Sat, 20 Aug 2011 19:21:03 +0200 reverted to join_bodies/join_proofs based on fold_body_thms to regain performance (escpecially of HOL-Proofs) -- see also aa9c1e9ef2ce and 4e2abb045eac;
wenzelm [Sat, 20 Aug 2011 19:21:03 +0200] rev 44333
reverted to join_bodies/join_proofs based on fold_body_thms to regain performance (escpecially of HOL-Proofs) -- see also aa9c1e9ef2ce and 4e2abb045eac;
Sat, 20 Aug 2011 18:11:17 +0200 tuned future priorities (again);
wenzelm [Sat, 20 Aug 2011 18:11:17 +0200] rev 44332
tuned future priorities (again);
Sat, 20 Aug 2011 16:06:27 +0200 clarified fulfill_norm_proof: no join_thms yet;
wenzelm [Sat, 20 Aug 2011 16:06:27 +0200] rev 44331
clarified fulfill_norm_proof: no join_thms yet; clarified priority of fulfill_proof_future, which is followed by explicit join_thms; explicit Thm.future_body_of without join yet; tuned Thm.future_result: join_promises without fulfill_norm_proof;
Sat, 20 Aug 2011 15:52:29 +0200 added Future.joins convenience;
wenzelm [Sat, 20 Aug 2011 15:52:29 +0200] rev 44330
added Future.joins convenience; clarified Future.map: based on Future.cond_forks;
Sat, 20 Aug 2011 09:42:34 +0200 merged
haftmann [Sat, 20 Aug 2011 09:42:34 +0200] rev 44329
merged
Sat, 20 Aug 2011 09:42:12 +0200 deactivated »unknown« nitpick example
haftmann [Sat, 20 Aug 2011 09:42:12 +0200] rev 44328
deactivated »unknown« nitpick example
Sat, 20 Aug 2011 09:30:23 +0200 merged
haftmann [Sat, 20 Aug 2011 09:30:23 +0200] rev 44327
merged
Sat, 20 Aug 2011 01:40:22 +0200 tuned proof
haftmann [Sat, 20 Aug 2011 01:40:22 +0200] rev 44326
tuned proof
Sat, 20 Aug 2011 01:39:27 +0200 more uniform formatting of specifications
haftmann [Sat, 20 Aug 2011 01:39:27 +0200] rev 44325
more uniform formatting of specifications
Sat, 20 Aug 2011 01:33:58 +0200 compatibility layer
haftmann [Sat, 20 Aug 2011 01:33:58 +0200] rev 44324
compatibility layer
Sat, 20 Aug 2011 01:21:22 +0200 merged
haftmann [Sat, 20 Aug 2011 01:21:22 +0200] rev 44323
merged
Fri, 19 Aug 2011 19:33:31 +0200 more concise definition for Inf, Sup on bool
haftmann [Fri, 19 Aug 2011 19:33:31 +0200] rev 44322
more concise definition for Inf, Sup on bool
Thu, 18 Aug 2011 13:37:41 +0200 do not call ghc with -fglasgow-exts
noschinl [Thu, 18 Aug 2011 13:37:41 +0200] rev 44321
do not call ghc with -fglasgow-exts
Fri, 19 Aug 2011 19:01:00 -0700 remove some redundant simp rules about sqrt
huffman [Fri, 19 Aug 2011 19:01:00 -0700] rev 44320
remove some redundant simp rules about sqrt
Fri, 19 Aug 2011 18:42:41 -0700 move sin_coeff and cos_coeff lemmas to Transcendental.thy; simplify some proofs
huffman [Fri, 19 Aug 2011 18:42:41 -0700] rev 44319
move sin_coeff and cos_coeff lemmas to Transcendental.thy; simplify some proofs
Fri, 19 Aug 2011 18:08:05 -0700 remove unused lemma DERIV_sin_add
huffman [Fri, 19 Aug 2011 18:08:05 -0700] rev 44318
remove unused lemma DERIV_sin_add
Fri, 19 Aug 2011 18:06:27 -0700 remove redundant lemma lemma_DERIV_subst in favor of DERIV_cong
huffman [Fri, 19 Aug 2011 18:06:27 -0700] rev 44317
remove redundant lemma lemma_DERIV_subst in favor of DERIV_cong
Fri, 19 Aug 2011 17:59:19 -0700 remove redundant lemma exp_ln_eq in favor of ln_unique
huffman [Fri, 19 Aug 2011 17:59:19 -0700] rev 44316
remove redundant lemma exp_ln_eq in favor of ln_unique
Fri, 19 Aug 2011 16:55:43 -0700 merged
huffman [Fri, 19 Aug 2011 16:55:43 -0700] rev 44315
merged
Fri, 19 Aug 2011 15:54:43 -0700 Lim.thy: legacy theorems
huffman [Fri, 19 Aug 2011 15:54:43 -0700] rev 44314
Lim.thy: legacy theorems
Fri, 19 Aug 2011 15:07:10 -0700 SEQ.thy: legacy theorem names
huffman [Fri, 19 Aug 2011 15:07:10 -0700] rev 44313
SEQ.thy: legacy theorem names
Fri, 19 Aug 2011 14:46:45 -0700 delete unused lemmas about limits
huffman [Fri, 19 Aug 2011 14:46:45 -0700] rev 44312
delete unused lemmas about limits
Fri, 19 Aug 2011 14:17:28 -0700 Transcendental.thy: add tendsto_intros lemmas;
huffman [Fri, 19 Aug 2011 14:17:28 -0700] rev 44311
Transcendental.thy: add tendsto_intros lemmas; new isCont theorems; simplify some proofs.
Fri, 19 Aug 2011 11:49:53 -0700 add lemma isCont_tendsto_compose
huffman [Fri, 19 Aug 2011 11:49:53 -0700] rev 44310
add lemma isCont_tendsto_compose
Fri, 19 Aug 2011 23:48:18 +0200 merged
wenzelm [Fri, 19 Aug 2011 23:48:18 +0200] rev 44309
merged
Fri, 19 Aug 2011 10:46:54 -0700 Transcendental.thy: remove several unused lemmas and simplify some proofs
huffman [Fri, 19 Aug 2011 10:46:54 -0700] rev 44308
Transcendental.thy: remove several unused lemmas and simplify some proofs
Fri, 19 Aug 2011 08:40:15 -0700 remove unused lemmas
huffman [Fri, 19 Aug 2011 08:40:15 -0700] rev 44307
remove unused lemmas
Fri, 19 Aug 2011 08:39:43 -0700 fold definitions of sin_coeff and cos_coeff in Maclaurin lemmas
huffman [Fri, 19 Aug 2011 08:39:43 -0700] rev 44306
fold definitions of sin_coeff and cos_coeff in Maclaurin lemmas
Fri, 19 Aug 2011 07:45:22 -0700 remove some redundant simp rules
huffman [Fri, 19 Aug 2011 07:45:22 -0700] rev 44305
remove some redundant simp rules
Fri, 19 Aug 2011 23:25:47 +0200 maintain recent future proofs at transaction boundaries;
wenzelm [Fri, 19 Aug 2011 23:25:47 +0200] rev 44304
maintain recent future proofs at transaction boundaries;
Fri, 19 Aug 2011 21:40:52 +0200 incremental Proofterm.join_body, with join_thms step in fulfill_norm_proof -- avoid full graph traversal of former Proofterm.join_bodies;
wenzelm [Fri, 19 Aug 2011 21:40:52 +0200] rev 44303
incremental Proofterm.join_body, with join_thms step in fulfill_norm_proof -- avoid full graph traversal of former Proofterm.join_bodies;
Fri, 19 Aug 2011 18:01:23 +0200 tuned;
wenzelm [Fri, 19 Aug 2011 18:01:23 +0200] rev 44302
tuned;
Fri, 19 Aug 2011 17:39:37 +0200 tuned signature (again);
wenzelm [Fri, 19 Aug 2011 17:39:37 +0200] rev 44301
tuned signature (again); tuned;
Fri, 19 Aug 2011 16:13:26 +0200 tuned signature -- treat structure Task_Queue as private to implementation;
wenzelm [Fri, 19 Aug 2011 16:13:26 +0200] rev 44300
tuned signature -- treat structure Task_Queue as private to implementation;
Fri, 19 Aug 2011 15:56:26 +0200 refined Future.cancel: explicit future allows to join actual cancellation;
wenzelm [Fri, 19 Aug 2011 15:56:26 +0200] rev 44299
refined Future.cancel: explicit future allows to join actual cancellation; Document.cancel_execution: join nested future groups as well;
Fri, 19 Aug 2011 14:01:20 +0200 Future.promise: explicit abort operation (like uninterruptible future job);
wenzelm [Fri, 19 Aug 2011 14:01:20 +0200] rev 44298
Future.promise: explicit abort operation (like uninterruptible future job); explicit cancel_scala message -- still unused;
Fri, 19 Aug 2011 13:55:32 +0200 editable raw text areas: allow user to clear content;
wenzelm [Fri, 19 Aug 2011 13:55:32 +0200] rev 44297
editable raw text areas: allow user to clear content;
Fri, 19 Aug 2011 13:32:27 +0200 more robust use of set_exn_serial, which is based on PolyML.raiseWithLocation internally;
wenzelm [Fri, 19 Aug 2011 13:32:27 +0200] rev 44296
more robust use of set_exn_serial, which is based on PolyML.raiseWithLocation internally;
Fri, 19 Aug 2011 12:51:14 +0200 more focused use of Multithreading.interrupted: retain interrupts within task group boundary, without loss of information;
wenzelm [Fri, 19 Aug 2011 12:51:14 +0200] rev 44295
more focused use of Multithreading.interrupted: retain interrupts within task group boundary, without loss of information;
Fri, 19 Aug 2011 12:03:44 +0200 clarified Future.cond_forks: more uniform handling of exceptional situations;
wenzelm [Fri, 19 Aug 2011 12:03:44 +0200] rev 44294
clarified Future.cond_forks: more uniform handling of exceptional situations;
Fri, 19 Aug 2011 17:05:10 +0900 Quotient_Examples: Cset, List_Cset: Lift Inf and Sup directly.
Cezary Kaliszyk <kaliszyk@in.tum.de> [Fri, 19 Aug 2011 17:05:10 +0900] rev 44293
Quotient_Examples: Cset, List_Cset: Lift Inf and Sup directly.
Thu, 18 Aug 2011 22:32:19 -0700 merged
huffman [Thu, 18 Aug 2011 22:32:19 -0700] rev 44292
merged
Thu, 18 Aug 2011 22:31:52 -0700 define complex exponential 'expi' as abbreviation for 'exp'
huffman [Thu, 18 Aug 2011 22:31:52 -0700] rev 44291
define complex exponential 'expi' as abbreviation for 'exp'
Thu, 18 Aug 2011 21:23:31 -0700 remove more bounded_linear locale interpretations (cf. f0de18b62d63)
huffman [Thu, 18 Aug 2011 21:23:31 -0700] rev 44290
remove more bounded_linear locale interpretations (cf. f0de18b62d63)
Thu, 18 Aug 2011 19:53:03 -0700 optimize some proofs
huffman [Thu, 18 Aug 2011 19:53:03 -0700] rev 44289
optimize some proofs
Thu, 18 Aug 2011 18:10:23 -0700 add Multivariate_Analysis dependencies
huffman [Thu, 18 Aug 2011 18:10:23 -0700] rev 44288
add Multivariate_Analysis dependencies
Thu, 18 Aug 2011 18:08:43 -0700 import Library/Sum_of_Squares instead of reloading positivstellensatz.ML
huffman [Thu, 18 Aug 2011 18:08:43 -0700] rev 44287
import Library/Sum_of_Squares instead of reloading positivstellensatz.ML
Thu, 18 Aug 2011 17:32:02 -0700 declare euclidean_component_zero[simp] at the point it is proved
huffman [Thu, 18 Aug 2011 17:32:02 -0700] rev 44286
declare euclidean_component_zero[simp] at the point it is proved
Fri, 19 Aug 2011 10:23:16 +0900 Quotient Package: Regularization: do not fail if no progress is made, leave the subgoal to the user. Injection: try assumptions before extensionality to avoid looping.
Cezary Kaliszyk <kaliszyk@in.tum.de> [Fri, 19 Aug 2011 10:23:16 +0900] rev 44285
Quotient Package: Regularization: do not fail if no progress is made, leave the subgoal to the user. Injection: try assumptions before extensionality to avoid looping.
Thu, 18 Aug 2011 23:43:22 +0200 merged;
wenzelm [Thu, 18 Aug 2011 23:43:22 +0200] rev 44284
merged;
Thu, 18 Aug 2011 14:08:39 -0700 merged
huffman [Thu, 18 Aug 2011 14:08:39 -0700] rev 44283
merged
Thu, 18 Aug 2011 13:36:58 -0700 remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
huffman [Thu, 18 Aug 2011 13:36:58 -0700] rev 44282
remove bounded_(bi)linear locale interpretations, to avoid duplicating so many lemmas
Thu, 18 Aug 2011 22:50:28 +0200 merged
haftmann [Thu, 18 Aug 2011 22:50:28 +0200] rev 44281
merged
Thu, 18 Aug 2011 22:50:17 +0200 merged
haftmann [Thu, 18 Aug 2011 22:50:17 +0200] rev 44280
merged
Thu, 18 Aug 2011 14:01:06 +0200 avoid duplicated simp add option
haftmann [Thu, 18 Aug 2011 14:01:06 +0200] rev 44279
avoid duplicated simp add option
Thu, 18 Aug 2011 13:55:26 +0200 observe distinction between sets and predicates more properly
haftmann [Thu, 18 Aug 2011 13:55:26 +0200] rev 44278
observe distinction between sets and predicates more properly
Thu, 18 Aug 2011 13:25:17 +0200 moved fundamental lemma fun_eq_iff to theory HOL; tuned whitespace
haftmann [Thu, 18 Aug 2011 13:25:17 +0200] rev 44277
moved fundamental lemma fun_eq_iff to theory HOL; tuned whitespace
Thu, 18 Aug 2011 13:10:24 +0200 avoid case-sensitive name for example theory
haftmann [Thu, 18 Aug 2011 13:10:24 +0200] rev 44276
avoid case-sensitive name for example theory
Thu, 18 Aug 2011 17:42:35 +0200 merged
nipkow [Thu, 18 Aug 2011 17:42:35 +0200] rev 44275
merged
Thu, 18 Aug 2011 17:42:18 +0200 case_names NEWS
nipkow [Thu, 18 Aug 2011 17:42:18 +0200] rev 44274
case_names NEWS
Thu, 18 Aug 2011 17:00:15 +0200 adding documentation about simps equation in the inductive package
bulwahn [Thu, 18 Aug 2011 17:00:15 +0200] rev 44273
adding documentation about simps equation in the inductive package
Thu, 18 Aug 2011 12:06:17 +0200 activating narrowing-based quickcheck by default
bulwahn [Thu, 18 Aug 2011 12:06:17 +0200] rev 44272
activating narrowing-based quickcheck by default
Thu, 18 Aug 2011 18:07:40 +0200 more precise treatment of exception nesting and serial numbers;
wenzelm [Thu, 18 Aug 2011 18:07:40 +0200] rev 44271
more precise treatment of exception nesting and serial numbers;
Thu, 18 Aug 2011 17:53:32 +0200 more careful treatment of exception serial numbers, with propagation to message channel;
wenzelm [Thu, 18 Aug 2011 17:53:32 +0200] rev 44270
more careful treatment of exception serial numbers, with propagation to message channel;
Thu, 18 Aug 2011 17:30:47 +0200 updated sequential version (cf. b94951f06e48);
wenzelm [Thu, 18 Aug 2011 17:30:47 +0200] rev 44269
updated sequential version (cf. b94951f06e48);
Thu, 18 Aug 2011 16:07:58 +0200 tuned comments;
wenzelm [Thu, 18 Aug 2011 16:07:58 +0200] rev 44268
tuned comments;
Thu, 18 Aug 2011 15:51:34 +0200 tuned document;
wenzelm [Thu, 18 Aug 2011 15:51:34 +0200] rev 44267
tuned document; tuned proofs;
Thu, 18 Aug 2011 15:39:00 +0200 clarified Par_Exn.release_first: prefer plain exn, before falling back on full pack of parallel exceptions;
wenzelm [Thu, 18 Aug 2011 15:39:00 +0200] rev 44266
clarified Par_Exn.release_first: prefer plain exn, before falling back on full pack of parallel exceptions;
Thu, 18 Aug 2011 15:37:01 +0200 export Par_List.managed_results, to enable specific treatment of results apart from default Par_Exn.release_first;
wenzelm [Thu, 18 Aug 2011 15:37:01 +0200] rev 44265
export Par_List.managed_results, to enable specific treatment of results apart from default Par_Exn.release_first;
Thu, 18 Aug 2011 15:15:43 +0200 tune Par_Exn.make: balance merge;
wenzelm [Thu, 18 Aug 2011 15:15:43 +0200] rev 44264
tune Par_Exn.make: balance merge; clarified Par_Exn.dest: later exceptions first;
Thu, 18 Aug 2011 16:52:19 +0900 Quotient_Examples/DList: explicit proof of remdups_eq_member_eq needed for explicit set type.
Cezary Kaliszyk <kaliszyk@in.tum.de> [Thu, 18 Aug 2011 16:52:19 +0900] rev 44263
Quotient_Examples/DList: explicit proof of remdups_eq_member_eq needed for explicit set type.
Wed, 17 Aug 2011 15:12:34 -0700 merged
huffman [Wed, 17 Aug 2011 15:12:34 -0700] rev 44262
merged
Wed, 17 Aug 2011 15:03:30 -0700 HOL-IMP: respect set/pred distinction
huffman [Wed, 17 Aug 2011 15:03:30 -0700] rev 44261
HOL-IMP: respect set/pred distinction
Wed, 17 Aug 2011 15:02:17 -0700 Determinants.thy: avoid using mem_def/Collect_def
huffman [Wed, 17 Aug 2011 15:02:17 -0700] rev 44260
Determinants.thy: avoid using mem_def/Collect_def
Wed, 17 Aug 2011 14:42:59 -0700 Wfrec.thy: respect set/pred distinction
huffman [Wed, 17 Aug 2011 14:42:59 -0700] rev 44259
Wfrec.thy: respect set/pred distinction
Thu, 18 Aug 2011 00:02:44 +0200 follow updates of Isabelle/Pure;
wenzelm [Thu, 18 Aug 2011 00:02:44 +0200] rev 44258
follow updates of Isabelle/Pure;
Wed, 17 Aug 2011 23:41:47 +0200 merged
wenzelm [Wed, 17 Aug 2011 23:41:47 +0200] rev 44257
merged
Wed, 17 Aug 2011 14:32:48 -0700 IsaMakefile: target HOLCF-Library now compiles HOL/HOLCF/Library instead of HOL/Library
huffman [Wed, 17 Aug 2011 14:32:48 -0700] rev 44256
IsaMakefile: target HOLCF-Library now compiles HOL/HOLCF/Library instead of HOL/Library
Wed, 17 Aug 2011 13:10:49 -0700 merged
huffman [Wed, 17 Aug 2011 13:10:49 -0700] rev 44255
merged
Wed, 17 Aug 2011 13:10:11 -0700 Lim.thy: generalize and simplify proofs of LIM/LIMSEQ theorems
huffman [Wed, 17 Aug 2011 13:10:11 -0700] rev 44254
Lim.thy: generalize and simplify proofs of LIM/LIMSEQ theorems
Wed, 17 Aug 2011 11:39:09 -0700 add lemma tendsto_compose_eventually; use it to shorten some proofs
huffman [Wed, 17 Aug 2011 11:39:09 -0700] rev 44253
add lemma tendsto_compose_eventually; use it to shorten some proofs
Wed, 17 Aug 2011 11:07:32 -0700 Topology_Euclidean_Space.thy: simplify some proofs
huffman [Wed, 17 Aug 2011 11:07:32 -0700] rev 44252
Topology_Euclidean_Space.thy: simplify some proofs
Wed, 17 Aug 2011 11:06:39 -0700 add lemma metric_tendsto_imp_tendsto
huffman [Wed, 17 Aug 2011 11:06:39 -0700] rev 44251
add lemma metric_tendsto_imp_tendsto
Wed, 17 Aug 2011 09:59:10 -0700 simplify proofs of lemmas open_interval, closed_interval
huffman [Wed, 17 Aug 2011 09:59:10 -0700] rev 44250
simplify proofs of lemmas open_interval, closed_interval
Wed, 17 Aug 2011 23:37:23 +0200 identify parallel exceptions where they emerge first -- to achieve unique results within evaluation graph;
wenzelm [Wed, 17 Aug 2011 23:37:23 +0200] rev 44249
identify parallel exceptions where they emerge first -- to achieve unique results within evaluation graph;
Wed, 17 Aug 2011 22:25:00 +0200 clarified Par_Exn.release_first: traverse topmost list structure only, not arbitrary depths of nested Par_Exn;
wenzelm [Wed, 17 Aug 2011 22:25:00 +0200] rev 44248
clarified Par_Exn.release_first: traverse topmost list structure only, not arbitrary depths of nested Par_Exn;
Wed, 17 Aug 2011 22:14:22 +0200 more systematic handling of parallel exceptions;
wenzelm [Wed, 17 Aug 2011 22:14:22 +0200] rev 44247
more systematic handling of parallel exceptions; distinguish exception concatanation EXCEPTIONS from parallel Par_Exn;
Wed, 17 Aug 2011 20:08:36 +0200 tuned signature;
wenzelm [Wed, 17 Aug 2011 20:08:36 +0200] rev 44246
tuned signature;
Wed, 17 Aug 2011 18:52:21 +0200 merged
haftmann [Wed, 17 Aug 2011 18:52:21 +0200] rev 44245
merged
Wed, 17 Aug 2011 18:51:27 +0200 merged
haftmann [Wed, 17 Aug 2011 18:51:27 +0200] rev 44244
merged
Wed, 17 Aug 2011 07:13:13 +0200 merged
haftmann [Wed, 17 Aug 2011 07:13:13 +0200] rev 44243
merged
Tue, 16 Aug 2011 19:47:50 +0200 avoid Collect_def in proof
haftmann [Tue, 16 Aug 2011 19:47:50 +0200] rev 44242
avoid Collect_def in proof
Wed, 17 Aug 2011 18:05:31 +0200 modernized signature of Term.absfree/absdummy;
wenzelm [Wed, 17 Aug 2011 18:05:31 +0200] rev 44241
modernized signature of Term.absfree/absdummy; eliminated obsolete Term.list_abs_free;
Wed, 17 Aug 2011 16:46:58 +0200 improved default context for ML toplevel pretty-printing;
wenzelm [Wed, 17 Aug 2011 16:46:58 +0200] rev 44240
improved default context for ML toplevel pretty-printing;
Wed, 17 Aug 2011 16:30:38 +0200 less verbosity for 'function' and 'fun': observe "int" flag more carefully (cf. a32ca9165928);
wenzelm [Wed, 17 Aug 2011 16:30:38 +0200] rev 44239
less verbosity for 'function' and 'fun': observe "int" flag more carefully (cf. a32ca9165928);
Wed, 17 Aug 2011 16:01:27 +0200 some convenience actions/shortcuts for control symbols;
wenzelm [Wed, 17 Aug 2011 16:01:27 +0200] rev 44238
some convenience actions/shortcuts for control symbols;
Wed, 17 Aug 2011 15:14:48 +0200 export Function_Fun.fun_config for user convenience;
wenzelm [Wed, 17 Aug 2011 15:14:48 +0200] rev 44237
export Function_Fun.fun_config for user convenience;
Wed, 17 Aug 2011 13:14:20 +0200 moved theory Nested_Environment to HOL-Unix (a bit too specific for HOL-Library);
wenzelm [Wed, 17 Aug 2011 13:14:20 +0200] rev 44236
moved theory Nested_Environment to HOL-Unix (a bit too specific for HOL-Library);
Wed, 17 Aug 2011 10:03:58 +0200 distinguish THF syntax with and without choice (Satallax vs. LEO-II)
blanchet [Wed, 17 Aug 2011 10:03:58 +0200] rev 44235
distinguish THF syntax with and without choice (Satallax vs. LEO-II)
Tue, 16 Aug 2011 15:02:20 -0700 merged
huffman [Tue, 16 Aug 2011 15:02:20 -0700] rev 44234
merged
Tue, 16 Aug 2011 09:31:23 -0700 add simp rules for isCont
huffman [Tue, 16 Aug 2011 09:31:23 -0700] rev 44233
add simp rules for isCont
Tue, 16 Aug 2011 23:39:58 +0200 updated keywords -- old codegen is no longer in Pure;
wenzelm [Tue, 16 Aug 2011 23:39:58 +0200] rev 44232
updated keywords -- old codegen is no longer in Pure;
Tue, 16 Aug 2011 23:39:30 +0200 include HOL-Library keywords for the sake of recdef;
wenzelm [Tue, 16 Aug 2011 23:39:30 +0200] rev 44231
include HOL-Library keywords for the sake of recdef;
Tue, 16 Aug 2011 23:25:02 +0200 merged
wenzelm [Tue, 16 Aug 2011 23:25:02 +0200] rev 44230
merged
Tue, 16 Aug 2011 13:07:52 -0700 Multivariate_Analysis includes Determinants.thy, but doesn't import it by default
huffman [Tue, 16 Aug 2011 13:07:52 -0700] rev 44229
Multivariate_Analysis includes Determinants.thy, but doesn't import it by default
Tue, 16 Aug 2011 07:56:17 -0700 get Multivariate_Analysis/Determinants.thy compiled and working again
huffman [Tue, 16 Aug 2011 07:56:17 -0700] rev 44228
get Multivariate_Analysis/Determinants.thy compiled and working again
Tue, 16 Aug 2011 07:06:54 -0700 get Library/Permutations.thy compiled and working again
huffman [Tue, 16 Aug 2011 07:06:54 -0700] rev 44227
get Library/Permutations.thy compiled and working again
Tue, 16 Aug 2011 23:17:26 +0200 workaround for Cygwin, to make it work in the important special case without extra files;
wenzelm [Tue, 16 Aug 2011 23:17:26 +0200] rev 44226
workaround for Cygwin, to make it work in the important special case without extra files;
Tue, 16 Aug 2011 22:48:31 +0200 more robust Thy_Header.base_name, with minimal assumptions about path syntax;
wenzelm [Tue, 16 Aug 2011 22:48:31 +0200] rev 44225
more robust Thy_Header.base_name, with minimal assumptions about path syntax; Isabelle.buffer_path: keep platform syntax;
Tue, 16 Aug 2011 21:54:06 +0200 tuned message;
wenzelm [Tue, 16 Aug 2011 21:54:06 +0200] rev 44224
tuned message;
Tue, 16 Aug 2011 21:50:53 +0200 more robust treatment of node dependencies in incremental edits;
wenzelm [Tue, 16 Aug 2011 21:50:53 +0200] rev 44223
more robust treatment of node dependencies in incremental edits;
Tue, 16 Aug 2011 21:13:52 +0200 use full .thy file name as node name, which makes MiscUtilities.resolveSymlinks/File.getCanonicalPath more predictable;
wenzelm [Tue, 16 Aug 2011 21:13:52 +0200] rev 44222
use full .thy file name as node name, which makes MiscUtilities.resolveSymlinks/File.getCanonicalPath more predictable; more robust treatment of node dependencies; misc tuning;
Tue, 16 Aug 2011 12:06:49 +0200 omit MiscUtilities.resolveSymlinks for now -- odd effects on case-insensible file-system;
wenzelm [Tue, 16 Aug 2011 12:06:49 +0200] rev 44221
omit MiscUtilities.resolveSymlinks for now -- odd effects on case-insensible file-system;
Mon, 15 Aug 2011 19:42:52 -0700 merged
huffman [Mon, 15 Aug 2011 19:42:52 -0700] rev 44220
merged
Mon, 15 Aug 2011 18:35:36 -0700 generalize lemmas open_Collect_less, closed_Collect_le, closed_Collect_eq to class topological_space
huffman [Mon, 15 Aug 2011 18:35:36 -0700] rev 44219
generalize lemmas open_Collect_less, closed_Collect_le, closed_Collect_eq to class topological_space
Mon, 15 Aug 2011 16:48:05 -0700 add lemma tendsto_compose
huffman [Mon, 15 Aug 2011 16:48:05 -0700] rev 44218
add lemma tendsto_compose
Mon, 15 Aug 2011 16:18:13 -0700 remove extraneous subsection heading
huffman [Mon, 15 Aug 2011 16:18:13 -0700] rev 44217
remove extraneous subsection heading
Mon, 15 Aug 2011 15:11:55 -0700 generalized lemma closed_Collect_eq
huffman [Mon, 15 Aug 2011 15:11:55 -0700] rev 44216
generalized lemma closed_Collect_eq
Mon, 15 Aug 2011 14:50:24 -0700 remove duplicate lemma disjoint_iff
huffman [Mon, 15 Aug 2011 14:50:24 -0700] rev 44215
remove duplicate lemma disjoint_iff
Mon, 15 Aug 2011 14:29:17 -0700 Library/Product_Vector.thy: class instances for t0_space, t1_space, and t2_space
huffman [Mon, 15 Aug 2011 14:29:17 -0700] rev 44214
Library/Product_Vector.thy: class instances for t0_space, t1_space, and t2_space
Mon, 15 Aug 2011 14:09:39 -0700 add lemmas open_Collect_less, closed_Collect_le, closed_Collect_eq;
huffman [Mon, 15 Aug 2011 14:09:39 -0700] rev 44213
add lemmas open_Collect_less, closed_Collect_le, closed_Collect_eq; simplify and generalize some proofs;
Mon, 15 Aug 2011 12:18:34 -0700 generalize lemma continuous_uniform_limit to class metric_space
huffman [Mon, 15 Aug 2011 12:18:34 -0700] rev 44212
generalize lemma continuous_uniform_limit to class metric_space
Mon, 15 Aug 2011 12:13:46 -0700 remove duplicate lemmas eventually_conjI, eventually_and, eventually_false
huffman [Mon, 15 Aug 2011 12:13:46 -0700] rev 44211
remove duplicate lemmas eventually_conjI, eventually_and, eventually_false
Mon, 15 Aug 2011 10:49:48 -0700 Topology_Euclidean_Space.thy: organize section headings
huffman [Mon, 15 Aug 2011 10:49:48 -0700] rev 44210
Topology_Euclidean_Space.thy: organize section headings
Mon, 15 Aug 2011 09:08:17 -0700 simplify some proofs
huffman [Mon, 15 Aug 2011 09:08:17 -0700] rev 44209
simplify some proofs
Sun, 14 Aug 2011 13:04:57 -0700 generalize lemma convergent_subseq_convergent
huffman [Sun, 14 Aug 2011 13:04:57 -0700] rev 44208
generalize lemma convergent_subseq_convergent
Sun, 14 Aug 2011 11:44:12 -0700 locale-ize some definitions, so perfect_space and heine_borel can inherit from the proper superclasses
huffman [Sun, 14 Aug 2011 11:44:12 -0700] rev 44207
locale-ize some definitions, so perfect_space and heine_borel can inherit from the proper superclasses
Sun, 14 Aug 2011 10:47:47 -0700 locale-ize some constant definitions, so complete_space can inherit from metric_space
huffman [Sun, 14 Aug 2011 10:47:47 -0700] rev 44206
locale-ize some constant definitions, so complete_space can inherit from metric_space
Sun, 14 Aug 2011 10:25:43 -0700 generalize constant 'lim' and limit uniqueness theorems to class t2_space
huffman [Sun, 14 Aug 2011 10:25:43 -0700] rev 44205
generalize constant 'lim' and limit uniqueness theorems to class t2_space
Tue, 16 Aug 2011 07:17:15 +0900 Quotient Package: make quotient_type work with separate set type
Cezary Kaliszyk <kaliszyk@in.tum.de> [Tue, 16 Aug 2011 07:17:15 +0900] rev 44204
Quotient Package: make quotient_type work with separate set type
Mon, 15 Aug 2011 22:31:17 +0200 updated README;
wenzelm [Mon, 15 Aug 2011 22:31:17 +0200] rev 44203
updated README;
Mon, 15 Aug 2011 21:54:32 +0200 touch descendants of edited nodes;
wenzelm [Mon, 15 Aug 2011 21:54:32 +0200] rev 44202
touch descendants of edited nodes; more precise handling of Graph exceptions;
Mon, 15 Aug 2011 21:05:30 +0200 parellel scheduling of node edits and execution;
wenzelm [Mon, 15 Aug 2011 21:05:30 +0200] rev 44201
parellel scheduling of node edits and execution;
Mon, 15 Aug 2011 20:38:16 +0200 tuned error message;
wenzelm [Mon, 15 Aug 2011 20:38:16 +0200] rev 44200
tuned error message;
Mon, 15 Aug 2011 20:19:41 +0200 retrieve imports from document state, with fall-back on theory loader for preloaded theories;
wenzelm [Mon, 15 Aug 2011 20:19:41 +0200] rev 44199
retrieve imports from document state, with fall-back on theory loader for preloaded theories; misc tuning;
Mon, 15 Aug 2011 19:27:55 +0200 explicit check of finished evaluation;
wenzelm [Mon, 15 Aug 2011 19:27:55 +0200] rev 44198
explicit check of finished evaluation;
Mon, 15 Aug 2011 16:38:42 +0200 refined Document.edit: less stateful update via Graph.schedule;
wenzelm [Mon, 15 Aug 2011 16:38:42 +0200] rev 44197
refined Document.edit: less stateful update via Graph.schedule; clarified node result -- more direct get_theory; clarified Document.joint_commands;
Mon, 15 Aug 2011 14:54:36 +0200 simplified exec: eliminated unused status flag;
wenzelm [Mon, 15 Aug 2011 14:54:36 +0200] rev 44196
simplified exec: eliminated unused status flag;
Sun, 14 Aug 2011 08:45:38 -0700 consistently use variable name 'F' for filters
huffman [Sun, 14 Aug 2011 08:45:38 -0700] rev 44195
consistently use variable name 'F' for filters
Sun, 14 Aug 2011 07:54:24 -0700 generalize lemmas about LIM and LIMSEQ to tendsto
huffman [Sun, 14 Aug 2011 07:54:24 -0700] rev 44194
generalize lemmas about LIM and LIMSEQ to tendsto
Sat, 13 Aug 2011 18:10:14 -0700 HOL-Nominal-Examples: respect distinction between sets and functions
huffman [Sat, 13 Aug 2011 18:10:14 -0700] rev 44193
HOL-Nominal-Examples: respect distinction between sets and functions
Sat, 13 Aug 2011 22:04:07 +0200 less verbosity in batch mode -- spam reduction and notable performance improvement;
wenzelm [Sat, 13 Aug 2011 22:04:07 +0200] rev 44192
less verbosity in batch mode -- spam reduction and notable performance improvement; clarified Proof_Display.print_consts;
Sat, 13 Aug 2011 21:28:01 +0200 merged
wenzelm [Sat, 13 Aug 2011 21:28:01 +0200] rev 44191
merged
Sat, 13 Aug 2011 07:56:55 -0700 HOL-Hahn_Banach: use Set_Algebras library
huffman [Sat, 13 Aug 2011 07:56:55 -0700] rev 44190
HOL-Hahn_Banach: use Set_Algebras library
Sat, 13 Aug 2011 07:39:35 -0700 ex/Quickcheck_Examples.thy: respect distinction between sets and functions
huffman [Sat, 13 Aug 2011 07:39:35 -0700] rev 44189
ex/Quickcheck_Examples.thy: respect distinction between sets and functions
Sat, 13 Aug 2011 21:06:01 +0200 clarified Toplevel.end_theory;
wenzelm [Sat, 13 Aug 2011 21:06:01 +0200] rev 44188
clarified Toplevel.end_theory;
Sat, 13 Aug 2011 20:49:41 +0200 simplified Toplevel.init_theory: discontinued special name argument;
wenzelm [Sat, 13 Aug 2011 20:49:41 +0200] rev 44187
simplified Toplevel.init_theory: discontinued special name argument;
Sat, 13 Aug 2011 20:41:29 +0200 simplified Toplevel.init_theory: discontinued special master argument;
wenzelm [Sat, 13 Aug 2011 20:41:29 +0200] rev 44186
simplified Toplevel.init_theory: discontinued special master argument;
Sat, 13 Aug 2011 20:20:36 +0200 provide node header via Scala layer;
wenzelm [Sat, 13 Aug 2011 20:20:36 +0200] rev 44185
provide node header via Scala layer; clarified node edit Clear: retain header information; run_command: node info via document model, error handling within transaction; node names without ".thy" suffix, to coincide with traditional theory loader treatment;
Sat, 13 Aug 2011 16:07:26 +0200 reduced verbosity;
wenzelm [Sat, 13 Aug 2011 16:07:26 +0200] rev 44184
reduced verbosity;
Sat, 13 Aug 2011 16:04:28 +0200 tuned signature;
wenzelm [Sat, 13 Aug 2011 16:04:28 +0200] rev 44183
tuned signature;
Sat, 13 Aug 2011 15:59:26 +0200 clarified node header -- exclude master_dir;
wenzelm [Sat, 13 Aug 2011 15:59:26 +0200] rev 44182
clarified node header -- exclude master_dir;
Sat, 13 Aug 2011 13:48:26 +0200 tuned;
wenzelm [Sat, 13 Aug 2011 13:48:26 +0200] rev 44181
tuned;
Sat, 13 Aug 2011 13:42:35 +0200 maintain node header;
wenzelm [Sat, 13 Aug 2011 13:42:35 +0200] rev 44180
maintain node header; misc tuning and clarification;
Sat, 13 Aug 2011 12:23:51 +0200 removed unused lemma; removed old-style ;
kleing [Sat, 13 Aug 2011 12:23:51 +0200] rev 44179
removed unused lemma; removed old-style ;
Sat, 13 Aug 2011 12:05:52 +0200 point isatest-statistics to the right afp log files
kleing [Sat, 13 Aug 2011 12:05:52 +0200] rev 44178
point isatest-statistics to the right afp log files
Sat, 13 Aug 2011 11:57:13 +0200 IMP/Util distinguishes between sets and functions again; imported only where used.
kleing [Sat, 13 Aug 2011 11:57:13 +0200] rev 44177
IMP/Util distinguishes between sets and functions again; imported only where used.
Fri, 12 Aug 2011 20:55:22 -0700 remove redundant lemma setsum_norm in favor of norm_setsum;
huffman [Fri, 12 Aug 2011 20:55:22 -0700] rev 44176
remove redundant lemma setsum_norm in favor of norm_setsum; remove finiteness assumption from setsum_norm_le;
Fri, 12 Aug 2011 16:47:53 -0700 merged
huffman [Fri, 12 Aug 2011 16:47:53 -0700] rev 44175
merged
Fri, 12 Aug 2011 14:45:50 -0700 make more HOL theories work with separate set type
huffman [Fri, 12 Aug 2011 14:45:50 -0700] rev 44174
make more HOL theories work with separate set type
Sat, 13 Aug 2011 00:34:54 +0200 immediate fork of initial workers -- avoid 5 ticks (250ms) for adaptive scheme (a07558eb5029);
wenzelm [Sat, 13 Aug 2011 00:34:54 +0200] rev 44173
immediate fork of initial workers -- avoid 5 ticks (250ms) for adaptive scheme (a07558eb5029); more careful treatment of last_round on startup/shutdown;
Fri, 12 Aug 2011 23:29:28 +0200 merged
wenzelm [Fri, 12 Aug 2011 23:29:28 +0200] rev 44172
merged
Fri, 12 Aug 2011 09:17:30 -0700 merged
huffman [Fri, 12 Aug 2011 09:17:30 -0700] rev 44171
merged
Fri, 12 Aug 2011 09:17:24 -0700 make Multivariate_Analysis work with separate set type
huffman [Fri, 12 Aug 2011 09:17:24 -0700] rev 44170
make Multivariate_Analysis work with separate set type
Fri, 12 Aug 2011 07:18:28 -0700 make HOLCF work with separate set type
huffman [Fri, 12 Aug 2011 07:18:28 -0700] rev 44169
make HOLCF work with separate set type
Fri, 12 Aug 2011 07:13:12 -0700 merged
huffman [Fri, 12 Aug 2011 07:13:12 -0700] rev 44168
merged
Thu, 11 Aug 2011 14:24:05 -0700 avoid duplicate rule warnings
huffman [Thu, 11 Aug 2011 14:24:05 -0700] rev 44167
avoid duplicate rule warnings
Thu, 11 Aug 2011 13:05:56 -0700 modify euclidean_space class to include basis set
huffman [Thu, 11 Aug 2011 13:05:56 -0700] rev 44166
modify euclidean_space class to include basis set
Thu, 11 Aug 2011 09:11:15 -0700 remove lemma stupid_ext
huffman [Thu, 11 Aug 2011 09:11:15 -0700] rev 44165
remove lemma stupid_ext
Fri, 12 Aug 2011 17:01:30 +0200 documented extended version of case_names attribute
nipkow [Fri, 12 Aug 2011 17:01:30 +0200] rev 44164
documented extended version of case_names attribute
Fri, 12 Aug 2011 22:10:49 +0200 normalized theory dependencies wrt. file_store;
wenzelm [Fri, 12 Aug 2011 22:10:49 +0200] rev 44163
normalized theory dependencies wrt. file_store;
Fri, 12 Aug 2011 20:32:25 +0200 general Graph.schedule;
wenzelm [Fri, 12 Aug 2011 20:32:25 +0200] rev 44162
general Graph.schedule;
Fri, 12 Aug 2011 15:30:12 +0200 allow "$" within basic path elements (NB: initial "$" refers to path variable);
wenzelm [Fri, 12 Aug 2011 15:30:12 +0200] rev 44161
allow "$" within basic path elements (NB: initial "$" refers to path variable);
Fri, 12 Aug 2011 15:28:30 +0200 clarified document model header: master_dir (native wrt. editor, potentially URL) and node_name (full canonical path);
wenzelm [Fri, 12 Aug 2011 15:28:30 +0200] rev 44160
clarified document model header: master_dir (native wrt. editor, potentially URL) and node_name (full canonical path);
Fri, 12 Aug 2011 12:03:17 +0200 simplified class Thy_Header;
wenzelm [Fri, 12 Aug 2011 12:03:17 +0200] rev 44159
simplified class Thy_Header;
Fri, 12 Aug 2011 11:41:26 +0200 clarified Exn.message;
wenzelm [Fri, 12 Aug 2011 11:41:26 +0200] rev 44158
clarified Exn.message;
Thu, 11 Aug 2011 20:32:44 +0200 uniform treatment of header edits as document edits;
wenzelm [Thu, 11 Aug 2011 20:32:44 +0200] rev 44157
uniform treatment of header edits as document edits;
Thu, 11 Aug 2011 18:01:28 +0200 explicit datatypes for document node edits;
wenzelm [Thu, 11 Aug 2011 18:01:28 +0200] rev 44156
explicit datatypes for document node edits;
Thu, 11 Aug 2011 13:24:49 +0200 tuned;
wenzelm [Thu, 11 Aug 2011 13:24:49 +0200] rev 44155
tuned;
Thu, 11 Aug 2011 13:22:22 +0200 disentangled nested ML files;
wenzelm [Thu, 11 Aug 2011 13:22:22 +0200] rev 44154
disentangled nested ML files;
Thu, 11 Aug 2011 13:05:23 +0200 minimal script to run raw Poly/ML with concurrency library;
wenzelm [Thu, 11 Aug 2011 13:05:23 +0200] rev 44153
minimal script to run raw Poly/ML with concurrency library;
Thu, 11 Aug 2011 12:53:41 +0200 somewhat more uniform THIS;
wenzelm [Thu, 11 Aug 2011 12:53:41 +0200] rev 44152
somewhat more uniform THIS;
Thu, 11 Aug 2011 12:49:14 +0200 more trimming;
wenzelm [Thu, 11 Aug 2011 12:49:14 +0200] rev 44151
more trimming;
Thu, 11 Aug 2011 12:30:41 +0200 recovered some ML toplevel pp;
wenzelm [Thu, 11 Aug 2011 12:30:41 +0200] rev 44150
recovered some ML toplevel pp;
Thu, 11 Aug 2011 12:24:10 +0200 some trimming;
wenzelm [Thu, 11 Aug 2011 12:24:10 +0200] rev 44149
some trimming;
Thu, 11 Aug 2011 12:11:50 +0200 prefix of Pure/ROOT.ML required for concurrency within the ML runtime;
wenzelm [Thu, 11 Aug 2011 12:11:50 +0200] rev 44148
prefix of Pure/ROOT.ML required for concurrency within the ML runtime;
Thu, 11 Aug 2011 11:40:25 +0200 redundant use of misc_legacy.ML;
wenzelm [Thu, 11 Aug 2011 11:40:25 +0200] rev 44147
redundant use of misc_legacy.ML;
Thu, 11 Aug 2011 10:36:34 +0200 eliminated use of recdef
krauss [Thu, 11 Aug 2011 10:36:34 +0200] rev 44146
eliminated use of recdef
Thu, 11 Aug 2011 09:41:21 +0200 removed obsolete recdef-related examples
krauss [Thu, 11 Aug 2011 09:41:21 +0200] rev 44145
removed obsolete recdef-related examples
Thu, 11 Aug 2011 09:15:45 +0200 removed unused material, which does not really belong here
krauss [Thu, 11 Aug 2011 09:15:45 +0200] rev 44144
removed unused material, which does not really belong here
Wed, 10 Aug 2011 18:07:32 -0700 merged
huffman [Wed, 10 Aug 2011 18:07:32 -0700] rev 44143
merged
Wed, 10 Aug 2011 18:02:16 -0700 avoid warnings about duplicate rules
huffman [Wed, 10 Aug 2011 18:02:16 -0700] rev 44142
avoid warnings about duplicate rules
Wed, 10 Aug 2011 17:02:03 -0700 follow standard naming scheme for sgn_vec_def
huffman [Wed, 10 Aug 2011 17:02:03 -0700] rev 44141
follow standard naming scheme for sgn_vec_def
Wed, 10 Aug 2011 16:35:50 -0700 remove several redundant and unused theorems about derivatives
huffman [Wed, 10 Aug 2011 16:35:50 -0700] rev 44140
remove several redundant and unused theorems about derivatives
Wed, 10 Aug 2011 15:56:48 -0700 remove redundant lemma
huffman [Wed, 10 Aug 2011 15:56:48 -0700] rev 44139
remove redundant lemma
Wed, 10 Aug 2011 14:25:56 -0700 simplify proof of lemma bounded_component
huffman [Wed, 10 Aug 2011 14:25:56 -0700] rev 44138
simplify proof of lemma bounded_component
Wed, 10 Aug 2011 14:10:52 -0700 simplify some proofs
huffman [Wed, 10 Aug 2011 14:10:52 -0700] rev 44137
simplify some proofs
Wed, 10 Aug 2011 13:13:37 -0700 more uniform naming scheme for finite cartesian product type and related theorems
huffman [Wed, 10 Aug 2011 13:13:37 -0700] rev 44136
more uniform naming scheme for finite cartesian product type and related theorems
Wed, 10 Aug 2011 10:13:16 -0700 move euclidean_space instance from Cartesian_Euclidean_Space.thy to Finite_Cartesian_Product.thy
huffman [Wed, 10 Aug 2011 10:13:16 -0700] rev 44135
move euclidean_space instance from Cartesian_Euclidean_Space.thy to Finite_Cartesian_Product.thy
Wed, 10 Aug 2011 21:24:26 +0200 merged
wenzelm [Wed, 10 Aug 2011 21:24:26 +0200] rev 44134
merged
Wed, 10 Aug 2011 09:23:42 -0700 split Linear_Algebra.thy from Euclidean_Space.thy
huffman [Wed, 10 Aug 2011 09:23:42 -0700] rev 44133
split Linear_Algebra.thy from Euclidean_Space.thy
Wed, 10 Aug 2011 08:42:26 -0700 full import paths
huffman [Wed, 10 Aug 2011 08:42:26 -0700] rev 44132
full import paths
Wed, 10 Aug 2011 01:36:53 -0700 declare tendsto_const [intro] (accidentally removed in 230a8665c919)
huffman [Wed, 10 Aug 2011 01:36:53 -0700] rev 44131
declare tendsto_const [intro] (accidentally removed in 230a8665c919)
Wed, 10 Aug 2011 00:31:51 -0700 merged
huffman [Wed, 10 Aug 2011 00:31:51 -0700] rev 44130
merged
Wed, 10 Aug 2011 00:29:31 -0700 simplified definition of class euclidean_space;
huffman [Wed, 10 Aug 2011 00:29:31 -0700] rev 44129
simplified definition of class euclidean_space; removed classes real_basis and real_basis_with_inner
Tue, 09 Aug 2011 13:09:35 -0700 bounded_linear interpretation for euclidean_component
huffman [Tue, 09 Aug 2011 13:09:35 -0700] rev 44128
bounded_linear interpretation for euclidean_component
Tue, 09 Aug 2011 12:50:22 -0700 lemma bounded_linear_intro
huffman [Tue, 09 Aug 2011 12:50:22 -0700] rev 44127
lemma bounded_linear_intro
Tue, 09 Aug 2011 10:42:07 -0700 avoid duplicate rewrite warnings
huffman [Tue, 09 Aug 2011 10:42:07 -0700] rev 44126
avoid duplicate rewrite warnings
Tue, 09 Aug 2011 10:30:00 -0700 mark some redundant theorems as legacy
huffman [Tue, 09 Aug 2011 10:30:00 -0700] rev 44125
mark some redundant theorems as legacy
Tue, 09 Aug 2011 08:53:12 -0700 Derivative.thy: more sensible subsection headings
huffman [Tue, 09 Aug 2011 08:53:12 -0700] rev 44124
Derivative.thy: more sensible subsection headings
Tue, 09 Aug 2011 07:37:18 -0700 Derivative.thy: clean up formatting
huffman [Tue, 09 Aug 2011 07:37:18 -0700] rev 44123
Derivative.thy: clean up formatting
Mon, 08 Aug 2011 21:17:52 -0700 instance real_basis_with_inner < perfect_space
huffman [Mon, 08 Aug 2011 21:17:52 -0700] rev 44122
instance real_basis_with_inner < perfect_space
Wed, 10 Aug 2011 20:53:43 +0200 old term operations are legacy;
wenzelm [Wed, 10 Aug 2011 20:53:43 +0200] rev 44121
old term operations are legacy;
Wed, 10 Aug 2011 20:12:36 +0200 moved old code generator to src/Tools/;
wenzelm [Wed, 10 Aug 2011 20:12:36 +0200] rev 44120
moved old code generator to src/Tools/;
Wed, 10 Aug 2011 19:46:48 +0200 avoid OldTerm operations -- with subtle changes of semantics;
wenzelm [Wed, 10 Aug 2011 19:46:48 +0200] rev 44119
avoid OldTerm operations -- with subtle changes of semantics;
Wed, 10 Aug 2011 19:45:57 +0200 avoid OldTerm operations -- with subtle changes of semantics;
wenzelm [Wed, 10 Aug 2011 19:45:57 +0200] rev 44118
avoid OldTerm operations -- with subtle changes of semantics;
Wed, 10 Aug 2011 19:45:41 +0200 avoid OldTerm operations -- with subtle changes of semantics;
wenzelm [Wed, 10 Aug 2011 19:45:41 +0200] rev 44117
avoid OldTerm operations -- with subtle changes of semantics;
Wed, 10 Aug 2011 19:21:28 +0200 avoid OldTerm operations -- with subtle changes of semantics;
wenzelm [Wed, 10 Aug 2011 19:21:28 +0200] rev 44116
avoid OldTerm operations -- with subtle changes of semantics;
Wed, 10 Aug 2011 16:26:05 +0200 tuned signature;
wenzelm [Wed, 10 Aug 2011 16:26:05 +0200] rev 44115
tuned signature;
Wed, 10 Aug 2011 16:24:39 +0200 Goal.forked: clarified handling of interrupts;
wenzelm [Wed, 10 Aug 2011 16:24:39 +0200] rev 44114
Goal.forked: clarified handling of interrupts;
Wed, 10 Aug 2011 16:05:14 +0200 future_job: explicit indication of interrupts;
wenzelm [Wed, 10 Aug 2011 16:05:14 +0200] rev 44113
future_job: explicit indication of interrupts;
Wed, 10 Aug 2011 15:17:24 +0200 more explicit Simple_Thread.interrupt_unsynchronized, to emphasize its meaning;
wenzelm [Wed, 10 Aug 2011 15:17:24 +0200] rev 44112
more explicit Simple_Thread.interrupt_unsynchronized, to emphasize its meaning;
Wed, 10 Aug 2011 14:28:55 +0200 synchronized cancel and flushing of Multithreading.interrupted state, to ensure that interrupts stay within task boundaries;
wenzelm [Wed, 10 Aug 2011 14:28:55 +0200] rev 44111
synchronized cancel and flushing of Multithreading.interrupted state, to ensure that interrupts stay within task boundaries;
Wed, 10 Aug 2011 14:04:45 +0200 tuned source structure;
wenzelm [Wed, 10 Aug 2011 14:04:45 +0200] rev 44110
tuned source structure;
Wed, 10 Aug 2011 10:59:37 +0200 bash_output_fifo blocks on Cygwin 1.7.x;
wenzelm [Wed, 10 Aug 2011 10:59:37 +0200] rev 44109
bash_output_fifo blocks on Cygwin 1.7.x;
Tue, 09 Aug 2011 23:54:17 +0200 rename_bvs now avoids introducing name clashes between schematic variables
berghofe [Tue, 09 Aug 2011 23:54:17 +0200] rev 44108
rename_bvs now avoids introducing name clashes between schematic variables
Tue, 09 Aug 2011 22:37:33 +0200 merged
wenzelm [Tue, 09 Aug 2011 22:37:33 +0200] rev 44107
merged
Tue, 09 Aug 2011 20:24:48 +0200 tuned proofs
haftmann [Tue, 09 Aug 2011 20:24:48 +0200] rev 44106
tuned proofs
Tue, 09 Aug 2011 18:52:18 +0200 merged
haftmann [Tue, 09 Aug 2011 18:52:18 +0200] rev 44105
merged
Tue, 09 Aug 2011 08:07:22 +0200 tuned header
haftmann [Tue, 09 Aug 2011 08:07:22 +0200] rev 44104
tuned header
Tue, 09 Aug 2011 08:06:15 +0200 more uniform naming scheme for Inf/INF and Sup/SUP lemmas
haftmann [Tue, 09 Aug 2011 08:06:15 +0200] rev 44103
more uniform naming scheme for Inf/INF and Sup/SUP lemmas
Tue, 09 Aug 2011 16:09:10 +0200 removed "extremely ambigous" warning; has been ignored by everyone for years.
kleing [Tue, 09 Aug 2011 16:09:10 +0200] rev 44102
removed "extremely ambigous" warning; has been ignored by everyone for years.
Tue, 09 Aug 2011 22:30:33 +0200 misc tuning and clarification;
wenzelm [Tue, 09 Aug 2011 22:30:33 +0200] rev 44101
misc tuning and clarification;
Tue, 09 Aug 2011 21:48:36 +0200 tuned whitespace;
wenzelm [Tue, 09 Aug 2011 21:48:36 +0200] rev 44100
tuned whitespace;
Tue, 09 Aug 2011 17:33:17 +0200 support local HOATPs
blanchet [Tue, 09 Aug 2011 17:33:17 +0200] rev 44099
support local HOATPs
Tue, 09 Aug 2011 17:33:17 +0200 document local HOATPs
blanchet [Tue, 09 Aug 2011 17:33:17 +0200] rev 44098
document local HOATPs
Tue, 09 Aug 2011 17:33:17 +0200 workaround THF parser limitation
blanchet [Tue, 09 Aug 2011 17:33:17 +0200] rev 44097
workaround THF parser limitation
Tue, 09 Aug 2011 17:33:17 +0200 LEO-II also supports FOF
blanchet [Tue, 09 Aug 2011 17:33:17 +0200] rev 44096
LEO-II also supports FOF
Tue, 09 Aug 2011 15:50:13 +0200 misc tuning and simplification;
wenzelm [Tue, 09 Aug 2011 15:50:13 +0200] rev 44095
misc tuning and simplification;
Tue, 09 Aug 2011 15:41:00 +0200 updated documentation of method "split" according to e6a4bb832b46;
wenzelm [Tue, 09 Aug 2011 15:41:00 +0200] rev 44094
updated documentation of method "split" according to e6a4bb832b46;
Tue, 09 Aug 2011 09:39:49 +0200 updated references to CADE-23
blanchet [Tue, 09 Aug 2011 09:39:49 +0200] rev 44093
updated references to CADE-23
Tue, 09 Aug 2011 09:33:50 +0200 renamed E wrappers for consistency with CASC conventions
blanchet [Tue, 09 Aug 2011 09:33:50 +0200] rev 44092
renamed E wrappers for consistency with CASC conventions
Tue, 09 Aug 2011 09:33:01 +0200 updated Sledgehammer docs
blanchet [Tue, 09 Aug 2011 09:33:01 +0200] rev 44091
updated Sledgehammer docs
Tue, 09 Aug 2011 09:24:34 +0200 add line number prefix to output file name
blanchet [Tue, 09 Aug 2011 09:24:34 +0200] rev 44090
add line number prefix to output file name
Tue, 09 Aug 2011 09:07:59 +0200 added "sound" option to Mirabelle
blanchet [Tue, 09 Aug 2011 09:07:59 +0200] rev 44089
added "sound" option to Mirabelle
Tue, 09 Aug 2011 09:05:22 +0200 move lambda-lifting code to ATP encoding, so it can be used by Metis
blanchet [Tue, 09 Aug 2011 09:05:22 +0200] rev 44088
move lambda-lifting code to ATP encoding, so it can be used by Metis
Tue, 09 Aug 2011 09:05:21 +0200 load lambda-lifting structure earlier, so it can be used in Metis
blanchet [Tue, 09 Aug 2011 09:05:21 +0200] rev 44087
load lambda-lifting structure earlier, so it can be used in Metis
Tue, 09 Aug 2011 07:44:17 +0200 merged
haftmann [Tue, 09 Aug 2011 07:44:17 +0200] rev 44086
merged
Mon, 08 Aug 2011 22:33:36 +0200 move legacy candiates to bottom; marked candidates for default simp rules
haftmann [Mon, 08 Aug 2011 22:33:36 +0200] rev 44085
move legacy candiates to bottom; marked candidates for default simp rules
Mon, 08 Aug 2011 22:11:00 +0200 merged
haftmann [Mon, 08 Aug 2011 22:11:00 +0200] rev 44084
merged
Mon, 08 Aug 2011 19:30:18 +0200 dropped lemmas (Inf|Sup)_(singleton|binary)
haftmann [Mon, 08 Aug 2011 19:30:18 +0200] rev 44083
dropped lemmas (Inf|Sup)_(singleton|binary)
Mon, 08 Aug 2011 19:21:11 +0200 dropped lemmas (Inf|Sup)_(singleton|binary)
haftmann [Mon, 08 Aug 2011 19:21:11 +0200] rev 44082
dropped lemmas (Inf|Sup)_(singleton|binary)
Mon, 08 Aug 2011 19:26:53 -0700 rename type 'a net to 'a filter, following standard mathematical terminology
huffman [Mon, 08 Aug 2011 19:26:53 -0700] rev 44081
rename type 'a net to 'a filter, following standard mathematical terminology
Mon, 08 Aug 2011 18:36:32 -0700 HOLCF: fix warnings about unreferenced identifiers
huffman [Mon, 08 Aug 2011 18:36:32 -0700] rev 44080
HOLCF: fix warnings about unreferenced identifiers
Mon, 08 Aug 2011 16:57:37 -0700 remove duplicate lemmas
huffman [Mon, 08 Aug 2011 16:57:37 -0700] rev 44079
remove duplicate lemmas
Mon, 08 Aug 2011 16:19:57 -0700 merged
huffman [Mon, 08 Aug 2011 16:19:57 -0700] rev 44078
merged
Mon, 08 Aug 2011 16:04:58 -0700 fix perfect_space instance proof for finite cartesian product (cf. 5b970711fb39)
huffman [Mon, 08 Aug 2011 16:04:58 -0700] rev 44077
fix perfect_space instance proof for finite cartesian product (cf. 5b970711fb39)
Mon, 08 Aug 2011 15:27:24 -0700 generalize sequence lemmas
huffman [Mon, 08 Aug 2011 15:27:24 -0700] rev 44076
generalize sequence lemmas
Mon, 08 Aug 2011 15:11:38 -0700 generalize more lemmas about compactness
huffman [Mon, 08 Aug 2011 15:11:38 -0700] rev 44075
generalize more lemmas about compactness
Mon, 08 Aug 2011 15:03:34 -0700 generalize compactness equivalence lemmas
huffman [Mon, 08 Aug 2011 15:03:34 -0700] rev 44074
generalize compactness equivalence lemmas
Mon, 08 Aug 2011 14:59:01 -0700 lemma bolzano_weierstrass_imp_compact
huffman [Mon, 08 Aug 2011 14:59:01 -0700] rev 44073
lemma bolzano_weierstrass_imp_compact
Mon, 08 Aug 2011 14:44:20 -0700 class perfect_space inherits from topological_space;
huffman [Mon, 08 Aug 2011 14:44:20 -0700] rev 44072
class perfect_space inherits from topological_space; generalized several lemmas
Mon, 08 Aug 2011 21:55:01 +0200 merged
wenzelm [Mon, 08 Aug 2011 21:55:01 +0200] rev 44071
merged
Mon, 08 Aug 2011 16:47:55 +0200 import constant folding theory into IMP
kleing [Mon, 08 Aug 2011 16:47:55 +0200] rev 44070
import constant folding theory into IMP
Sat, 06 Aug 2011 15:48:08 +0200 make syntax ambiguity warnings a config option
kleing [Sat, 06 Aug 2011 15:48:08 +0200] rev 44069
make syntax ambiguity warnings a config option
Mon, 08 Aug 2011 11:47:41 -0700 add lemmas INF_image, SUP_image
huffman [Mon, 08 Aug 2011 11:47:41 -0700] rev 44068
add lemmas INF_image, SUP_image
Mon, 08 Aug 2011 11:25:18 -0700 declare {INF,SUP}_empty [simp]
huffman [Mon, 08 Aug 2011 11:25:18 -0700] rev 44067
declare {INF,SUP}_empty [simp]
Mon, 08 Aug 2011 10:32:55 -0700 rename Pair_fst_snd_eq to prod_eq_iff (keeping old name too)
huffman [Mon, 08 Aug 2011 10:32:55 -0700] rev 44066
rename Pair_fst_snd_eq to prod_eq_iff (keeping old name too)
Mon, 08 Aug 2011 10:26:26 -0700 standard theorem naming scheme: complex_eqI, complex_eq_iff
huffman [Mon, 08 Aug 2011 10:26:26 -0700] rev 44065
standard theorem naming scheme: complex_eqI, complex_eq_iff
Mon, 08 Aug 2011 09:52:09 -0700 moved division ring stuff from Rings.thy to Fields.thy
huffman [Mon, 08 Aug 2011 09:52:09 -0700] rev 44064
moved division ring stuff from Rings.thy to Fields.thy
Mon, 08 Aug 2011 08:55:49 -0700 Library/Product_ord: wellorder instance for products
huffman [Mon, 08 Aug 2011 08:55:49 -0700] rev 44063
Library/Product_ord: wellorder instance for products
Mon, 08 Aug 2011 21:11:10 +0200 modernized file proof_checker.ML;
wenzelm [Mon, 08 Aug 2011 21:11:10 +0200] rev 44062
modernized file proof_checker.ML;
Mon, 08 Aug 2011 20:47:12 +0200 tuned thm_of_proof: build lookup table within closure;
wenzelm [Mon, 08 Aug 2011 20:47:12 +0200] rev 44061
tuned thm_of_proof: build lookup table within closure;
Mon, 08 Aug 2011 20:21:49 +0200 added Reconstruct.proof_of convenience;
wenzelm [Mon, 08 Aug 2011 20:21:49 +0200] rev 44060
added Reconstruct.proof_of convenience;
Mon, 08 Aug 2011 19:59:35 +0200 ship message in one piece;
wenzelm [Mon, 08 Aug 2011 19:59:35 +0200] rev 44059
ship message in one piece;
Mon, 08 Aug 2011 17:23:15 +0200 misc tuning -- eliminated old-fashioned rep_thm;
wenzelm [Mon, 08 Aug 2011 17:23:15 +0200] rev 44058
misc tuning -- eliminated old-fashioned rep_thm;
Mon, 08 Aug 2011 16:38:59 +0200 modernized strcture Proof_Checker;
wenzelm [Mon, 08 Aug 2011 16:38:59 +0200] rev 44057
modernized strcture Proof_Checker;
Mon, 08 Aug 2011 16:09:34 +0200 less ambitious use of AttributedString, for proper caret painting within \<^sup>\<foobar>;
wenzelm [Mon, 08 Aug 2011 16:09:34 +0200] rev 44056
less ambitious use of AttributedString, for proper caret painting within \<^sup>\<foobar>;
Mon, 08 Aug 2011 13:48:38 +0200 updated imports;
wenzelm [Mon, 08 Aug 2011 13:48:38 +0200] rev 44055
updated imports;
Mon, 08 Aug 2011 13:40:24 +0200 proper signature;
wenzelm [Mon, 08 Aug 2011 13:40:24 +0200] rev 44054
proper signature;
Mon, 08 Aug 2011 13:39:51 +0200 made SML/NJ happy;
wenzelm [Mon, 08 Aug 2011 13:39:51 +0200] rev 44053
made SML/NJ happy;
Mon, 08 Aug 2011 13:29:54 +0200 slightly more uniform messages;
wenzelm [Mon, 08 Aug 2011 13:29:54 +0200] rev 44052
slightly more uniform messages;
Mon, 08 Aug 2011 13:19:19 +0200 avoid pointless completion of illegal control commands;
wenzelm [Mon, 08 Aug 2011 13:19:19 +0200] rev 44051
avoid pointless completion of illegal control commands;
Mon, 08 Aug 2011 08:56:58 +0200 removed old expand_fun_eq
nipkow [Mon, 08 Aug 2011 08:56:58 +0200] rev 44050
removed old expand_fun_eq
Mon, 08 Aug 2011 08:25:28 +0200 fixed index entry
nipkow [Mon, 08 Aug 2011 08:25:28 +0200] rev 44049
fixed index entry
Mon, 08 Aug 2011 07:35:42 +0200 removed old recdef and types usage
nipkow [Mon, 08 Aug 2011 07:35:42 +0200] rev 44048
removed old recdef and types usage
Mon, 08 Aug 2011 07:13:16 +0200 merged
nipkow [Mon, 08 Aug 2011 07:13:16 +0200] rev 44047
merged
Sat, 06 Aug 2011 14:16:23 +0200 extended user-level attribute case_names with names for case hypotheses
nipkow [Sat, 06 Aug 2011 14:16:23 +0200] rev 44046
extended user-level attribute case_names with names for case hypotheses
Mon, 01 Aug 2011 12:08:53 +0200 infrastructure for attaching names to hypothesis in cases; realised via the same tag mechanism as case names
nipkow [Mon, 01 Aug 2011 12:08:53 +0200] rev 44045
infrastructure for attaching names to hypothesis in cases; realised via the same tag mechanism as case names
Sun, 07 Aug 2011 23:08:07 +0200 workaround for Java 1.7 where javax.swing.JComboBox<E> is generic;
wenzelm [Sun, 07 Aug 2011 23:08:07 +0200] rev 44044
workaround for Java 1.7 where javax.swing.JComboBox<E> is generic;
Sun, 07 Aug 2011 23:05:50 +0200 updated version information;
wenzelm [Sun, 07 Aug 2011 23:05:50 +0200] rev 44043
updated version information;
Sun, 07 Aug 2011 18:38:36 +0200 fixed document;
wenzelm [Sun, 07 Aug 2011 18:38:36 +0200] rev 44042
fixed document;
Fri, 05 Aug 2011 23:06:54 +0200 tuned order: pushing INF and SUP to Inf and Sup
haftmann [Fri, 05 Aug 2011 23:06:54 +0200] rev 44041
tuned order: pushing INF and SUP to Inf and Sup
Fri, 05 Aug 2011 22:58:17 +0200 tuned order: pushing INF and SUP to Inf and Sup
haftmann [Fri, 05 Aug 2011 22:58:17 +0200] rev 44040
tuned order: pushing INF and SUP to Inf and Sup
Fri, 05 Aug 2011 22:45:57 +0200 generalized lemmas to complete lattices
haftmann [Fri, 05 Aug 2011 22:45:57 +0200] rev 44039
generalized lemmas to complete lattices
Fri, 05 Aug 2011 17:22:28 +0200 merged
Andreas Lochbihler [Fri, 05 Aug 2011 17:22:28 +0200] rev 44038
merged
Fri, 05 Aug 2011 16:55:14 +0200 replace old SML code generator by new code generator in MicroJava/J
Andreas Lochbihler [Fri, 05 Aug 2011 16:55:14 +0200] rev 44037
replace old SML code generator by new code generator in MicroJava/J
Thu, 04 Aug 2011 16:49:57 +0200 new state syntax with less conflicts
kleing [Thu, 04 Aug 2011 16:49:57 +0200] rev 44036
new state syntax with less conflicts
Fri, 05 Aug 2011 14:16:44 +0200 replace old SML code generator by new code generator in MicroJava/JVM and /BV
Andreas Lochbihler [Fri, 05 Aug 2011 14:16:44 +0200] rev 44035
replace old SML code generator by new code generator in MicroJava/JVM and /BV
Fri, 05 Aug 2011 00:14:08 +0200 merged
haftmann [Fri, 05 Aug 2011 00:14:08 +0200] rev 44034
merged
Thu, 04 Aug 2011 20:11:39 +0200 more fine-granular instantiation
haftmann [Thu, 04 Aug 2011 20:11:39 +0200] rev 44033
more fine-granular instantiation
Thu, 04 Aug 2011 19:29:52 +0200 solving duality problem for complete_distrib_lattice; tuned
haftmann [Thu, 04 Aug 2011 19:29:52 +0200] rev 44032
solving duality problem for complete_distrib_lattice; tuned
Thu, 04 Aug 2011 23:21:04 +0200 merged
berghofe [Thu, 04 Aug 2011 23:21:04 +0200] rev 44031
merged
Thu, 04 Aug 2011 17:40:48 +0200 Pending FDL types may now be associated with Isabelle types as well.
berghofe [Thu, 04 Aug 2011 17:40:48 +0200] rev 44030
Pending FDL types may now be associated with Isabelle types as well.
Thu, 04 Aug 2011 07:33:08 +0200 tuned orthography
haftmann [Thu, 04 Aug 2011 07:33:08 +0200] rev 44029
tuned orthography
Thu, 04 Aug 2011 07:31:59 +0200 avoid yet unknown fact antiquotation
haftmann [Thu, 04 Aug 2011 07:31:59 +0200] rev 44028
avoid yet unknown fact antiquotation
Thu, 04 Aug 2011 07:31:43 +0200 NEWS
haftmann [Thu, 04 Aug 2011 07:31:43 +0200] rev 44027
NEWS
Wed, 03 Aug 2011 23:21:53 +0200 more specific instantiation
haftmann [Wed, 03 Aug 2011 23:21:53 +0200] rev 44026
more specific instantiation
Wed, 03 Aug 2011 23:21:52 +0200 tuned
haftmann [Wed, 03 Aug 2011 23:21:52 +0200] rev 44025
tuned
Wed, 03 Aug 2011 23:21:52 +0200 class complete_distrib_lattice
haftmann [Wed, 03 Aug 2011 23:21:52 +0200] rev 44024
class complete_distrib_lattice
Wed, 03 Aug 2011 16:08:02 +0200 NEWS
bulwahn [Wed, 03 Aug 2011 16:08:02 +0200] rev 44023
NEWS
Wed, 03 Aug 2011 14:24:23 +0200 removing value invocations with the SML code generator
bulwahn [Wed, 03 Aug 2011 14:24:23 +0200] rev 44022
removing value invocations with the SML code generator
Wed, 03 Aug 2011 13:59:59 +0200 removing the SML evaluator
bulwahn [Wed, 03 Aug 2011 13:59:59 +0200] rev 44021
removing the SML evaluator
Wed, 03 Aug 2011 11:09:12 +0200 fixed wrong isubs in IMP/Types
kleing [Wed, 03 Aug 2011 11:09:12 +0200] rev 44020
fixed wrong isubs in IMP/Types
Tue, 02 Aug 2011 08:28:34 -0700 Extended_Nat.thy: renamed iSuc to eSuc, standardized theorem names
huffman [Tue, 02 Aug 2011 08:28:34 -0700] rev 44019
Extended_Nat.thy: renamed iSuc to eSuc, standardized theorem names
Tue, 02 Aug 2011 07:36:58 -0700 NEWS: fix typo
huffman [Tue, 02 Aug 2011 07:36:58 -0700] rev 44018
NEWS: fix typo
Tue, 02 Aug 2011 13:07:00 +0200 updated unchecked forward reference
krauss [Tue, 02 Aug 2011 13:07:00 +0200] rev 44017
updated unchecked forward reference
Tue, 02 Aug 2011 12:27:24 +0200 replaced Nitpick's hardwired basic_ersatz_table by context data
krauss [Tue, 02 Aug 2011 12:27:24 +0200] rev 44016
replaced Nitpick's hardwired basic_ersatz_table by context data
Tue, 02 Aug 2011 12:17:48 +0200 NEWS
krauss [Tue, 02 Aug 2011 12:17:48 +0200] rev 44015
NEWS
Tue, 02 Aug 2011 11:52:57 +0200 moved recursion combinator to HOL/Library/Wfrec.thy -- it is so fundamental and well-known that it should survive recdef
krauss [Tue, 02 Aug 2011 11:52:57 +0200] rev 44014
moved recursion combinator to HOL/Library/Wfrec.thy -- it is so fundamental and well-known that it should survive recdef
Tue, 02 Aug 2011 10:36:50 +0200 moved recdef package to HOL/Library/Old_Recdef.thy
krauss [Tue, 02 Aug 2011 10:36:50 +0200] rev 44013
moved recdef package to HOL/Library/Old_Recdef.thy
Tue, 02 Aug 2011 10:03:14 +0200 added dynamic ersatz_table to Nitpick's data slot
krauss [Tue, 02 Aug 2011 10:03:14 +0200] rev 44012
added dynamic ersatz_table to Nitpick's data slot
Tue, 02 Aug 2011 10:03:12 +0200 eliminated obsolete recdef/wfrec related declarations
krauss [Tue, 02 Aug 2011 10:03:12 +0200] rev 44011
eliminated obsolete recdef/wfrec related declarations
Mon, 01 Aug 2011 20:21:11 +0200 more consistent naming in IMP/Comp_Rev
kleing [Mon, 01 Aug 2011 20:21:11 +0200] rev 44010
more consistent naming in IMP/Comp_Rev
Mon, 01 Aug 2011 19:53:30 +0200 merged
haftmann [Mon, 01 Aug 2011 19:53:30 +0200] rev 44009
merged
Sat, 30 Jul 2011 08:24:46 +0200 tuned proofs
haftmann [Sat, 30 Jul 2011 08:24:46 +0200] rev 44008
tuned proofs
Fri, 29 Jul 2011 19:47:55 +0200 tuned proofs
haftmann [Fri, 29 Jul 2011 19:47:55 +0200] rev 44007
tuned proofs
Mon, 01 Aug 2011 09:31:10 -0700 new theory HOL/Library/Product_Lattice.thy
huffman [Mon, 01 Aug 2011 09:31:10 -0700] rev 44006
new theory HOL/Library/Product_Lattice.thy
Sun, 31 Jul 2011 11:13:38 -0700 domain package: more informative error message for illegal indirect recursion
huffman [Sun, 31 Jul 2011 11:13:38 -0700] rev 44005
domain package: more informative error message for illegal indirect recursion
Thu, 28 Jul 2011 16:56:14 +0200 compiler proof cleanup
kleing [Thu, 28 Jul 2011 16:56:14 +0200] rev 44004
compiler proof cleanup
Thu, 28 Jul 2011 16:32:49 +0200 added helpers for "All" and "Ex"
blanchet [Thu, 28 Jul 2011 16:32:49 +0200] rev 44003
added helpers for "All" and "Ex"
Thu, 28 Jul 2011 16:32:48 +0200 put parentheses around non-trivial metis call
blanchet [Thu, 28 Jul 2011 16:32:48 +0200] rev 44002
put parentheses around non-trivial metis call
Thu, 28 Jul 2011 16:32:39 +0200 no needless mangling
blanchet [Thu, 28 Jul 2011 16:32:39 +0200] rev 44001
no needless mangling
Thu, 28 Jul 2011 15:15:26 +0200 resolved code_pred FIXME in IMP; clearer notation for exec_n
kleing [Thu, 28 Jul 2011 15:15:26 +0200] rev 44000
resolved code_pred FIXME in IMP; clearer notation for exec_n
Thu, 28 Jul 2011 11:49:03 +0200 clean up temporary directory hack
blanchet [Thu, 28 Jul 2011 11:49:03 +0200] rev 43999
clean up temporary directory hack
Thu, 28 Jul 2011 11:43:45 +0200 tuning
blanchet [Thu, 28 Jul 2011 11:43:45 +0200] rev 43998
tuning
Thu, 28 Jul 2011 11:43:45 +0200 fixed lambda concealing
blanchet [Thu, 28 Jul 2011 11:43:45 +0200] rev 43997
fixed lambda concealing
Thu, 28 Jul 2011 11:43:45 +0200 make SML/NJ happy
blanchet [Thu, 28 Jul 2011 11:43:45 +0200] rev 43996
make SML/NJ happy
Thu, 28 Jul 2011 10:42:24 +0200 simplified definition of vector (also removed Cartesian_Euclidean_Space.from_nat which collides with Countable.from_nat)
hoelzl [Thu, 28 Jul 2011 10:42:24 +0200] rev 43995
simplified definition of vector (also removed Cartesian_Euclidean_Space.from_nat which collides with Countable.from_nat)
Thu, 28 Jul 2011 05:52:28 -0200 document coercions
noschinl [Thu, 28 Jul 2011 05:52:28 -0200] rev 43994
document coercions
Wed, 27 Jul 2011 20:28:00 +0200 rudimentary documentation of the quotient package in the isar reference manual
bulwahn [Wed, 27 Jul 2011 20:28:00 +0200] rev 43993
rudimentary documentation of the quotient package in the isar reference manual
Wed, 27 Jul 2011 19:35:00 +0200 to_nat is injective on arbitrary domains
hoelzl [Wed, 27 Jul 2011 19:35:00 +0200] rev 43992
to_nat is injective on arbitrary domains
Wed, 27 Jul 2011 19:34:30 +0200 finite vimage on arbitrary domains
hoelzl [Wed, 27 Jul 2011 19:34:30 +0200] rev 43991
finite vimage on arbitrary domains
Tue, 26 Jul 2011 22:53:06 +0200 updated Sledgehammer documentation
blanchet [Tue, 26 Jul 2011 22:53:06 +0200] rev 43990
updated Sledgehammer documentation
Tue, 26 Jul 2011 22:53:06 +0200 renamed "preds" encodings to "guards"
blanchet [Tue, 26 Jul 2011 22:53:06 +0200] rev 43989
renamed "preds" encodings to "guards"
Tue, 26 Jul 2011 18:11:38 +0200 more precise dependencies
bulwahn [Tue, 26 Jul 2011 18:11:38 +0200] rev 43988
more precise dependencies
Tue, 26 Jul 2011 14:53:00 +0200 further worked around LEO-II parser limitation, with eta-expansion
blanchet [Tue, 26 Jul 2011 14:53:00 +0200] rev 43987
further worked around LEO-II parser limitation, with eta-expansion
Tue, 26 Jul 2011 14:53:00 +0200 use syntactic sugar whenever possible in THF problems, to work around current LEO-II parser limitation (bang bang and query query are not handled correctly)
blanchet [Tue, 26 Jul 2011 14:53:00 +0200] rev 43986
use syntactic sugar whenever possible in THF problems, to work around current LEO-II parser limitation (bang bang and query query are not handled correctly)
Tue, 26 Jul 2011 14:53:00 +0200 no need for existential witnesses for sorts in TFF and THF formats
blanchet [Tue, 26 Jul 2011 14:53:00 +0200] rev 43985
no need for existential witnesses for sorts in TFF and THF formats
Tue, 26 Jul 2011 14:53:00 +0200 mangle "undefined"
blanchet [Tue, 26 Jul 2011 14:53:00 +0200] rev 43984
mangle "undefined"
Tue, 26 Jul 2011 14:53:00 +0200 tuning -- remove useless function (at this point combinators are already in)
blanchet [Tue, 26 Jul 2011 14:53:00 +0200] rev 43983
tuning -- remove useless function (at this point combinators are already in)
Tue, 26 Jul 2011 14:53:00 +0200 remove spurious message
blanchet [Tue, 26 Jul 2011 14:53:00 +0200] rev 43982
remove spurious message
Tue, 26 Jul 2011 14:53:00 +0200 give E at least two seconds -- anything else risks causing too early timeouts in the minimizer, because of too conservative time computations in E and eproof scripts
blanchet [Tue, 26 Jul 2011 14:53:00 +0200] rev 43981
give E at least two seconds -- anything else risks causing too early timeouts in the minimizer, because of too conservative time computations in E and eproof scripts
Tue, 26 Jul 2011 14:50:15 +0200 merged
Andreas Lochbihler [Tue, 26 Jul 2011 14:50:15 +0200] rev 43980
merged
Tue, 26 Jul 2011 14:05:28 +0200 fixed code generator setup in List_Cset
Andreas Lochbihler [Tue, 26 Jul 2011 14:05:28 +0200] rev 43979
fixed code generator setup in List_Cset
Tue, 26 Jul 2011 13:50:03 +0200 enat is a complete_linorder instance
hoelzl [Tue, 26 Jul 2011 13:50:03 +0200] rev 43978
enat is a complete_linorder instance
Tue, 26 Jul 2011 12:44:36 +0200 merged
Andreas Lochbihler [Tue, 26 Jul 2011 12:44:36 +0200] rev 43977
merged
Tue, 26 Jul 2011 10:49:34 +0200 Add theory for setting up monad syntax for Cset
Andreas Lochbihler [Tue, 26 Jul 2011 10:49:34 +0200] rev 43976
Add theory for setting up monad syntax for Cset
Tue, 26 Jul 2011 11:48:11 +0200 merged
bulwahn [Tue, 26 Jul 2011 11:48:11 +0200] rev 43975
merged
(0) -30000 -10000 -3000 -1000 -480 +480 +1000 +3000 +10000 +30000 tip