Wed, 27 Mar 2013 16:46:52 +0100 separate option editor_skip_proofs, to avoid accidental change of preferences for skip_proofs, which would invalidate batch builds;
wenzelm [Wed, 27 Mar 2013 16:46:52 +0100] rev 51554
separate option editor_skip_proofs, to avoid accidental change of preferences for skip_proofs, which would invalidate batch builds;
Wed, 27 Mar 2013 16:38:25 +0100 more ambitious Goal.skip_proofs: covers Goal.prove forms as well, and do not insist in quick_and_dirty (for the sake of Isabelle/jEdit);
wenzelm [Wed, 27 Mar 2013 16:38:25 +0100] rev 51553
more ambitious Goal.skip_proofs: covers Goal.prove forms as well, and do not insist in quick_and_dirty (for the sake of Isabelle/jEdit);
Wed, 27 Mar 2013 14:50:30 +0100 clarified Skip_Proof.cheat_tac: more standard tactic;
wenzelm [Wed, 27 Mar 2013 14:50:30 +0100] rev 51552
clarified Skip_Proof.cheat_tac: more standard tactic; clarified Method.cheating: check quick_and_dirty when it is actually applied;
Wed, 27 Mar 2013 14:19:18 +0100 tuned signature and module arrangement;
wenzelm [Wed, 27 Mar 2013 14:19:18 +0100] rev 51551
tuned signature and module arrangement;
Wed, 27 Mar 2013 14:08:03 +0100 tuned;
wenzelm [Wed, 27 Mar 2013 14:08:03 +0100] rev 51550
tuned;
Wed, 27 Mar 2013 11:54:53 +0100 tuned GUI;
wenzelm [Wed, 27 Mar 2013 11:54:53 +0100] rev 51549
tuned GUI;
Wed, 27 Mar 2013 10:55:05 +0100 centralized various multiset operations in theory multiset;
haftmann [Wed, 27 Mar 2013 10:55:05 +0100] rev 51548
centralized various multiset operations in theory multiset; more conversions between multisets and lists respectively
Tue, 26 Mar 2013 22:09:39 +0100 avoid odd foundational terms after interpretation;
haftmann [Tue, 26 Mar 2013 22:09:39 +0100] rev 51547
avoid odd foundational terms after interpretation; more uniform code setup
Tue, 26 Mar 2013 21:53:56 +0100 more uniform style for interpretation and sublocale declarations
haftmann [Tue, 26 Mar 2013 21:53:56 +0100] rev 51546
more uniform style for interpretation and sublocale declarations
Tue, 26 Mar 2013 20:55:21 +0100 merged
wenzelm [Tue, 26 Mar 2013 20:55:21 +0100] rev 51545
merged
Tue, 26 Mar 2013 20:37:32 +0100 tuned session specification;
wenzelm [Tue, 26 Mar 2013 20:37:32 +0100] rev 51544
tuned session specification;
Tue, 26 Mar 2013 20:36:32 +0100 tuned proof;
wenzelm [Tue, 26 Mar 2013 20:36:32 +0100] rev 51543
tuned proof;
Tue, 26 Mar 2013 20:02:02 +0100 tuned imports;
wenzelm [Tue, 26 Mar 2013 20:02:02 +0100] rev 51542
tuned imports;
Tue, 26 Mar 2013 19:43:31 +0100 tuned proofs;
wenzelm [Tue, 26 Mar 2013 19:43:31 +0100] rev 51541
tuned proofs;
Tue, 26 Mar 2013 20:49:57 +0100 explicit sublocale dependency for Min/Max yields more appropriate Min/Max prefix for a couple of facts
haftmann [Tue, 26 Mar 2013 20:49:57 +0100] rev 51540
explicit sublocale dependency for Min/Max yields more appropriate Min/Max prefix for a couple of facts
Tue, 26 Mar 2013 15:10:28 +0100 merged
wenzelm [Tue, 26 Mar 2013 15:10:28 +0100] rev 51539
merged
Tue, 26 Mar 2013 14:38:44 +0100 proper input event handling;
wenzelm [Tue, 26 Mar 2013 14:38:44 +0100] rev 51538
proper input event handling;
Tue, 26 Mar 2013 14:14:39 +0100 more standard imports;
wenzelm [Tue, 26 Mar 2013 14:14:39 +0100] rev 51537
more standard imports;
Tue, 26 Mar 2013 14:05:08 +0100 more specific Entry painting;
wenzelm [Tue, 26 Mar 2013 14:05:08 +0100] rev 51536
more specific Entry painting; ignore theories with all commands below threshold;
Tue, 26 Mar 2013 14:03:31 +0100 tuned;
wenzelm [Tue, 26 Mar 2013 14:03:31 +0100] rev 51535
tuned;
Tue, 26 Mar 2013 12:40:51 +0100 mixed theory/command entries;
wenzelm [Tue, 26 Mar 2013 12:40:51 +0100] rev 51534
mixed theory/command entries; tuned;
Tue, 26 Mar 2013 11:26:13 +0100 dockable window for timing information;
wenzelm [Tue, 26 Mar 2013 11:26:13 +0100] rev 51533
dockable window for timing information;
Tue, 26 Mar 2013 13:54:24 +0100 no \FIXME macro for ProgProve (moved to book)
kleing [Tue, 26 Mar 2013 13:54:24 +0100] rev 51532
no \FIXME macro for ProgProve (moved to book)
Tue, 26 Mar 2013 12:21:01 +0100 remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
hoelzl [Tue, 26 Mar 2013 12:21:01 +0100] rev 51531
remove Metric_Spaces and move its content into Limits and Real_Vector_Spaces
Tue, 26 Mar 2013 12:21:00 +0100 rename eventually_at / _within, to distinguish them from the lemmas in the HOL image
hoelzl [Tue, 26 Mar 2013 12:21:00 +0100] rev 51530
rename eventually_at / _within, to distinguish them from the lemmas in the HOL image
Tue, 26 Mar 2013 12:21:00 +0100 move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
hoelzl [Tue, 26 Mar 2013 12:21:00 +0100] rev 51529
move theorems about compactness of real closed intervals, the intermediate value theorem, and lemmas about continuity of bijective functions from Deriv.thy to Limits.thy
Tue, 26 Mar 2013 12:20:59 +0100 Series.thy is based on Limits.thy and not Deriv.thy
hoelzl [Tue, 26 Mar 2013 12:20:59 +0100] rev 51528
Series.thy is based on Limits.thy and not Deriv.thy
Tue, 26 Mar 2013 12:20:59 +0100 move Ln.thy and Log.thy to Transcendental.thy
hoelzl [Tue, 26 Mar 2013 12:20:59 +0100] rev 51527
move Ln.thy and Log.thy to Transcendental.thy
Tue, 26 Mar 2013 12:20:58 +0100 move SEQ.thy and Lim.thy to Limits.thy
hoelzl [Tue, 26 Mar 2013 12:20:58 +0100] rev 51526
move SEQ.thy and Lim.thy to Limits.thy
Tue, 26 Mar 2013 12:20:58 +0100 HOL-NSA should only import Complex_Main
hoelzl [Tue, 26 Mar 2013 12:20:58 +0100] rev 51525
HOL-NSA should only import Complex_Main
(0) -30000 -10000 -3000 -1000 -300 -100 -50 -30 +30 +50 +100 +300 +1000 +3000 +10000 tip