Sun, 29 Mar 2009 16:13:24 +0200 wenzelm simplified roundup activation interface;
Sat, 28 Mar 2009 20:52:52 +0100 wenzelm merged
Sat, 28 Mar 2009 18:18:01 +0100 haftmann merged
Sat, 28 Mar 2009 18:17:44 +0100 haftmann merged
Sat, 28 Mar 2009 18:17:21 +0100 haftmann second attempt for code_deps command
Sat, 28 Mar 2009 16:33:32 +0100 haftmann merged
Sat, 28 Mar 2009 16:29:39 +0100 haftmann corrected projection of required statement names
Sat, 28 Mar 2009 16:29:38 +0100 haftmann corrected check for additional type variables on rhs of code equations
Sat, 28 Mar 2009 16:29:37 +0100 haftmann not yet fruitful tex experiments with bounding boxes
Sat, 28 Mar 2009 20:25:23 +0100 wenzelm simplified Locale.activate operations, using generic context;
Sat, 28 Mar 2009 17:53:33 +0100 wenzelm renamed ProofContext.add_fixes_i to ProofContext.add_fixes, eliminated obsolete external version;
Sat, 28 Mar 2009 17:21:49 +0100 wenzelm define_prefs: removed redundant Drule.gen_all, which is already part of the norm_hhf stage of Assumption.assume;
Sat, 28 Mar 2009 17:21:11 +0100 wenzelm renamed ProofContext.note_thmss_i to ProofContext.note_thmss, eliminated obsolete external version;
Sat, 28 Mar 2009 17:10:43 +0100 wenzelm simplified references to facts, eliminated external note_thmss;
Sat, 28 Mar 2009 17:08:49 +0100 wenzelm added map_facts_refs;
Sat, 28 Mar 2009 17:08:18 +0100 wenzelm tuned;
Sat, 28 Mar 2009 16:31:16 +0100 wenzelm replaced add_binds(_i) by bind_terms -- internal version only;
Sat, 28 Mar 2009 16:30:09 +0100 wenzelm replaced add_binds by singleton bind_term;
Sat, 28 Mar 2009 16:00:54 +0100 wenzelm simplified internal locale parameters: maintain proper name and type, instead of binding and constraint;
Sat, 28 Mar 2009 12:48:31 +0100 wenzelm minor tuning;
Sat, 28 Mar 2009 12:26:21 +0100 wenzelm merged
Sat, 28 Mar 2009 00:13:01 +0100 ballarin Merged.
Sat, 28 Mar 2009 00:11:02 +0100 ballarin Corrections to locale syntax.
Fri, 27 Mar 2009 23:43:48 +0100 ballarin Update explanation of locale expressions to locale reimplementation.
Fri, 27 Mar 2009 20:25:07 +0100 ballarin Comments updated.
Fri, 27 Mar 2009 17:35:21 +0000 chaieb fixed proof
Fri, 27 Mar 2009 14:44:18 +0000 chaieb merged
Fri, 27 Mar 2009 14:43:47 +0000 chaieb fps made instance of number_ring
Fri, 27 Mar 2009 21:46:20 +0100 wenzelm updated keywords with polyml-experimental;
Fri, 27 Mar 2009 15:42:53 +0100 wenzelm export position_of;
Fri, 27 Mar 2009 12:22:02 +0100 haftmann dropped infix union
Fri, 27 Mar 2009 12:22:01 +0100 haftmann tuned notoriously slow metis proof
Fri, 27 Mar 2009 10:12:55 +0100 haftmann merged
Fri, 27 Mar 2009 10:05:13 +0100 haftmann dropped toy example Code_Antiq
Fri, 27 Mar 2009 10:05:12 +0100 haftmann more convenient name uniqueness
Fri, 27 Mar 2009 10:05:11 +0100 haftmann normalized imports
Fri, 27 Mar 2009 10:05:08 +0100 haftmann dropped legacy goal package call
Fri, 27 Mar 2009 09:58:48 +0100 haftmann merged
Thu, 26 Mar 2009 13:02:12 +0100 haftmann merged
Thu, 26 Mar 2009 13:01:09 +0100 haftmann step towards proper pictures in dvi
Thu, 26 Mar 2009 20:09:58 +0100 wenzelm merged
Thu, 26 Mar 2009 11:33:50 -0700 huffman parameterize assoc_fold with is_numeral predicate
Thu, 26 Mar 2009 14:30:20 +0000 paulson merged
Thu, 26 Mar 2009 14:10:48 +0000 paulson New theorems mostly concerning infinite series.
Thu, 26 Mar 2009 20:08:55 +0100 wenzelm interpretation/interpret: prefixes are mandatory by default;
Thu, 26 Mar 2009 19:24:21 +0100 wenzelm interpretation/interpret: prefixes are mandatory by default;
Thu, 26 Mar 2009 19:00:29 +0100 wenzelm interpretation/interpret: prefixes within locale expression are mandatory by default;
Thu, 26 Mar 2009 18:59:25 +0100 wenzelm locale_expression: mandatory as parameter;
Thu, 26 Mar 2009 17:00:59 +0100 wenzelm register_locale: produce stamps at the spot where elements are registered;
Thu, 26 Mar 2009 15:20:50 +0100 wenzelm pretty_rule/print_results: no thm status here -- it is potentially slow and mostly uninformative/confusing as long as proofs are still unfinished;
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
(0) -30000 -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip