Fri, 14 Jan 2011 14:21:26 +0100 hoelzl tuned theorem order
Fri, 14 Jan 2011 13:59:06 +0100 haftmann configuration file for mira
Thu, 13 Jan 2011 23:50:16 +0100 wenzelm eliminated global prems;
Thu, 13 Jan 2011 21:50:13 +0100 wenzelm more precise pretty printing -- to accomodate Scala message layout;
Thu, 13 Jan 2011 20:54:07 +0100 wenzelm less verbosity -- avoid slightly odd tracing information on warning channel;
Thu, 13 Jan 2011 18:00:13 +0100 wenzelm updated Isabelle/jEdit limitations and workarounds;
Thu, 13 Jan 2011 17:39:35 +0100 wenzelm full theory path enables loading parents via master directory and keeps files strictly separate;
Thu, 13 Jan 2011 17:34:45 +0100 wenzelm Toplevel.init_theory: maintain optional master directory, to allow bypassing global Thy_Load.master_path;
Thu, 13 Jan 2011 17:30:52 +0100 wenzelm clarified split_thy_path;
Thu, 13 Jan 2011 17:27:52 +0100 wenzelm less verbosity;
Wed, 12 Jan 2011 16:04:47 -0800 huffman proper 'domain' class instance for 'a defl, with deflation combinator
Wed, 12 Jan 2011 21:57:01 +0100 krauss documented Option.bind
Wed, 12 Jan 2011 21:49:04 +0100 krauss CONTRIBUTORS
Wed, 12 Jan 2011 17:33:47 +0100 wenzelm updated keywords;
Wed, 12 Jan 2011 17:19:50 +0100 wenzelm eliminated global prems;
Wed, 12 Jan 2011 17:14:27 +0100 wenzelm eliminated global prems;
Wed, 12 Jan 2011 16:41:49 +0100 wenzelm updated to ProofGeneral-4.x;
Wed, 12 Jan 2011 16:33:04 +0100 wenzelm eliminated global prems;
Wed, 12 Jan 2011 15:53:37 +0100 wenzelm tuned proof;
Wed, 12 Jan 2011 15:38:57 +0100 wenzelm eliminated global prems;
Wed, 12 Jan 2011 15:22:24 +0100 wenzelm compile;
Wed, 12 Jan 2011 15:15:51 +0100 wenzelm more FIXMEs concerning bad catch-all exception handlers;
Wed, 12 Jan 2011 15:09:26 +0100 wenzelm eliminated obsolete print_sign_exn_unit;
Wed, 12 Jan 2011 15:08:21 +0100 wenzelm reraise interrupts as usual;
Wed, 12 Jan 2011 15:07:29 +0100 wenzelm avoid catch-all exception handler, presumably TERM was meant here;
Wed, 12 Jan 2011 14:34:11 +0100 wenzelm disabled experimental treatment of replacement text for now, which leads to odd spacing and strange effects on non-poppler viewers;
Wed, 12 Jan 2011 14:13:04 +0100 wenzelm observe line length limit;
Wed, 12 Jan 2011 14:07:29 +0100 wenzelm smart_string_of_real: print integer values without fractional part;
Tue, 11 Jan 2011 21:52:10 +0100 wenzelm tuned (cf. 2fe62d602681);
Tue, 11 Jan 2011 20:18:48 +0100 wenzelm added dist/jedit symlink for convenience;
Tue, 11 Jan 2011 20:10:34 +0100 wenzelm record versions of both jEdit and Isabelle;
Tue, 11 Jan 2011 20:01:57 +0100 wenzelm updated to Isabelle2011;
Tue, 11 Jan 2011 19:55:34 +0100 wenzelm isabelle version -i;
Tue, 11 Jan 2011 18:23:29 +0100 haftmann NEWS
Tue, 11 Jan 2011 17:59:35 +0100 bulwahn NEWS
Tue, 11 Jan 2011 17:38:03 +0100 krauss eliminated duplication
Tue, 11 Jan 2011 17:00:21 +0100 wenzelm merged
Tue, 11 Jan 2011 14:14:13 +0100 haftmann tuned text
Tue, 11 Jan 2011 14:12:37 +0100 haftmann "enriched_type" replaces less specific "type_lifting"
Tue, 11 Jan 2011 16:23:28 +0100 wenzelm clarified notion Position.is_reported;
Mon, 10 Jan 2011 22:03:24 +0100 wenzelm refined report_parse_tree: reverse reports happen to produce proper type information for inlined @{term}, @{typ} etc.;
Mon, 10 Jan 2011 21:45:44 +0100 wenzelm refined ML_Lex.flatten: ensure proper separation of tokens;
Mon, 10 Jan 2011 21:21:23 +0100 wenzelm ML compiler: more careful treatment of input tokens -- trailing space ensures proper separation and end position (cf. 82c1e348bc18, 08240feb69c7);
Mon, 10 Jan 2011 18:59:02 +0100 boehmes use just one data slot to VC-related information
Mon, 10 Jan 2011 18:58:54 +0100 boehmes be more precise: also merge option values
Mon, 10 Jan 2011 17:41:45 +0100 boehmes only print warning in a visible context (previously, the warning was printed more than once)
Mon, 10 Jan 2011 17:39:54 +0100 boehmes dropped superfluous error message
Mon, 10 Jan 2011 17:37:11 +0100 krauss removed obsolete make target (now in doc-src, cf. 28b487cd9e15)
Mon, 10 Jan 2011 17:22:48 +0100 wenzelm updated for polyml-5.4.0;
Mon, 10 Jan 2011 16:56:47 +0100 wenzelm made SML/NJ happy;
Mon, 10 Jan 2011 16:45:28 +0100 wenzelm added merge_options convenience;
Mon, 10 Jan 2011 16:07:16 +0100 wenzelm tuned string_of_int to avoid allocation for small integers;
Mon, 10 Jan 2011 15:45:46 +0100 wenzelm eliminated Int.toString;
Mon, 10 Jan 2011 15:30:17 +0100 wenzelm eliminated obsolete LargeInt -- Int is unbounded;
Mon, 10 Jan 2011 15:19:48 +0100 wenzelm standardized split_last/last_elem towards List.last;
Mon, 10 Jan 2011 08:18:49 +0100 bulwahn removing dead code; tuned
Mon, 10 Jan 2011 08:18:48 +0100 bulwahn made SML/NJ happy
Sun, 09 Jan 2011 21:33:41 +0100 wenzelm reverted 08240feb69c7 -- breaks positions of reports;
Sun, 09 Jan 2011 19:58:08 +0100 wenzelm ML_trace: observe context visibility flag (import for Latex mode, for example);
Sun, 09 Jan 2011 20:30:47 +0100 wenzelm more direct treatment of Position.end_offset;
Sun, 09 Jan 2011 16:03:56 +0100 wenzelm discontinued unused end_line, end_column;
Sun, 09 Jan 2011 13:58:31 +0100 wenzelm more scalable HTML.output_width;
Sun, 09 Jan 2011 12:56:00 +0100 wenzelm refined comment (again);
Sat, 08 Jan 2011 11:29:25 -0800 huffman merged
Sat, 08 Jan 2011 11:18:09 -0800 huffman use proper syntactic types for 'syntax' commands
Sat, 08 Jan 2011 10:02:43 -0800 huffman make print translation for Abs_cfun consistent with other binders: prevent eta-contraction, but don't force eta-expansion
Sat, 08 Jan 2011 09:34:08 -0800 huffman use full path for library imports
Sat, 08 Jan 2011 09:30:52 -0800 huffman types -> type_synonym
Sat, 08 Jan 2011 18:01:10 +0100 wenzelm updated NEOS_SERVER, which is now provided via settings;
Sat, 08 Jan 2011 17:39:51 +0100 wenzelm renamed Sum_Of_Squares to Sum_of_Squares;
Sat, 08 Jan 2011 17:30:05 +0100 wenzelm Ord_List.merge convenience;
Sat, 08 Jan 2011 17:14:48 +0100 wenzelm misc tuning and comments based on review of Theory_Data, Proof_Data, Generic_Data usage;
Sat, 08 Jan 2011 16:01:51 +0100 wenzelm modernized structure Prop_Logic;
Sat, 08 Jan 2011 14:32:55 +0100 wenzelm added Context_Position.is_visible_proof, which treats a global theory as invisible (unlike the default);
Sat, 08 Jan 2011 14:30:54 +0100 wenzelm tuned;
Sat, 08 Jan 2011 00:28:31 +0100 wenzelm tuned;
Sat, 08 Jan 2011 00:02:11 +0100 wenzelm tuned headers;
Fri, 07 Jan 2011 23:46:06 +0100 wenzelm merged
Fri, 07 Jan 2011 18:10:43 +0100 bulwahn adding example theory for list comprehension to set comprehension simproc
Fri, 07 Jan 2011 18:10:42 +0100 bulwahn adopting proofs due to new list comprehension to set comprehension simproc
Fri, 07 Jan 2011 18:10:35 +0100 bulwahn adding simproc to rewrite list comprehensions to set comprehensions; adopting proofs
Fri, 07 Jan 2011 17:58:51 +0100 boehmes tuned text
Fri, 07 Jan 2011 15:59:10 +0100 bulwahn merged
Fri, 07 Jan 2011 14:46:28 +0100 bulwahn removing obselete Id comments from HOL/ex theories
Fri, 07 Jan 2011 15:39:13 +0100 boehmes added hints about licensing restrictions and how to enable Z3
Fri, 07 Jan 2011 15:37:53 +0100 boehmes tuned
Fri, 07 Jan 2011 23:30:29 +0100 wenzelm eliminated hard tabs;
Fri, 07 Jan 2011 23:10:33 +0100 wenzelm allow spaces in $SPASS_HOME value;
Fri, 07 Jan 2011 23:07:04 +0100 wenzelm tuned;
Fri, 07 Jan 2011 23:02:12 +0100 wenzelm eliminated alias;
Fri, 07 Jan 2011 22:44:07 +0100 wenzelm do not open ML structures;
Fri, 07 Jan 2011 21:51:28 +0100 wenzelm more standard package setup;
Fri, 07 Jan 2011 21:26:49 +0100 wenzelm do not open ML structures;
Fri, 07 Jan 2011 20:42:25 +0100 wenzelm updated scala;
Fri, 07 Jan 2011 18:32:19 +0100 wenzelm do not open ML structures;
Fri, 07 Jan 2011 18:07:27 +0100 wenzelm do not open Codegen;
Fri, 07 Jan 2011 17:07:00 +0100 wenzelm tuned whitespace, indentation, comments;
Fri, 07 Jan 2011 16:11:02 +0100 wenzelm updated for release;
Fri, 07 Jan 2011 15:55:27 +0100 wenzelm tuned;
Fri, 07 Jan 2011 15:35:00 +0100 wenzelm more precise parentheses and indentation;
Fri, 07 Jan 2011 14:58:15 +0100 wenzelm comments;
Fri, 07 Jan 2011 14:36:41 +0100 wenzelm updated for 2011;
Fri, 07 Jan 2011 13:24:09 +0100 boehmes shortened the warning about uninstalled SMT solvers (the additional hint might get obsolete without further notice)
Fri, 07 Jan 2011 10:28:45 +0100 krauss tuned NEWS
Fri, 07 Jan 2011 09:41:48 +0100 boehmes avoid ML structure aliases (especially single-letter abbreviations)
Fri, 07 Jan 2011 09:26:27 +0100 boehmes made SML/NJ happy
Thu, 06 Jan 2011 17:40:38 -0800 huffman rename constant u_defl to u_liftdefl;
Thu, 06 Jan 2011 16:52:35 -0800 huffman rename constant pdefl to liftdefl_of
Thu, 06 Jan 2011 21:06:18 +0100 ballarin Diagnostic command to show locale dependencies.
Thu, 06 Jan 2011 21:06:17 +0100 ballarin Documentation for 'interpret' and 'sublocale' with mixins.
Thu, 06 Jan 2011 21:06:17 +0100 ballarin Abelian group facts obtained from group facts via interpretation (sublocale).
Thu, 06 Jan 2011 17:51:56 +0100 boehmes differentiate between local and remote SMT solvers (e.g., "z3" vs. "remote_z3");
Tue, 04 Jan 2011 15:46:38 -0800 huffman remove various lemmas redundant with lub_eq_bottom_iff
Tue, 04 Jan 2011 15:32:56 -0800 huffman change some lemma names containing 'UU' to 'bottom'
Tue, 04 Jan 2011 15:03:27 -0800 huffman renamed constant 'UU' to 'bottom', keeping 'UU' as alternative input syntax;
Mon, 03 Jan 2011 17:10:32 +0100 boehmes merged
Mon, 03 Jan 2011 16:49:28 +0100 boehmes updated SMT certificates
Mon, 03 Jan 2011 16:22:08 +0100 boehmes re-implemented support for datatypes (including records and typedefs);
Mon, 03 Jan 2011 14:01:42 +0100 haftmann tuned whitespace
Fri, 31 Dec 2010 00:11:24 +0100 wenzelm do not open structure Codegen;
Thu, 30 Dec 2010 23:42:06 +0100 wenzelm do not open auxiliary ML structures;
Thu, 30 Dec 2010 22:34:53 +0100 wenzelm uniform treatment of type vs. term environment (cf. b654fa27fbc4);
Thu, 30 Dec 2010 22:07:18 +0100 wenzelm uniform treatment of typ_match and raw_match (cf. b654fa27fbc4);
Thu, 30 Dec 2010 13:31:32 +0100 wenzelm tuned isatest settings;
Wed, 29 Dec 2010 22:51:33 +0100 wenzelm merged
Wed, 29 Dec 2010 21:52:44 +0100 krauss more robust decomposition of simultaneous goals
Wed, 29 Dec 2010 21:52:41 +0100 krauss function (default) is legacy feature
Wed, 29 Dec 2010 21:21:11 +0100 wenzelm more scalable Symbol_Pos.explode;
Wed, 29 Dec 2010 20:41:33 +0100 wenzelm tuned ML toplevel pp for type string: observe depth limit;
Wed, 29 Dec 2010 18:18:42 +0100 wenzelm theory loader: implicit load path is considered legacy;
Wed, 29 Dec 2010 17:34:41 +0100 wenzelm explicit file specifications -- avoid secondary load path;
Wed, 29 Dec 2010 13:51:17 +0100 wenzelm check_file: secondary load path is legacy feature;
Wed, 29 Dec 2010 12:37:15 +0100 wenzelm share_common_data dummy;
Wed, 29 Dec 2010 12:34:33 +0100 wenzelm made SML/NJ happy;
Wed, 29 Dec 2010 12:25:22 +0100 wenzelm made SML/NJ happy;
Wed, 29 Dec 2010 12:22:38 +0100 wenzelm tuned comments;
Wed, 29 Dec 2010 12:16:49 +0100 wenzelm made SML/NJ happy;
Tue, 28 Dec 2010 18:28:52 +0100 wenzelm made SML/NJ happy;
Mon, 27 Dec 2010 12:33:21 +0100 krauss function (tailrec) is a legacy feature
Sat, 25 Dec 2010 22:18:58 +0100 krauss dropped duplicate unused lemmas;
Sat, 25 Dec 2010 22:18:55 +0100 krauss partial_function (tailrec) replaces function (tailrec);
Fri, 24 Dec 2010 14:26:10 -0800 huffman remove lemma ideal_completion.principal_induct2, use principal_induct twice instead
Thu, 23 Dec 2010 13:11:40 -0800 huffman NEWS updates for HOLCF
Thu, 23 Dec 2010 11:52:26 -0800 huffman replaced separate lemmas seq{1,2,3} with seq_simps
Thu, 23 Dec 2010 11:51:59 -0800 huffman changed syntax of powerdomain binary union operators
Thu, 23 Dec 2010 12:20:09 +0100 haftmann tuned order of NEWS
Thu, 23 Dec 2010 12:04:29 +0100 haftmann NEWS
Thu, 23 Dec 2010 12:01:02 +0100 haftmann documentation stub on type_lifting
Thu, 23 Dec 2010 09:20:43 +0100 haftmann tuned comments and line breaks
Wed, 22 Dec 2010 18:24:04 -0800 huffman rename function ideal_completion.basis_fun to ideal_completion.extension
Wed, 22 Dec 2010 18:23:48 -0800 huffman fix another proof script broken by a35af5180c01
Wed, 22 Dec 2010 17:51:22 -0800 huffman fix proof script broken by a35af5180c01
Wed, 22 Dec 2010 22:21:14 +0100 haftmann merged
Wed, 22 Dec 2010 22:20:57 +0100 haftmann full localization with possibly multiple entries;
Wed, 22 Dec 2010 21:14:57 +0100 haftmann tool-compliant mapper declaration
Wed, 22 Dec 2010 20:57:13 +0100 haftmann more proof contexts; formal declaration
Wed, 22 Dec 2010 20:44:36 +0100 haftmann mapper is arbitrary term, not only constant;
Wed, 22 Dec 2010 20:08:40 +0100 haftmann tuned comment
Wed, 22 Dec 2010 14:44:03 +0100 wenzelm merged
Wed, 22 Dec 2010 09:02:43 +0100 blanchet made SML/NJ happy
Wed, 22 Dec 2010 13:49:06 +0100 wenzelm check JVM later, to avoid potential conflict with jEdit splash screen;
Wed, 22 Dec 2010 13:30:58 +0100 wenzelm explicit JVM check on startup;
Wed, 22 Dec 2010 12:05:17 +0100 wenzelm more explicit jvm_name;
Wed, 22 Dec 2010 11:52:57 +0100 wenzelm isabelle java: prefer -server here;
Tue, 21 Dec 2010 21:54:51 +0100 wenzelm configuration option "rule_trace";
Tue, 21 Dec 2010 21:31:36 +0100 wenzelm configuration option "syntax_branching_level";
Tue, 21 Dec 2010 21:21:21 +0100 wenzelm configuration option "syntax_ast_trace" and "syntax_ast_stat";
Tue, 21 Dec 2010 21:05:50 +0100 wenzelm more robust ML antiquotations -- allow original tokens without adjacent whitespace;
Tue, 21 Dec 2010 19:35:36 +0100 wenzelm configuration option "ML_trace";
Tue, 21 Dec 2010 17:52:35 +0100 haftmann merged
Tue, 21 Dec 2010 17:52:23 +0100 haftmann id_const replaces mk_id
Tue, 21 Dec 2010 17:52:23 +0100 haftmann tuned type_lifting declarations
Tue, 21 Dec 2010 16:14:46 +0100 haftmann prove more algebraic version of functorial properties; retain old properties for convenience
Tue, 21 Dec 2010 08:43:39 -0800 huffman declare more simp rules, rewrite proofs in Isar-style
Tue, 21 Dec 2010 16:41:31 +0100 hoelzl merged
Tue, 21 Dec 2010 15:00:59 +0100 hoelzl use DERIV_intros
Tue, 21 Dec 2010 14:50:53 +0100 hoelzl generalized monoseq, decseq and incseq; simplified proof for seq_monosub
Tue, 21 Dec 2010 15:16:27 +0100 haftmann merged
Tue, 21 Dec 2010 15:15:55 +0100 haftmann proper static closures
Tue, 21 Dec 2010 15:15:55 +0100 haftmann tuned names
Tue, 21 Dec 2010 14:54:23 +0100 haftmann renamed mk_id to the more canonical id_const
Tue, 21 Dec 2010 14:18:45 +0100 blanchet merged
Tue, 21 Dec 2010 13:57:35 +0100 blanchet better parsing of options, in case the value has '='
Tue, 21 Dec 2010 13:57:19 +0100 blanchet show the relation
Tue, 21 Dec 2010 10:25:17 +0100 blanchet merged
Tue, 21 Dec 2010 10:24:56 +0100 blanchet renamed "sledgehammer_tactic.ML" to "sledgehammer_tactics.ML" (cf. module name);
Tue, 21 Dec 2010 10:18:56 +0100 blanchet added "sledgehammer_tac" as possible reconstructor in Mirabelle
Tue, 21 Dec 2010 12:48:47 +0100 wenzelm merged
Tue, 21 Dec 2010 12:02:05 +0100 boehmes merged
Tue, 21 Dec 2010 11:05:30 +0100 boehmes also provide a view on arguments for "external" built-in symbols (similar to "internal" (real) built-in symbols)
Tue, 21 Dec 2010 01:12:14 +0100 traytel Enabled non fully polymorphic map functions in subtyping
Tue, 21 Dec 2010 11:54:35 +0100 wenzelm make SML/NJ and Poly/ML agree on the type of "before";
Tue, 21 Dec 2010 10:20:33 +0100 haftmann only depend on exisiting statements
Tue, 21 Dec 2010 09:29:53 +0100 haftmann merged
Tue, 21 Dec 2010 09:29:33 +0100 haftmann evaluator separating static and dynamic operations
Tue, 21 Dec 2010 09:19:37 +0100 haftmann tuned naming
Tue, 21 Dec 2010 09:18:29 +0100 haftmann evaluator separating static and dynamic operations
Tue, 21 Dec 2010 09:18:29 +0100 haftmann canonical handling of theory context argument
Tue, 21 Dec 2010 09:16:03 +0100 haftmann merged
Tue, 21 Dec 2010 08:40:39 +0100 haftmann evaluator separating static and dynamic operations
Tue, 21 Dec 2010 08:40:39 +0100 haftmann program is separate argument to serializer
Tue, 21 Dec 2010 07:45:04 +0100 haftmann more explicit structure for serializer invocation
Tue, 21 Dec 2010 08:38:03 +0100 nipkow merged
Tue, 21 Dec 2010 08:37:48 +0100 nipkow tuned proof
Tue, 21 Dec 2010 07:23:21 +0100 haftmann HOLogic.mk_id
Tue, 21 Dec 2010 06:53:20 +0100 blanchet avoid weird symbols in path
Tue, 21 Dec 2010 06:06:28 +0100 blanchet mechanism to keep SMT input and output files around in Mirabelle
Tue, 21 Dec 2010 04:33:17 +0100 blanchet proper handling of the arguments of SMT builtins -- for numerals, ignore the arguments (Pls, Bit0, Bit1, ..), for functions, consider them;
Tue, 21 Dec 2010 03:56:51 +0100 blanchet added "smt_triggers" option to experiment with triggers in Sledgehammer;
Tue, 21 Dec 2010 01:12:17 +0100 blanchet enable E weight generation with unofficial latest version of E (tentatively called E 1.2B) -- backed by Judgment Day
Mon, 20 Dec 2010 23:36:58 +0100 wenzelm Cygwin: Poly/ML 5.4.0 requires libgmp3;
Mon, 20 Dec 2010 23:30:32 +0100 wenzelm updated to polyml-5.4.0;
Mon, 20 Dec 2010 23:26:17 +0100 wenzelm tuned;
Mon, 20 Dec 2010 23:19:16 +0100 wenzelm updated for Poly/ML 5.4.0;
Mon, 20 Dec 2010 22:27:26 +0100 boehmes merged
Mon, 20 Dec 2010 22:02:57 +0100 boehmes avoid ML structure aliases (especially single-letter abbreviations)
Mon, 20 Dec 2010 21:04:45 +0100 boehmes added an additional beta reduction: unfolding of special quantifiers might leave terms unnormalized wrt to beta reductions
Mon, 20 Dec 2010 11:11:51 -0800 huffman merged
Mon, 20 Dec 2010 10:57:01 -0800 huffman configure domain package to work with HOL option type
Mon, 20 Dec 2010 10:48:01 -0800 huffman make internal proofs for deflation and isodefl theorems more robust, by avoiding calls to the simplifier for beta-reduction
Mon, 20 Dec 2010 09:48:16 -0800 huffman simplify proofs
Mon, 20 Dec 2010 09:41:55 -0800 huffman beta-reduction simproc uses lemma Abs_cfun_inverse2 instead of beta_cfun, to be more robust against eta-contraction
Mon, 20 Dec 2010 08:26:47 -0800 huffman configure domain package to work with HOL sum type
Mon, 20 Dec 2010 07:50:47 -0800 huffman replace list_map function with an abbreviation
Mon, 20 Dec 2010 18:48:13 +0100 blanchet merged
Mon, 20 Dec 2010 14:55:24 +0100 blanchet run SPASS and Vampire in SOS mode only if >= 50 facts are passed -- otherwise we are probably minimizing and then it's better if the prover is run only once with a full strategy
Mon, 20 Dec 2010 14:17:49 +0100 blanchet disable feature that was enabled by mistake
Mon, 20 Dec 2010 14:10:40 +0100 blanchet make exceptions more transparent in "debug" mode
Mon, 20 Dec 2010 14:09:45 +0100 blanchet remove spurious line
Mon, 20 Dec 2010 13:52:44 +0100 blanchet use the options provided by Stephan Schulz -- much better
Mon, 20 Dec 2010 12:12:35 +0100 blanchet optionally supply constant weights to E -- turned off by default until properly parameterized
Mon, 20 Dec 2010 17:31:58 +0100 haftmann merged
Mon, 20 Dec 2010 15:37:25 +0100 haftmann type_lifting for predicates
Mon, 20 Dec 2010 16:44:33 +0100 wenzelm proper identifiers for consts and types;
Mon, 20 Dec 2010 15:24:25 +0100 wenzelm some attempts to fit diagnostic output into regular TTY (75-80 characters per line);
Mon, 20 Dec 2010 15:19:15 +0100 wenzelm tuned/clarified some component settings;
Mon, 20 Dec 2010 14:44:00 +0100 wenzelm slightly more standard Isabelle_System.with_tmp_file/with_tmp_dir (cf. Scala version);
Mon, 20 Dec 2010 13:36:25 +0100 wenzelm purged some comments (Locale_Test is already clean thanks to configuration options);
Mon, 20 Dec 2010 13:24:04 +0100 wenzelm actually enable show_hyps option, unlike local_setup in 6da953d30f48 which merely affects the (temporary) auxiliary context;
Mon, 20 Dec 2010 09:45:26 +0100 boehmes merged
Mon, 20 Dec 2010 09:31:47 +0100 boehmes updated SMT certificates
Mon, 20 Dec 2010 09:06:37 +0100 boehmes re-introduced support for nonlinear multiplication in Z3 (overriding the built-in linear multiplication of the SMT-LIB class of solvers)
Mon, 20 Dec 2010 08:45:27 +0100 boehmes derived SMT solver classes override inherited properties (properties of derived classes have a higher priority than properties of base classes)
Mon, 20 Dec 2010 08:17:23 +0100 boehmes perform monomorphization during normalization: schematic numerals might be monomorphized into built-in numerals and then numeral normalization is required
Mon, 20 Dec 2010 08:55:36 +0100 haftmann merge
Fri, 17 Dec 2010 22:00:54 +0100 haftmann more convenient order of type variables
Sun, 19 Dec 2010 18:38:50 -0800 huffman rename function cprod_map to prod_map
Sun, 19 Dec 2010 18:15:21 -0800 huffman switch to transparent ascription, to avoid warning messages
Sun, 19 Dec 2010 18:11:20 -0800 huffman types -> type_synonym
Sun, 19 Dec 2010 18:10:54 -0800 huffman fix typo
Sun, 19 Dec 2010 17:39:20 -0800 huffman merged
Sun, 19 Dec 2010 17:37:19 -0800 huffman use deflations over type 'udom u' to represent predomains;
Sun, 19 Dec 2010 10:33:46 -0800 huffman add lemma u_map_oo
Sun, 19 Dec 2010 09:52:33 -0800 huffman replace foo_approx functions with foo_emb, foo_prj functions for universal domain embeddings
Sun, 19 Dec 2010 06:59:01 -0800 huffman minimize imports; move domain class instances for powerdomain types into Powerdomains.thy
Sun, 19 Dec 2010 06:39:19 -0800 huffman powerdomain theories require class 'bifinite' instead of 'domain'
(0) -30000 -10000 -3000 -1000 -256 +256 +1000 +3000 +10000 +30000 tip