Sat, 15 Mar 2014 11:22:25 +0100 wenzelm more explicit treatment of verbose mode, which includes concealed entries;
Sat, 15 Mar 2014 10:29:42 +0100 wenzelm removed dead code;
Sat, 15 Mar 2014 10:24:49 +0100 wenzelm clarified retrieve_generic: local error takes precedence, which is relevant for completion;
Sat, 15 Mar 2014 10:14:42 +0100 wenzelm clarified print_local_facts;
Sat, 15 Mar 2014 08:31:33 +0100 haftmann more complete set of lemmas wrt. image and composition
Sat, 15 Mar 2014 03:37:22 +0100 panny merge
Sat, 15 Mar 2014 01:36:38 +0100 panny add error messages for invalid inputs
Fri, 14 Mar 2014 13:27:38 -0700 huffman add lemmas about nhds filter; tuned proof
Fri, 14 Mar 2014 10:59:43 -0700 huffman remove unused lemma which was a direct consequence of tendsto_intros
Fri, 14 Mar 2014 19:15:50 +0100 wenzelm merged
Fri, 14 Mar 2014 17:32:11 +0100 wenzelm merged
Fri, 14 Mar 2014 16:54:01 +0100 wenzelm prefer more robust Synchronized.var;
Fri, 14 Mar 2014 15:41:29 +0100 wenzelm discontinued somewhat pointless "thy_script" keyword kind;
Fri, 14 Mar 2014 15:26:52 +0100 wenzelm conceal improper cases, e.g. relevant for completion (and potentially for markup);
Fri, 14 Mar 2014 15:12:22 +0100 wenzelm conceal somewhat obscure internal facts, e.g. relevant for 'print_theorems', 'find_theorems';
Fri, 14 Mar 2014 14:59:43 +0100 wenzelm more accurate resolution of hybrid facts, which actually changes the sort order of results;
Fri, 14 Mar 2014 14:29:33 +0100 wenzelm tuned -- command 'text' was localized some years ago;
Fri, 14 Mar 2014 12:23:59 +0100 wenzelm back to a form of hybrid facts, to reduce performance impact of ed92ce2ac88e;
Fri, 14 Mar 2014 10:08:36 +0100 wenzelm just one cumulative Proof_Context.facts, with uniform retrieval (including PIDE markup, completion etc.);
Thu, 13 Mar 2014 17:26:22 +0100 wenzelm more frugal recording of changes: join merely requires information from one side;
Thu, 13 Mar 2014 15:05:56 +0100 wenzelm do not test details of error messages;
Thu, 13 Mar 2014 12:28:35 +0100 wenzelm minor tuning -- NB: props are usually empty for global facts;
Thu, 13 Mar 2014 12:09:43 +0100 wenzelm even smarter Path.smart_implode;
Thu, 13 Mar 2014 11:34:05 +0100 wenzelm added ML antiquotation @{path};
Thu, 13 Mar 2014 10:34:48 +0100 wenzelm clarified Path.smart_implode;
Fri, 14 Mar 2014 09:09:33 -0700 huffman generalization of differential_zero_maxmin to class real_normed_vector
Fri, 14 Mar 2014 12:09:51 +0100 blanchet delayed construction of command (and of noncommercial check) + tuning
Fri, 14 Mar 2014 11:52:03 +0100 blanchet tuning
Fri, 14 Mar 2014 11:44:11 +0100 blanchet consolidate consecutive steps that prove the same formula
Fri, 14 Mar 2014 11:31:39 +0100 blanchet remove '__' skolem suffixes before showing terms to users
Fri, 14 Mar 2014 11:15:46 +0100 blanchet undo rewrite rules (e.g. for 'fun_app') in Isar
Fri, 14 Mar 2014 11:05:45 +0100 blanchet debugging stuff
Fri, 14 Mar 2014 11:05:44 +0100 blanchet more simplification of trivial steps
Fri, 14 Mar 2014 11:05:37 +0100 blanchet tuning
Fri, 14 Mar 2014 10:17:32 +0100 blanchet tuned wording (pun)
Fri, 14 Mar 2014 10:08:33 +0100 blanchet document the new 'nonexhaustive' option (cf. 52e8f110fec3)
Fri, 14 Mar 2014 09:56:06 +0100 blanchet made SML/NJ happier
Fri, 14 Mar 2014 02:54:00 +0100 panny print warning if some constructors are missing;
Fri, 14 Mar 2014 01:28:15 +0100 blanchet updated Sledgehammer docs w.r.t. 'smt2' and 'z3_new'
Fri, 14 Mar 2014 01:28:14 +0100 blanchet updated documentation w.r.t. 'z3_non_commercial' option in Isabelle/jEdit
Fri, 14 Mar 2014 01:28:13 +0100 blanchet updated NEWS and CONTRIBUTORS (BNF, SMT2, Sledgehammer)
Thu, 13 Mar 2014 16:07:27 -0700 huffman remove ordered_euclidean_space constraint from brouwer/derivative lemmas;
Thu, 13 Mar 2014 17:36:56 +0100 nipkow typos
Thu, 13 Mar 2014 16:39:08 +0100 traytel merged
Thu, 13 Mar 2014 16:28:25 +0100 traytel tuned tactics
Thu, 13 Mar 2014 11:15:04 +0100 traytel simplified internal codatatype construction
Thu, 13 Mar 2014 16:21:09 +0100 blanchet updated SMT2 examples and certificates
Thu, 13 Mar 2014 16:17:14 +0100 blanchet updated SMT2 certificates
Thu, 13 Mar 2014 15:54:41 +0100 blanchet added Z3 4.3.0 as component (for use with 'smt2' method)
Thu, 13 Mar 2014 14:55:38 +0100 blanchet updated SMT example certificates
Thu, 13 Mar 2014 14:48:20 +0100 blanchet added 'smt2_status' to keywords
Thu, 13 Mar 2014 14:48:20 +0100 blanchet avoid name clash
Thu, 13 Mar 2014 14:48:20 +0100 blanchet simplify index handling
Thu, 13 Mar 2014 14:48:20 +0100 blanchet more robust indices
Thu, 13 Mar 2014 14:48:20 +0100 blanchet correctly reconstruct helper facts (e.g. 'nat_int') in Isar proofs
Thu, 13 Mar 2014 14:48:20 +0100 blanchet move lemmas to theory file, towards textual proof reconstruction
Thu, 13 Mar 2014 14:48:05 +0100 blanchet simpler translation of 'div' and 'mod' for Z3
Thu, 13 Mar 2014 13:18:14 +0100 blanchet tuning
Thu, 13 Mar 2014 13:18:14 +0100 blanchet tuning
Thu, 13 Mar 2014 13:18:14 +0100 blanchet thread through step IDs from Z3 to Sledgehammer
Thu, 13 Mar 2014 13:18:14 +0100 blanchet adapted to ML structure renaming
Thu, 13 Mar 2014 13:18:14 +0100 blanchet tuning
Thu, 13 Mar 2014 13:18:14 +0100 blanchet avoid names that may clash with Z3's output (e.g. '')
Thu, 13 Mar 2014 13:18:14 +0100 blanchet do less work in 'filter' mode
Thu, 13 Mar 2014 13:18:14 +0100 blanchet let exception pass through in debug mode
Thu, 13 Mar 2014 13:18:14 +0100 blanchet simplified preplaying information
Thu, 13 Mar 2014 13:18:14 +0100 blanchet renamed (hardly used) 'prod_pred' and 'option_pred' to 'pred_prod' and 'pred_option'
Thu, 13 Mar 2014 13:18:14 +0100 blanchet simplified solution parsing
Thu, 13 Mar 2014 13:18:14 +0100 blanchet adapted to renamed ML files
Thu, 13 Mar 2014 13:18:13 +0100 blanchet renamed ML files
Thu, 13 Mar 2014 13:18:13 +0100 blanchet reintroduced old model reconstruction code -- still needs to be ported
Thu, 13 Mar 2014 13:18:13 +0100 blanchet slacker error code policy for Z3
Thu, 13 Mar 2014 13:18:13 +0100 blanchet repaired 'if' logic
Thu, 13 Mar 2014 13:18:13 +0100 blanchet killed a few 'metis' calls
Thu, 13 Mar 2014 13:18:13 +0100 blanchet honor the fact that the new Z3 can generate Isar proofs
Thu, 13 Mar 2014 13:18:13 +0100 blanchet have Sledgehammer generate Isar proofs from Z3 proofs
Thu, 13 Mar 2014 13:18:13 +0100 blanchet tuned ML interface
Thu, 13 Mar 2014 13:18:13 +0100 blanchet integrate SMT2 with Sledgehammer
Thu, 13 Mar 2014 13:18:13 +0100 blanchet removed tracing output
Thu, 13 Mar 2014 13:18:13 +0100 blanchet use 'smt2' in SMT examples as much as currently possible
Thu, 13 Mar 2014 13:18:13 +0100 blanchet moved 'SMT2' (SMT-LIB-2-based SMT module) into Isabelle
Thu, 13 Mar 2014 08:56:08 +0100 haftmann tuned proofs
Thu, 13 Mar 2014 08:56:08 +0100 haftmann dropped redundant theorems
Thu, 13 Mar 2014 08:56:08 +0100 haftmann tuned
Thu, 13 Mar 2014 08:56:07 +0100 haftmann monotonicity in complete lattices
Thu, 13 Mar 2014 07:07:07 +0100 nipkow enhanced simplifier solver for preconditions of rewrite rule, can now deal with conjunctions
Wed, 12 Mar 2014 22:57:50 +0100 wenzelm tuned signature -- clarified module name;
Wed, 12 Mar 2014 22:44:55 +0100 wenzelm added ML antiquotation @{here};
Wed, 12 Mar 2014 22:41:04 +0100 wenzelm ML_Context.check_antiquotation still required;
Wed, 12 Mar 2014 21:58:48 +0100 wenzelm simplified programming interface to define ML antiquotations -- NB: the transformed context ignores updates of the context parser;
Wed, 12 Mar 2014 21:29:46 +0100 wenzelm proper base comparison;
Wed, 12 Mar 2014 21:28:09 +0100 wenzelm tuned;
Wed, 12 Mar 2014 17:25:28 +0100 wenzelm tuned proofs;
Wed, 12 Mar 2014 17:02:05 +0100 wenzelm more explicit markup and explanation of the improper status of 'back', following the AFP style-guide;
Wed, 12 Mar 2014 16:43:17 +0100 wenzelm clarified Markup.operator vs. Markup.delimiter;
Wed, 12 Mar 2014 16:11:47 +0100 wenzelm more explicit markup for Token.Literal;
Wed, 12 Mar 2014 14:37:14 +0100 wenzelm tuned signature;
Wed, 12 Mar 2014 14:23:26 +0100 wenzelm modernized setup;
Wed, 12 Mar 2014 14:22:51 +0100 wenzelm tuned;
Wed, 12 Mar 2014 14:17:13 +0100 wenzelm some document antiquotations for Isabelle/jEdit elements;
Wed, 12 Mar 2014 12:18:41 +0100 wenzelm merged
Wed, 12 Mar 2014 10:42:28 +0100 wenzelm more explicit Sign.change_check -- detect structural mistakes where they emerge, not at later theory merges;
Tue, 11 Mar 2014 22:49:28 +0100 wenzelm more efficient local theory operations, by imposing a linear change discipline on the main types/consts tables, in order to speed-up Proof_Context.transfer_syntax required for Local_Theory.raw_theory_result;
Tue, 11 Mar 2014 21:58:41 +0100 wenzelm slightly more rubust (and opportunistic) exit for old-fashioned theory_to_proof, which is used by global 'sublocale' with Named_Target.init but without proper exit;
Tue, 11 Mar 2014 18:36:17 +0100 wenzelm more standard internal data integrity;
Tue, 11 Mar 2014 18:26:47 +0100 wenzelm tables with changes relative to some common base version -- support for efficient join/merge of big global tables with small local updates;
Tue, 11 Mar 2014 14:28:39 +0100 wenzelm tuned signature;
Tue, 11 Mar 2014 13:58:22 +0100 wenzelm tuned comment;
Tue, 11 Mar 2014 10:14:45 +0100 wenzelm minor performance tuning via fast matching filter;
Tue, 11 Mar 2014 17:18:42 +0100 blanchet added missing theorems to unfolding set
Tue, 11 Mar 2014 17:18:41 +0100 blanchet moved 'Quickcheck_Narrowing' further down the theory graph
Tue, 11 Mar 2014 17:18:39 +0100 blanchet make it possible to load Quickcheck exhaustive & narrowing in parallel
Tue, 11 Mar 2014 15:34:38 +0100 blanchet full path
Tue, 11 Mar 2014 11:32:32 +0100 hoelzl measurable_lfp/gfp: indirection not necessary
Mon, 10 Mar 2014 23:03:51 +0100 wenzelm merged
Mon, 10 Mar 2014 23:03:15 +0100 wenzelm tuned proofs;
Mon, 10 Mar 2014 22:40:48 +0100 wenzelm proper Char comparison, despite weakly-typed Scala (cf. 5ff5208de089);
Mon, 10 Mar 2014 22:39:37 +0100 wenzelm tuned message;
Mon, 10 Mar 2014 22:28:20 +0100 wenzelm tuned message;
Mon, 10 Mar 2014 22:22:03 +0100 wenzelm include long identifiers in the reckoning of words (e.g. "integer.lifting" vs. 'lifting_update');
(0) -30000 -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 tip