huffman [Tue, 23 Aug 2011 16:17:22 -0700] rev 44465
move connected_real_lemma to the one place it is used
wenzelm [Wed, 24 Aug 2011 17:30:25 +0200] rev 44464
merged
blanchet [Wed, 24 Aug 2011 15:25:39 +0200] rev 44463
make sure that all facts are passed to ATP from minimizer
blanchet [Wed, 24 Aug 2011 11:17:33 +0200] rev 44462
more reliable "sledgehammer\_tac" reconstruction, by avoiding "insert_tac"
blanchet [Wed, 24 Aug 2011 11:17:33 +0200] rev 44461
specify timeout for "sledgehammer_tac"
blanchet [Wed, 24 Aug 2011 11:17:33 +0200] rev 44460
tuning
Cezary Kaliszyk <kaliszyk@in.tum.de> [Wed, 24 Aug 2011 10:59:22 +0900] rev 44459
Quotient Package: add mem_rsp, mem_prs, tune proofs.
huffman [Tue, 23 Aug 2011 15:46:53 -0700] rev 44458
merged
huffman [Tue, 23 Aug 2011 14:11:02 -0700] rev 44457
declare euclidean_simps [simp] at the point they are proved;
avoid duplicate rule warnings;
huffman [Tue, 23 Aug 2011 07:12:05 -0700] rev 44456
merged
huffman [Mon, 22 Aug 2011 18:15:33 -0700] rev 44455
merged
huffman [Mon, 22 Aug 2011 17:22:49 -0700] rev 44454
avoid warnings
huffman [Mon, 22 Aug 2011 16:49:45 -0700] rev 44453
comment out dead code to avoid compiler warnings
huffman [Mon, 22 Aug 2011 10:43:10 -0700] rev 44452
legacy theorem names
huffman [Mon, 22 Aug 2011 10:19:39 -0700] rev 44451
remove duplicate lemma
blanchet [Tue, 23 Aug 2011 23:18:13 +0200] rev 44450
fixed "hBOOL" of existential variables, and generate more helpers
blanchet [Tue, 23 Aug 2011 22:44:08 +0200] rev 44449
don't select facts when using sledgehammer_tac for reconstruction
blanchet [Tue, 23 Aug 2011 20:35:41 +0200] rev 44448
don't perform a triviality check if the goal is skipped anyway
blanchet [Tue, 23 Aug 2011 19:50:25 +0200] rev 44447
optional reconstructor
wenzelm [Wed, 24 Aug 2011 17:25:45 +0200] rev 44446
misc tuning and simplification;
wenzelm [Wed, 24 Aug 2011 17:16:48 +0200] rev 44445
tuned pri: prefer purging of canceled execution;
wenzelm [Wed, 24 Aug 2011 17:14:31 +0200] rev 44444
tuned Document.node: maintain "touched" flag to indicate changes in entries etc.;
wenzelm [Wed, 24 Aug 2011 16:49:48 +0200] rev 44443
clarified Document.Node.clear -- retain header (cf. ML version);
wenzelm [Wed, 24 Aug 2011 16:27:27 +0200] rev 44442
clarified norm_header/header_edit -- disallow update of loaded theories;
wenzelm [Wed, 24 Aug 2011 15:55:43 +0200] rev 44441
misc tuning and simplification;
wenzelm [Wed, 24 Aug 2011 15:30:43 +0200] rev 44440
ignore irrelevant timings;
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;
wenzelm [Wed, 24 Aug 2011 13:38:07 +0200] rev 44438
early filtering of unchanged perspective;
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);
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;
wenzelm [Tue, 23 Aug 2011 21:19:24 +0200] rev 44435
tuned;
wenzelm [Tue, 23 Aug 2011 21:14:59 +0200] rev 44434
handle potentially more approriate BufferUpdate.LOADED event;
wenzelm [Mon, 22 Aug 2011 23:39:05 +0200] rev 44433
special treatment of structure index 1 in Pure, including legacy warning;
blanchet [Tue, 23 Aug 2011 19:49:21 +0200] rev 44432
compile
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
blanchet [Tue, 23 Aug 2011 18:42:05 +0200] rev 44430
beef up "sledgehammer_tac" reconstructor
blanchet [Tue, 23 Aug 2011 18:42:05 +0200] rev 44429
clean up Sledgehammer tactic
wenzelm [Tue, 23 Aug 2011 17:44:31 +0200] rev 44428
fixed document;
wenzelm [Tue, 23 Aug 2011 17:43:06 +0200] rev 44427
tuned signature;
wenzelm [Tue, 23 Aug 2011 17:12:54 +0200] rev 44426
merged
blanchet [Tue, 23 Aug 2011 16:37:23 +0200] rev 44425
always use TFF if possible
blanchet [Tue, 23 Aug 2011 16:14:19 +0200] rev 44424
clearer separator in generated file names
blanchet [Tue, 23 Aug 2011 16:07:01 +0200] rev 44423
exploit TFF format in Z3 used as ATP, and renamed it "z3_tptp"
blanchet [Tue, 23 Aug 2011 15:50:27 +0200] rev 44422
updated known failures for Z3 3.0 TPTP
blanchet [Tue, 23 Aug 2011 15:18:46 +0200] rev 44421
updated Z3 docs
blanchet [Tue, 23 Aug 2011 15:15:43 +0200] rev 44420
avoid TFF format with older Vampire versions
blanchet [Tue, 23 Aug 2011 14:57:16 +0200] rev 44419
update the Vampire related parts of the documentation
blanchet [Tue, 23 Aug 2011 14:44:19 +0200] rev 44418
fixed TFF slicing
blanchet [Tue, 23 Aug 2011 14:44:19 +0200] rev 44417
kindly ask Vampire to output axiom names
blanchet [Tue, 23 Aug 2011 14:44:19 +0200] rev 44416
added formats to the slice and use TFF for remote Vampire
haftmann [Tue, 23 Aug 2011 07:14:09 +0200] rev 44415
tuned specifications, syntax and proofs
haftmann [Mon, 22 Aug 2011 22:00:36 +0200] rev 44414
tuned specifications and syntax
Cezary Kaliszyk <kaliszyk@in.tum.de> [Tue, 23 Aug 2011 03:34:17 +0900] rev 44413
Quotient Package: some infrastructure for lifting inside sets
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
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44411
change Metis's default settings if type information axioms are generated
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44410
we must tag any type whose ground types intersect a nonmonotonic type
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44409
prefer the lighter, slightly unsound monotonicity-based encodings for Metis
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44408
made reconstruction of type tag equalities "\?x = \?x" reliable
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44407
tuning ATP problem output
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44406
revert guard logic -- make sure that typing information is generated for existentials
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44405
generate tag equations for existential variables
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44404
tuning, plus started implementing tag equation generation for existential variables
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
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44402
clearer terminology
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44401
renamed "heavy" to "uniform", based on discussion with Nick Smallbone
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44400
removed unused configuration option
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44399
added caching for (in)finiteness checks
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44398
remove needless typing information
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44397
cleaner handling of polymorphic monotonicity inference
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44396
started cleaning up polymorphic monotonicity-based encodings, based on discussions with Nick Smallbone
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44395
more precise warning
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44394
added option to control soundness of encodings more precisely, for evaluation purposes
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44393
make sound mode more sound (and clean up code)
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
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44391
gracefully handle empty SPASS problems
blanchet [Mon, 22 Aug 2011 15:02:45 +0200] rev 44390
pass sound option to Sledgehammer tactic
wenzelm [Tue, 23 Aug 2011 16:53:05 +0200] rev 44389
tuned signature -- contrast physical output primitives versus Output.raw_message;
wenzelm [Tue, 23 Aug 2011 16:41:16 +0200] rev 44388
tuned signature;
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);
wenzelm [Tue, 23 Aug 2011 15:48:41 +0200] rev 44386
some support for toplevel printing wrt. editor perspective (still inactive);
wenzelm [Tue, 23 Aug 2011 12:20:12 +0200] rev 44385
propagate editor perspective through document model;
wenzelm [Mon, 22 Aug 2011 21:42:02 +0200] rev 44384
some support for editor perspective;
wenzelm [Mon, 22 Aug 2011 21:09:26 +0200] rev 44383
discontinued redundant Edit_Command_ID;
wenzelm [Mon, 22 Aug 2011 20:11:44 +0200] rev 44382
reduced warnings;
wenzelm [Mon, 22 Aug 2011 20:00:04 +0200] rev 44381
tuned message;
wenzelm [Mon, 22 Aug 2011 17:10:22 +0200] rev 44380
old-style numbered structure index is legacy feature (hardly ever used now);
wenzelm [Mon, 22 Aug 2011 16:12:23 +0200] rev 44379
added official Text.Range.Ordering;
some support for text perspective;
wenzelm [Mon, 22 Aug 2011 14:15:52 +0200] rev 44378
tuned signature;
wenzelm [Mon, 22 Aug 2011 12:17:22 +0200] rev 44377
reverted some odd changes to HOL/Import (cf. 74c08021ab2e);
krauss [Mon, 22 Aug 2011 10:57:33 +0200] rev 44376
merged
krauss [Sun, 21 Aug 2011 22:13:04 +0200] rev 44375
modernized specifications
krauss [Sun, 21 Aug 2011 22:13:04 +0200] rev 44374
removed session HOL/Subst -- now subsumed my more modern HOL/ex/Unification.thy
krauss [Sun, 21 Aug 2011 22:13:04 +0200] rev 44373
removed technical or trivial unused facts
krauss [Sun, 21 Aug 2011 22:13:04 +0200] rev 44372
more precise authors and comments;
tuned order and headers
krauss [Sun, 21 Aug 2011 22:13:04 +0200] rev 44371
added proof of idempotence, roughly after HOL/Subst/Unify.thy
krauss [Sun, 21 Aug 2011 22:13:04 +0200] rev 44370
tuned proofs, sledgehammering overly verbose parts
krauss [Sun, 21 Aug 2011 22:13:04 +0200] rev 44369
tuned notation
krauss [Sun, 21 Aug 2011 22:13:04 +0200] rev 44368
ported some lemmas from HOL/Subst/*;
tuned order
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.
huffman [Sun, 21 Aug 2011 21:18:59 -0700] rev 44366
merged
huffman [Sun, 21 Aug 2011 12:22:31 -0700] rev 44365
add lemmas interior_Times and closure_Times
haftmann [Sun, 21 Aug 2011 22:56:55 +0200] rev 44364
avoid pred/set mixture
haftmann [Sun, 21 Aug 2011 19:47:52 +0200] rev 44363
avoid pred/set mixture
wenzelm [Sun, 21 Aug 2011 22:04:01 +0200] rev 44362
merged
huffman [Sun, 21 Aug 2011 11:03:15 -0700] rev 44361
remove unnecessary euclidean_space class constraints
huffman [Sun, 21 Aug 2011 09:46:20 -0700] rev 44360
section -> subsection
huffman [Sun, 21 Aug 2011 09:38:31 -0700] rev 44359
scale dependency graph to fit on page
wenzelm [Sun, 21 Aug 2011 21:24:42 +0200] rev 44358
more robust initialization of token marker and line context wrt. session startup;
wenzelm [Sun, 21 Aug 2011 20:42:26 +0200] rev 44357
tuned Parse.group: delayed failure message;
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;
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;
wenzelm [Sun, 21 Aug 2011 19:32:20 +0200] rev 44354
tuned;
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;
wenzelm [Sun, 21 Aug 2011 13:42:55 +0200] rev 44352
discontinued obsolete Thy_Syntax.report_span -- information can be reproduced in Isabelle/Scala;
wenzelm [Sun, 21 Aug 2011 13:36:23 +0200] rev 44351
merged
huffman [Sat, 20 Aug 2011 15:19:35 -0700] rev 44350
replace lemma realpow_two_diff with new lemma square_diff_square_factored
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
huffman [Sat, 20 Aug 2011 13:07:00 -0700] rev 44348
move lemma add_eq_0_iff to Groups.thy
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
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