Thu, 26 Mar 2009 15:18:50 +0100 wenzelm pretty_thm_aux etc.: explicit show_status flag;
Thu, 26 Mar 2009 14:14:02 +0100 wenzelm simplified attribute and method setup: eliminating bottom-up styles makes it easier to keep things in one place, and also SML/NJ happy;
Wed, 25 Mar 2009 21:35:49 +0100 wenzelm @{binding} is not a constructor term and should not be inlined, otherwise we loose value polymorphism;
Wed, 25 Mar 2009 21:34:31 +0100 wenzelm tuned;
Wed, 25 Mar 2009 17:23:44 +0100 wenzelm use more informative Thm.proof_body_of for oracle demo;
Wed, 25 Mar 2009 16:54:49 +0100 wenzelm Proofterm.approximate_proof_body;
Wed, 25 Mar 2009 16:54:17 +0100 wenzelm fulfill_proof/thm_proof: pass whole proof_body, not just the projection to proof (which might be incomplete);
Wed, 25 Mar 2009 16:52:50 +0100 wenzelm removed misleading make_proof_body, make_oracles, make_thms, which essentially assume a *full* proof;
Wed, 25 Mar 2009 14:47:08 +0100 wenzelm avoid mixing of left/right associative infixes, to make it work with experimental Poly/ML 5.3 branch;
Tue, 24 Mar 2009 23:43:58 +0100 wenzelm simplified addPrettyPrinter setup: may pass (fn ...) directly if type constraints are omitted -- addPrettyPrinter treated as a special case internally;
Tue, 24 Mar 2009 22:56:17 +0100 wenzelm status_of: need to include local promises as well!
Tue, 24 Mar 2009 22:55:49 +0100 wenzelm status_of: simultaneous list;
Tue, 24 Mar 2009 21:24:53 +0100 wenzelm display derivation status of thms;
Tue, 24 Mar 2009 19:37:50 +0100 wenzelm recover old ids;
Tue, 24 Mar 2009 18:21:58 +0100 wenzelm report ML typing;
Tue, 24 Mar 2009 16:11:42 +0100 wenzelm merged
Tue, 24 Mar 2009 14:09:24 +0100 nipkow merged
Tue, 24 Mar 2009 14:08:13 +0100 nipkow NEWS: [arith]
Tue, 24 Mar 2009 16:11:09 +0100 wenzelm get_index: produce index of next pending token, not the last one;
Tue, 24 Mar 2009 15:47:55 +0100 wenzelm register token positions persistently with context;
Tue, 24 Mar 2009 15:43:37 +0100 wenzelm tuned;
Tue, 24 Mar 2009 15:43:13 +0100 wenzelm more markup elements for ML programs;
Tue, 24 Mar 2009 13:20:40 +0100 wenzelm merged
Tue, 24 Mar 2009 13:12:23 +0100 wenzelm process at-sml-dev last -- takes very long (why?);
Tue, 24 Mar 2009 13:13:18 +0100 nipkow fix
Tue, 24 Mar 2009 12:45:23 +0100 nipkow merged
Tue, 24 Mar 2009 12:45:01 +0100 nipkow presburger uses [arith] now
Tue, 24 Mar 2009 12:01:12 +0100 wenzelm merged
Tue, 24 Mar 2009 09:15:59 +0100 haftmann merged
Tue, 24 Mar 2009 09:15:51 +0100 haftmann added Imperative_HOL_ex
Tue, 24 Mar 2009 15:55:11 +1100 Timothy Bourke Use assms rather than prems in find_theorems solves.
Mon, 23 Mar 2009 14:29:59 -0700 huffman clean up proofs of sign rules for multiplication; add list of lemmas mult_sign_intros
Mon, 23 Mar 2009 13:26:52 -0700 huffman lemmas add_sign_intros
Mon, 23 Mar 2009 19:01:34 +0100 haftmann merged
Mon, 23 Mar 2009 19:01:17 +0100 haftmann moved Imperative_HOL examples to Imperative_HOL/ex
Mon, 23 Mar 2009 19:01:17 +0100 haftmann corrected variable renaming
Mon, 23 Mar 2009 19:01:16 +0100 haftmann tuned error messages
Mon, 23 Mar 2009 19:01:16 +0100 haftmann moved generic arith_tac (formerly silent_arith_tac), verbose_arith_tac (formerly arith_tac) to Arith_Data; simple_arith-tac now named linear_arith_tac
Mon, 23 Mar 2009 19:01:15 +0100 haftmann structure LinArith now named Lin_Arith
Mon, 23 Mar 2009 19:01:15 +0100 haftmann suddenly infix identifier oo occurs in generated code
Tue, 24 Mar 2009 11:57:41 +0100 wenzelm datatype antiquote: maintain original Position.range, which is eventually attached to the resulting ML tokens;
Tue, 24 Mar 2009 11:39:25 +0100 wenzelm eliminated non-canonical alias structure T = ML_Lex;
Tue, 24 Mar 2009 00:36:32 +0100 wenzelm error "Static Errors";
Tue, 24 Mar 2009 00:30:52 +0100 wenzelm more systematic type use_context;
Mon, 23 Mar 2009 22:57:27 +0100 wenzelm tuned;
Mon, 23 Mar 2009 22:56:03 +0100 wenzelm more systematic type use_context;
Mon, 23 Mar 2009 22:38:02 +0100 wenzelm eliminated Output.ml_output;
Mon, 23 Mar 2009 22:37:41 +0100 wenzelm pretty_ml/ml_pretty: proper handling of markup and string length;
Mon, 23 Mar 2009 21:57:52 +0100 wenzelm more systematic type use_context;
Mon, 23 Mar 2009 21:40:12 +0100 wenzelm removed obsolete ml_output;
Mon, 23 Mar 2009 21:40:11 +0100 wenzelm more systematic type use_context;
Mon, 23 Mar 2009 21:40:11 +0100 wenzelm more systematic type use_context, with particular values ML_Parse.global_context and ML_Context.local_context;
Mon, 23 Mar 2009 21:40:11 +0100 wenzelm de-camelized ML_Name_Space;
Mon, 23 Mar 2009 17:21:42 +0100 wenzelm suppress status output for traditional tty modes (including Proof General);
Mon, 23 Mar 2009 17:20:31 +0100 wenzelm added report_text -- status messages with text body;
Mon, 23 Mar 2009 15:33:35 +0100 wenzelm maintain parse trees cumulatively;
Mon, 23 Mar 2009 15:23:06 +0100 wenzelm Block markup: maintain output version within tree values (in accordance with String) -- changes operational behaviour wrt. print_mode;
Mon, 23 Mar 2009 11:20:46 +0100 wenzelm future scheduler: reduced wait timeout if tasks need to be canceled -- to improve reactivity of interrupts;
Mon, 23 Mar 2009 08:16:24 +0100 haftmann merged
Mon, 23 Mar 2009 08:14:58 +0100 haftmann Main is (Complex_Main) base entry point in library theories
Mon, 23 Mar 2009 08:14:24 +0100 haftmann Main is (Complex_Main) base entry point in library theories
Mon, 23 Mar 2009 08:14:23 +0100 haftmann added instances for bot, top, wellorder
Mon, 23 Mar 2009 08:14:23 +0100 haftmann tuned header
Mon, 23 Mar 2009 08:14:22 +0100 haftmann more canonical import, syntax fix
Mon, 23 Mar 2009 07:41:07 +0100 haftmann merged
Sun, 22 Mar 2009 20:47:49 +0100 haftmann merged
Sun, 22 Mar 2009 20:46:12 +0100 haftmann more antiquotations
Sun, 22 Mar 2009 20:46:12 +0100 haftmann moved import of module qelim to theory Presburger
Sun, 22 Mar 2009 20:46:11 +0100 haftmann tuned header
Sun, 22 Mar 2009 20:46:11 +0100 haftmann dropped theory Arith_Tools
Sun, 22 Mar 2009 20:46:11 +0100 haftmann lemma nat_dvd_not_less moved here from Arith_Tools
Sun, 22 Mar 2009 20:46:10 +0100 haftmann distributed contents of theory Arith_Tools to theories Int, IntDiv and NatBin accordingly
Sun, 22 Mar 2009 21:48:14 +0100 wenzelm merged
Sun, 22 Mar 2009 19:43:21 +0100 nipkow merged
Sun, 22 Mar 2009 19:36:04 +0100 nipkow 1. New cancellation simprocs for common factors in inequations
Sun, 22 Mar 2009 11:56:32 +0100 haftmann clarified relationship of modules Code_Name and Code_Printer
Sun, 22 Mar 2009 11:56:22 +0100 haftmann added Symreltab (binary relations of symbols) instance of TableFun
Sun, 22 Mar 2009 21:30:21 +0100 wenzelm proper signature;
Sun, 22 Mar 2009 20:50:02 +0100 wenzelm added read_antiq, with improved error reporting;
Sun, 22 Mar 2009 20:49:48 +0100 wenzelm ML_Lex.read_antiq;
Sun, 22 Mar 2009 20:49:48 +0100 wenzelm ML_Lex.read_antiq;
Sun, 22 Mar 2009 20:49:47 +0100 wenzelm simplified Antiquote.read (again);
Sun, 22 Mar 2009 20:49:47 +0100 wenzelm export report -- version that actually covers all cases;
Sun, 22 Mar 2009 19:12:36 +0100 wenzelm Test of advanced ML compiler invocation in Poly/ML 5.3.
Sun, 22 Mar 2009 19:11:00 +0100 wenzelm ML/ml_test.ML: test of advanced ML compiler invocation in Poly/ML 5.3;
Sun, 22 Mar 2009 19:10:59 +0100 wenzelm added pretty_ml;
Sun, 22 Mar 2009 19:10:59 +0100 wenzelm export eval_antiquotes: refined version that operates on ML tokens;
Sun, 22 Mar 2009 19:10:59 +0100 wenzelm ML_Lex.pos_of: regular position;
Sun, 22 Mar 2009 19:10:58 +0100 wenzelm replaced Antiquote.is_antiq by Antiquote.is_text;
Sat, 21 Mar 2009 20:39:38 +0100 wenzelm merged
Sat, 21 Mar 2009 20:38:49 +0100 wenzelm extra toplevel pretty-printing for Poly/ML; experimental version for Poly/ML 5.3;
Sat, 21 Mar 2009 20:22:13 +0100 wenzelm merged
Sat, 21 Mar 2009 09:42:55 -0700 huffman merged
Sat, 21 Mar 2009 03:24:35 -0700 huffman move field lemmas into class locale context
Sat, 21 Mar 2009 03:23:17 -0700 huffman move diff_eq_0_iff_eq into class locale context
Sat, 21 Mar 2009 20:00:23 +0100 wenzelm removed obsolete pprint operations;
Sat, 21 Mar 2009 20:00:23 +0100 wenzelm added polyml_pp.ML: toplevel pretty printing for Poly/ML 4.x and 5.x before 5.3;
Sat, 21 Mar 2009 19:58:45 +0100 wenzelm adapted toplevel_pp to ML_Pretty.pretty;
Sat, 21 Mar 2009 19:58:45 +0100 wenzelm replaced install_pp/make_pp by more general toplevel_pp based on use_text;
Sat, 21 Mar 2009 19:58:45 +0100 wenzelm simplified datatype ML_Pretty.pretty: model Isabelle not Poly/ML;
Sat, 21 Mar 2009 19:58:44 +0100 wenzelm simplified datatype ML_Pretty.pretty: model Isabelle not Poly/ML;
Sat, 21 Mar 2009 15:09:44 +0100 wenzelm Datatype for ML pretty printing (cf. mlsource/MLCompiler/Pretty.sml in Poly/ML 5.3).
Sat, 21 Mar 2009 15:08:00 +0100 wenzelm Pretty.position;
Sat, 21 Mar 2009 15:08:00 +0100 wenzelm added position;
Sat, 21 Mar 2009 15:08:00 +0100 wenzelm added generic ML_Pretty interface;
Sat, 21 Mar 2009 13:11:12 +0100 wenzelm restricted interrupts for tasks running as future worker thread -- attempt to prevent interrupt race conditions;
Sat, 21 Mar 2009 12:37:13 +0100 wenzelm more ambitious ML_OPTIONS;
Sat, 21 Mar 2009 12:35:34 +0100 wenzelm more stats;
Fri, 20 Mar 2009 21:32:12 +0100 wenzelm added ML syntax markup;
Fri, 20 Mar 2009 20:22:13 +0100 wenzelm report markup for ML tokens;
Fri, 20 Mar 2009 20:21:38 +0100 wenzelm Antiquote.read: argument for reporting text;
Fri, 20 Mar 2009 20:20:09 +0100 wenzelm future_job: do not inherit attributes, but enforce restricted interrupts -- attempt to prevent interrupt race conditions;
(0) -30000 -10000 -3000 -1000 -112 +112 +1000 +3000 +10000 +30000 tip