Fri, 08 Oct 2010 17:41:51 +0100 eliminated fancy \ML logo for the sake of simpler source text (less dependence on LaTeX);
wenzelm [Fri, 08 Oct 2010 17:41:51 +0100] rev 39825
eliminated fancy \ML logo for the sake of simpler source text (less dependence on LaTeX); eliminated Isar toplevel invocation functions, which belong to TTY/ProofGeneral model; moved remaining "ML toplevel" material to "Compile-time context";
Fri, 08 Oct 2010 16:50:01 +0100 misc tuning;
wenzelm [Fri, 08 Oct 2010 16:50:01 +0100] rev 39824
misc tuning;
Thu, 07 Oct 2010 21:24:18 +0100 more on Isabelle/ML;
wenzelm [Thu, 07 Oct 2010 21:24:18 +0100] rev 39823
more on Isabelle/ML;
Thu, 07 Oct 2010 19:05:42 +0100 basic setup for Chapter 0: Isabelle/ML;
wenzelm [Thu, 07 Oct 2010 19:05:42 +0100] rev 39822
basic setup for Chapter 0: Isabelle/ML;
Thu, 07 Oct 2010 12:39:01 +0100 minor tuning and updating;
wenzelm [Thu, 07 Oct 2010 12:39:01 +0100] rev 39821
minor tuning and updating;
Fri, 01 Oct 2010 17:23:26 +0200 made SML/NJ happy;
wenzelm [Fri, 01 Oct 2010 17:23:26 +0200] rev 39820
made SML/NJ happy;
Fri, 01 Oct 2010 16:44:13 +0200 merged
wenzelm [Fri, 01 Oct 2010 16:44:13 +0200] rev 39819
merged
Fri, 01 Oct 2010 14:15:49 +0200 use module integer for Eval
haftmann [Fri, 01 Oct 2010 14:15:49 +0200] rev 39818
use module integer for Eval
Fri, 01 Oct 2010 11:46:09 +0200 check whole target hierarchy for existing reserved symbols
haftmann [Fri, 01 Oct 2010 11:46:09 +0200] rev 39817
check whole target hierarchy for existing reserved symbols
Fri, 01 Oct 2010 11:46:09 +0200 added polyml_as_definition -- using external SML files as substitute for proper definitions -- only for polyml!
haftmann [Fri, 01 Oct 2010 11:46:09 +0200] rev 39816
added polyml_as_definition -- using external SML files as substitute for proper definitions -- only for polyml!
Fri, 01 Oct 2010 15:11:15 +0200 tuned default "Prover Session" perspective;
wenzelm [Fri, 01 Oct 2010 15:11:15 +0200] rev 39815
tuned default "Prover Session" perspective;
Fri, 01 Oct 2010 14:47:46 +0200 eliminated ancient OldTerm.term_frees;
wenzelm [Fri, 01 Oct 2010 14:47:46 +0200] rev 39814
eliminated ancient OldTerm.term_frees;
Fri, 01 Oct 2010 14:27:51 +0200 more antiquotations;
wenzelm [Fri, 01 Oct 2010 14:27:51 +0200] rev 39813
more antiquotations;
Fri, 01 Oct 2010 13:36:35 +0200 simplified outer syntax setup;
wenzelm [Fri, 01 Oct 2010 13:36:35 +0200] rev 39812
simplified outer syntax setup; slightly more uniform Isabelle/ML indentation style;
Fri, 01 Oct 2010 10:25:36 +0200 chop_while replace drop_while and take_while
haftmann [Fri, 01 Oct 2010 10:25:36 +0200] rev 39811
chop_while replace drop_while and take_while
Fri, 01 Oct 2010 08:25:23 +0200 merged
haftmann [Fri, 01 Oct 2010 08:25:23 +0200] rev 39810
merged
Thu, 30 Sep 2010 18:37:29 +0200 take_while, drop_while
haftmann [Thu, 30 Sep 2010 18:37:29 +0200] rev 39809
take_while, drop_while
Thu, 30 Sep 2010 18:46:19 -0700 rename cont2cont_split to cont2cont_prod_case; add lemmas prod_contI, prod_cont_iff; simplify some proofs
huffman [Thu, 30 Sep 2010 18:46:19 -0700] rev 39808
rename cont2cont_split to cont2cont_prod_case; add lemmas prod_contI, prod_cont_iff; simplify some proofs
Thu, 30 Sep 2010 17:06:25 -0700 fixrec: rename match_cpair to match_Pair
huffman [Thu, 30 Sep 2010 17:06:25 -0700] rev 39807
fixrec: rename match_cpair to match_Pair
Wed, 15 Sep 2010 13:26:21 -0700 remove code for obsolete 'fixpat' command
huffman [Wed, 15 Sep 2010 13:26:21 -0700] rev 39806
remove code for obsolete 'fixpat' command
Wed, 15 Sep 2010 12:54:17 -0700 clean up definition of compile_pat function
huffman [Wed, 15 Sep 2010 12:54:17 -0700] rev 39805
clean up definition of compile_pat function
Wed, 15 Sep 2010 10:34:39 -0700 rename some fixrec pattern-match compilation functions
huffman [Wed, 15 Sep 2010 10:34:39 -0700] rev 39804
rename some fixrec pattern-match compilation functions
Thu, 30 Sep 2010 15:37:12 +0200 adding example for case expressions
bulwahn [Thu, 30 Sep 2010 15:37:12 +0200] rev 39803
adding example for case expressions
Thu, 30 Sep 2010 15:37:11 +0200 applying case beta reduction to case term before matching in predicate compile function flattening; moving case beta reduction function to Predicate_Compile_Aux
bulwahn [Thu, 30 Sep 2010 15:37:11 +0200] rev 39802
applying case beta reduction to case term before matching in predicate compile function flattening; moving case beta reduction function to Predicate_Compile_Aux
Thu, 30 Sep 2010 11:52:22 +0200 merged
bulwahn [Thu, 30 Sep 2010 11:52:22 +0200] rev 39801
merged
Thu, 30 Sep 2010 10:48:12 +0200 adapting manual configuration in examples
bulwahn [Thu, 30 Sep 2010 10:48:12 +0200] rev 39800
adapting manual configuration in examples
Thu, 30 Sep 2010 10:48:12 +0200 finding the counterexample with different options (manually limited precisely, manually limited global, automatically limited global)
bulwahn [Thu, 30 Sep 2010 10:48:12 +0200] rev 39799
finding the counterexample with different options (manually limited precisely, manually limited global, automatically limited global)
Thu, 30 Sep 2010 10:48:11 +0200 adding option to globally limit the prolog execution
bulwahn [Thu, 30 Sep 2010 10:48:11 +0200] rev 39798
adding option to globally limit the prolog execution
Thu, 30 Sep 2010 10:48:09 +0200 removing dead code
bulwahn [Thu, 30 Sep 2010 10:48:09 +0200] rev 39797
removing dead code
Thu, 30 Sep 2010 09:45:18 +0200 value uses bare compiler invocation: generated code does not contain antiquotations
haftmann [Thu, 30 Sep 2010 09:45:18 +0200] rev 39796
value uses bare compiler invocation: generated code does not contain antiquotations
Thu, 30 Sep 2010 09:31:07 +0200 updated files to recent changes
haftmann [Thu, 30 Sep 2010 09:31:07 +0200] rev 39795
updated files to recent changes
Thu, 30 Sep 2010 08:50:45 +0200 corrected subsumption check: arguments have been reversed; addition of default equations to non-default equations is identity
haftmann [Thu, 30 Sep 2010 08:50:45 +0200] rev 39794
corrected subsumption check: arguments have been reversed; addition of default equations to non-default equations is identity
Thu, 30 Sep 2010 08:50:45 +0200 tuned
haftmann [Thu, 30 Sep 2010 08:50:45 +0200] rev 39793
tuned
Thu, 30 Sep 2010 07:34:06 +0200 merged
haftmann [Thu, 30 Sep 2010 07:34:06 +0200] rev 39792
merged
Wed, 29 Sep 2010 15:28:29 +0200 redundancy check: drop trailing Var arguments (avoids eta problems with equations)
haftmann [Wed, 29 Sep 2010 15:28:29 +0200] rev 39791
redundancy check: drop trailing Var arguments (avoids eta problems with equations)
Wed, 29 Sep 2010 17:59:20 +0200 merged
wenzelm [Wed, 29 Sep 2010 17:59:20 +0200] rev 39790
merged
Wed, 29 Sep 2010 11:55:08 +0200 removing obsolete distinction between prod_case and other case expressions after merging of split and prod_case (d3daea901123) in predicate compiler
bulwahn [Wed, 29 Sep 2010 11:55:08 +0200] rev 39789
removing obsolete distinction between prod_case and other case expressions after merging of split and prod_case (d3daea901123) in predicate compiler
Wed, 29 Sep 2010 11:36:16 +0200 merged
bulwahn [Wed, 29 Sep 2010 11:36:16 +0200] rev 39788
merged
Wed, 29 Sep 2010 10:33:15 +0200 adding splitting of conjuncts in assumptions as forward rule on theorems; replacing term transformation for splitting conjuncts by theorem transformation; removing obsolete functions; tuned
bulwahn [Wed, 29 Sep 2010 10:33:15 +0200] rev 39787
adding splitting of conjuncts in assumptions as forward rule on theorems; replacing term transformation for splitting conjuncts by theorem transformation; removing obsolete functions; tuned
Wed, 29 Sep 2010 10:33:15 +0200 added test case for predicate arguments in higher-order argument position
bulwahn [Wed, 29 Sep 2010 10:33:15 +0200] rev 39786
added test case for predicate arguments in higher-order argument position
Wed, 29 Sep 2010 10:33:15 +0200 improving the compilation to handle predicate arguments in higher-order argument positions
bulwahn [Wed, 29 Sep 2010 10:33:15 +0200] rev 39785
improving the compilation to handle predicate arguments in higher-order argument positions
Wed, 29 Sep 2010 10:33:15 +0200 added a test case to Predicate_Compile_Tests
bulwahn [Wed, 29 Sep 2010 10:33:15 +0200] rev 39784
added a test case to Predicate_Compile_Tests
Wed, 29 Sep 2010 10:33:14 +0200 putting the last step of the proof in a TRY block to handle the case that the simplifier already solved the goal
bulwahn [Wed, 29 Sep 2010 10:33:14 +0200] rev 39783
putting the last step of the proof in a TRY block to handle the case that the simplifier already solved the goal
Wed, 29 Sep 2010 11:02:24 +0200 backed out my old attempt at single_hyp_subst_tac (67cd6ed76446)
krauss [Wed, 29 Sep 2010 11:02:24 +0200] rev 39782
backed out my old attempt at single_hyp_subst_tac (67cd6ed76446) It never was totally reliable, and better alternatives now exist (Subgoal.FOCUS).
Wed, 29 Sep 2010 10:05:44 +0200 scala is reserved identifier
haftmann [Wed, 29 Sep 2010 10:05:44 +0200] rev 39781
scala is reserved identifier
Wed, 29 Sep 2010 09:21:26 +0200 platform-sensitive contrib paths for ghc, ocaml
haftmann [Wed, 29 Sep 2010 09:21:26 +0200] rev 39780
platform-sensitive contrib paths for ghc, ocaml
Wed, 29 Sep 2010 09:08:01 +0200 fact listsum now names listsum_foldl
haftmann [Wed, 29 Sep 2010 09:08:01 +0200] rev 39779
fact listsum now names listsum_foldl
Wed, 29 Sep 2010 09:08:00 +0200 delete code lemma explicitly
haftmann [Wed, 29 Sep 2010 09:08:00 +0200] rev 39778
delete code lemma explicitly
Wed, 29 Sep 2010 09:07:58 +0200 moved old_primrec source to nominal package, where it is still used
haftmann [Wed, 29 Sep 2010 09:07:58 +0200] rev 39777
moved old_primrec source to nominal package, where it is still used
Tue, 28 Sep 2010 15:39:59 +0200 dropped old primrec package
haftmann [Tue, 28 Sep 2010 15:39:59 +0200] rev 39776
dropped old primrec package
Tue, 28 Sep 2010 15:34:47 +0200 merged
haftmann [Tue, 28 Sep 2010 15:34:47 +0200] rev 39775
merged
Tue, 28 Sep 2010 15:21:45 +0200 localized listsum
haftmann [Tue, 28 Sep 2010 15:21:45 +0200] rev 39774
localized listsum
Tue, 28 Sep 2010 15:21:45 +0200 lemma listsum_conv_fold
haftmann [Tue, 28 Sep 2010 15:21:45 +0200] rev 39773
lemma listsum_conv_fold
Tue, 28 Sep 2010 15:34:30 +0200 merged
haftmann [Tue, 28 Sep 2010 15:34:30 +0200] rev 39772
merged
Tue, 28 Sep 2010 15:33:56 +0200 NEWS
haftmann [Tue, 28 Sep 2010 15:33:56 +0200] rev 39771
NEWS
Tue, 28 Sep 2010 15:32:59 +0200 dropped syntax for old primrec package
haftmann [Tue, 28 Sep 2010 15:32:59 +0200] rev 39770
dropped syntax for old primrec package
Tue, 28 Sep 2010 15:31:10 +0200 modernized session
haftmann [Tue, 28 Sep 2010 15:31:10 +0200] rev 39769
modernized session
Tue, 28 Sep 2010 13:44:06 +0200 merged
bulwahn [Tue, 28 Sep 2010 13:44:06 +0200] rev 39768
merged
Tue, 28 Sep 2010 11:59:58 +0200 using SUBPROOF to ensure that rewriting is not done on the further subgoals of proof
bulwahn [Tue, 28 Sep 2010 11:59:58 +0200] rev 39767
using SUBPROOF to ensure that rewriting is not done on the further subgoals of proof
Tue, 28 Sep 2010 11:59:57 +0200 avoiding instable rotate_tac and using the nice Subgoal.FOCUS_PREMS instead
bulwahn [Tue, 28 Sep 2010 11:59:57 +0200] rev 39766
avoiding instable rotate_tac and using the nice Subgoal.FOCUS_PREMS instead
Tue, 28 Sep 2010 11:59:53 +0200 adding test case for interpretation of arguments that are predicates simply as input
bulwahn [Tue, 28 Sep 2010 11:59:53 +0200] rev 39765
adding test case for interpretation of arguments that are predicates simply as input
Tue, 28 Sep 2010 11:59:52 +0200 only modes but not types are used to destruct terms and types; this allows to interpret arguments that are predicates simply as input
bulwahn [Tue, 28 Sep 2010 11:59:52 +0200] rev 39764
only modes but not types are used to destruct terms and types; this allows to interpret arguments that are predicates simply as input
Tue, 28 Sep 2010 11:59:51 +0200 weakening check for higher-order relations, but adding check for consistent modes
bulwahn [Tue, 28 Sep 2010 11:59:51 +0200] rev 39763
weakening check for higher-order relations, but adding check for consistent modes
Tue, 28 Sep 2010 11:59:51 +0200 handling higher-order relations in output terms; improving proof procedure; added test case
bulwahn [Tue, 28 Sep 2010 11:59:51 +0200] rev 39762
handling higher-order relations in output terms; improving proof procedure; added test case
Tue, 28 Sep 2010 11:59:50 +0200 renaming use_random to use_generators in the predicate compiler
bulwahn [Tue, 28 Sep 2010 11:59:50 +0200] rev 39761
renaming use_random to use_generators in the predicate compiler
Tue, 28 Sep 2010 11:59:48 +0200 fixed a typo that caused the preference of non-random modes to be ignored
bulwahn [Tue, 28 Sep 2010 11:59:48 +0200] rev 39760
fixed a typo that caused the preference of non-random modes to be ignored
Tue, 28 Sep 2010 12:48:05 +0200 merged
haftmann [Tue, 28 Sep 2010 12:48:05 +0200] rev 39759
merged
Tue, 28 Sep 2010 12:47:55 +0200 modernized primrecs
haftmann [Tue, 28 Sep 2010 12:47:55 +0200] rev 39758
modernized primrecs
Tue, 28 Sep 2010 12:47:55 +0200 modernized session
haftmann [Tue, 28 Sep 2010 12:47:55 +0200] rev 39757
modernized session
Tue, 28 Sep 2010 12:34:41 +0200 consolidated tupled_lambda; moved to structure HOLogic
krauss [Tue, 28 Sep 2010 12:34:41 +0200] rev 39756
consolidated tupled_lambda; moved to structure HOLogic
Tue, 28 Sep 2010 12:10:37 +0200 added dependency to base image to ensure that the doc test actually rebuilds the tutorial
haftmann [Tue, 28 Sep 2010 12:10:37 +0200] rev 39755
added dependency to base image to ensure that the doc test actually rebuilds the tutorial
Tue, 28 Sep 2010 09:54:07 +0200 no longer declare .psimps rules as [simp].
krauss [Tue, 28 Sep 2010 09:54:07 +0200] rev 39754
no longer declare .psimps rules as [simp]. This regularly caused confusion (e.g., they show up in simp traces when the regular simp rules are disabled). In the few places where the rules are used, explicitly mentioning them actually clarifies the proof text.
Tue, 28 Sep 2010 09:43:13 +0200 added dependency to base images to ensure that the doc test actually rebuilds the tutorials
krauss [Tue, 28 Sep 2010 09:43:13 +0200] rev 39753
added dependency to base images to ensure that the doc test actually rebuilds the tutorials
Tue, 28 Sep 2010 09:34:20 +0200 removed unnecessary reference poking (cf. f45d332a90e3)
krauss [Tue, 28 Sep 2010 09:34:20 +0200] rev 39752
removed unnecessary reference poking (cf. f45d332a90e3)
Tue, 28 Sep 2010 09:17:33 +0200 merged
haftmann [Tue, 28 Sep 2010 09:17:33 +0200] rev 39751
merged
Tue, 28 Sep 2010 09:14:37 +0200 consider quick_and_dirty option before loading theory
haftmann [Tue, 28 Sep 2010 09:14:37 +0200] rev 39750
consider quick_and_dirty option before loading theory
Tue, 28 Sep 2010 08:38:20 +0200 dropped obsolete mk_tcl
krauss [Tue, 28 Sep 2010 08:38:20 +0200] rev 39749
dropped obsolete mk_tcl
Tue, 28 Sep 2010 08:35:00 +0200 make SML/NJ happy
blanchet [Tue, 28 Sep 2010 08:35:00 +0200] rev 39748
make SML/NJ happy
Mon, 27 Sep 2010 16:32:48 +0200 merged
haftmann [Mon, 27 Sep 2010 16:32:48 +0200] rev 39747
merged
Mon, 27 Sep 2010 16:27:32 +0200 combine quote and typewriter tag; typewriter considers isa@parindent
haftmann [Mon, 27 Sep 2010 16:27:32 +0200] rev 39746
combine quote and typewriter tag; typewriter considers isa@parindent
Mon, 27 Sep 2010 16:27:31 +0200 combine quote and typewriter/tt tag
haftmann [Mon, 27 Sep 2010 16:27:31 +0200] rev 39745
combine quote and typewriter/tt tag
Mon, 27 Sep 2010 16:19:37 +0200 combine quote and typewriter tag; typewriter considers isa@parindent
haftmann [Mon, 27 Sep 2010 16:19:37 +0200] rev 39744
combine quote and typewriter tag; typewriter considers isa@parindent
Mon, 27 Sep 2010 16:19:36 +0200 combine quote and typewriter tag
haftmann [Mon, 27 Sep 2010 16:19:36 +0200] rev 39743
combine quote and typewriter tag
Wed, 29 Sep 2010 17:58:27 +0200 CONTROL-mouse management: handle windowDeactivated as well;
wenzelm [Wed, 29 Sep 2010 17:58:27 +0200] rev 39742
CONTROL-mouse management: handle windowDeactivated as well; some workarounds to robustify html_popup;
Tue, 28 Sep 2010 23:47:45 +0200 CONTROL-mouse management: handle windowIconified;
wenzelm [Tue, 28 Sep 2010 23:47:45 +0200] rev 39741
CONTROL-mouse management: handle windowIconified; html_panel: tuned border;
Tue, 28 Sep 2010 23:02:05 +0200 basic support for message popups via HTML_Panel;
wenzelm [Tue, 28 Sep 2010 23:02:05 +0200] rev 39740
basic support for message popups via HTML_Panel; more systematic CONTROL-mouse management; tuned;
Tue, 28 Sep 2010 20:49:39 +0200 tuned default perspective;
wenzelm [Tue, 28 Sep 2010 20:49:39 +0200] rev 39739
tuned default perspective;
Tue, 28 Sep 2010 20:35:17 +0200 tuned README;
wenzelm [Tue, 28 Sep 2010 20:35:17 +0200] rev 39738
tuned README;
Tue, 28 Sep 2010 20:22:58 +0200 more defensive overview.paintComponent: avoid potential crash due to buffer change while painting;
wenzelm [Tue, 28 Sep 2010 20:22:58 +0200] rev 39737
more defensive overview.paintComponent: avoid potential crash due to buffer change while painting;
Tue, 28 Sep 2010 18:51:10 +0200 tuned README;
wenzelm [Tue, 28 Sep 2010 18:51:10 +0200] rev 39736
tuned README;
Tue, 28 Sep 2010 15:58:31 +0200 more uniform init/exit model/view in session_manager, trading race wrt. session.phase for race wrt. global editor state;
wenzelm [Tue, 28 Sep 2010 15:58:31 +0200] rev 39735
more uniform init/exit model/view in session_manager, trading race wrt. session.phase for race wrt. global editor state;
Mon, 27 Sep 2010 21:16:42 +0200 moved "auto-start" to options panel;
wenzelm [Mon, 27 Sep 2010 21:16:42 +0200] rev 39734
moved "auto-start" to options panel; tuned;
Mon, 27 Sep 2010 20:26:10 +0200 renamed raw output primitives to emphasize their meaning -- not to be used in user-space;
wenzelm [Mon, 27 Sep 2010 20:26:10 +0200] rev 39733
renamed raw output primitives to emphasize their meaning -- not to be used in user-space;
Mon, 27 Sep 2010 18:16:36 +0200 added Standard_System.unzip (for platform file-system);
wenzelm [Mon, 27 Sep 2010 18:16:36 +0200] rev 39732
added Standard_System.unzip (for platform file-system); tuned comments;
Mon, 27 Sep 2010 18:11:33 +0200 bulk read: observe EOF protocol more carefully -- 0 counts as successful read;
wenzelm [Mon, 27 Sep 2010 18:11:33 +0200] rev 39731
bulk read: observe EOF protocol more carefully -- 0 counts as successful read;
Mon, 27 Sep 2010 18:10:21 +0200 tuned whitespace;
wenzelm [Mon, 27 Sep 2010 18:10:21 +0200] rev 39730
tuned whitespace;
(0) -30000 -10000 -3000 -1000 -300 -100 -96 +96 +100 +300 +1000 +3000 +10000 +30000 tip