Sat, 13 Nov 2010 21:46:24 +0100 wenzelm always print state of proof commands (notably "qed" etc.);
Sat, 13 Nov 2010 21:01:03 +0100 wenzelm simplified message: malformed symbols are fully internalized, i.e. can be printed without crashing;
Sat, 13 Nov 2010 20:49:02 +0100 wenzelm tuned message;
Sat, 13 Nov 2010 20:20:05 +0100 wenzelm proper escape in regex;
Sat, 13 Nov 2010 20:13:35 +0100 wenzelm report malformed symbols;
Sat, 13 Nov 2010 20:06:52 +0100 wenzelm qualified Symbol_Pos.symbol;
Sat, 13 Nov 2010 19:55:45 +0100 wenzelm total Symbol.source;
Sat, 13 Nov 2010 19:47:23 +0100 wenzelm eliminated slightly odd pervasive Symbol_Pos.symbol;
Sat, 13 Nov 2010 19:27:41 +0100 wenzelm treat Unicode "replacement character" (i.e. decoding error) is malformed;
Sat, 13 Nov 2010 19:21:53 +0100 wenzelm simplified/robustified treatment of malformed symbols, which are now fully internalized (total Symbol.explode etc.);
Sat, 13 Nov 2010 16:46:00 +0100 wenzelm tuned;
Sat, 13 Nov 2010 12:32:21 +0100 wenzelm back to quick_and_dirty, which is still practically important since the scheduler does not jump over subproofs;
Sat, 13 Nov 2010 11:41:02 +0100 wenzelm await_cancellation in the main thread, independently of the execution futures, which might get interrupted or be absent after node deletetion;
Sat, 13 Nov 2010 00:24:41 +0100 wenzelm updated README;
Fri, 12 Nov 2010 21:37:01 +0100 wenzelm defensive defaults for more robust experience for new users;
Fri, 12 Nov 2010 17:44:03 +0100 wenzelm merged
Fri, 12 Nov 2010 15:56:11 +0100 boehmes preliminary support for newer versions of Z3
Fri, 12 Nov 2010 15:56:10 +0100 boehmes turned SMT counterexamples into verbose messages (they had been swallowed before, following the state of smt_trace -- which is off by default), because they might be useful for the user
Fri, 12 Nov 2010 15:56:08 +0100 boehmes let the theory formally depend on the Boogie output
Fri, 12 Nov 2010 15:56:07 +0100 boehmes look for certificates relative to the theory
Fri, 12 Nov 2010 15:56:06 +0100 boehmes dropped numerals from monomorphization blacklist (only particular numerals are builtin, all other numerals should be treated uninterpreted), this blacklist should contain only truely polymorphic builtin constants supported by SMT
Fri, 12 Nov 2010 06:11:29 -0800 huffman merged
Fri, 12 Nov 2010 06:05:26 -0800 huffman update Theory.requires with new theory name
Fri, 12 Nov 2010 14:51:28 +0100 wenzelm tuned signatures;
Fri, 12 Nov 2010 14:06:37 +0100 wenzelm never open Unsynchronized;
Fri, 12 Nov 2010 12:57:02 +0100 wenzelm merged
Wed, 10 Nov 2010 18:45:48 -0800 huffman section headings
Wed, 10 Nov 2010 18:37:11 -0800 huffman reorder chapters for generated document
Wed, 10 Nov 2010 18:30:17 -0800 huffman merge Representable.thy into Domain.thy
Wed, 10 Nov 2010 18:15:21 -0800 huffman move stuff from Domain.thy to Domain_Aux.thy
Wed, 10 Nov 2010 17:56:08 -0800 huffman move map functions to new theory file Map_Functions; add theory file Plain_HOLCF
Wed, 10 Nov 2010 14:59:52 -0800 huffman allow unpointed lazy arguments for definitional domain package
Wed, 10 Nov 2010 14:20:47 -0800 huffman add lemmas lub_below, below_lub; simplify some proofs; remove some unused lemmas
Wed, 10 Nov 2010 13:22:39 -0800 huffman merged
Wed, 10 Nov 2010 13:08:42 -0800 huffman removed unused lemma chain_mono2
Wed, 10 Nov 2010 11:42:35 -0800 huffman rename class 'bifinite' to 'domain'
Wed, 10 Nov 2010 09:59:08 -0800 huffman instance sum :: (predomain, predomain) predomain
Wed, 10 Nov 2010 09:52:50 -0800 huffman configure sum type for fixrec
Wed, 10 Nov 2010 08:18:32 -0800 huffman add class liftdomain, for bifinite domains where DEFL('a u) = u_defl('a)
Wed, 10 Nov 2010 06:02:37 -0800 huffman instance prod :: (predomain, predomain) predomain
Tue, 09 Nov 2010 19:37:11 -0800 huffman adapt isodefl proof script to unpointed types
Tue, 09 Nov 2010 16:37:13 -0800 huffman add 'predomain' class: unpointed version of bifinite
Tue, 09 Nov 2010 08:41:36 -0800 huffman add bifiniteness check for domain_isomorphism command
Tue, 09 Nov 2010 05:23:34 -0800 huffman implement map_of_typ using Pattern.rewrite_term
Tue, 09 Nov 2010 04:47:46 -0800 huffman avoid using stale theory
Mon, 08 Nov 2010 15:13:45 -0800 huffman implement defl_of_typ using Pattern.rewrite_term instead of DeflData theory data
Mon, 08 Nov 2010 14:36:17 -0800 huffman add function the_sort
Mon, 08 Nov 2010 14:09:07 -0800 huffman refactor tmp_thy code
Mon, 08 Nov 2010 06:58:09 -0800 huffman reorganize Bifinite.thy; simplify some proofs related to bifinite class instances
Fri, 12 Nov 2010 11:36:01 +0100 wenzelm treat pervasive "Interrupt" constructor as illegal -- superseded by Exn.Interrupt for internal use and Exn.is_interrupt/Exn.interrupt in user-space;
Fri, 12 Nov 2010 10:58:09 +0100 wenzelm Laze.force_result: more robust treatment of interrupts stemming from peer group cancellation;
Thu, 11 Nov 2010 19:58:07 +0100 wenzelm more precise treatment of deleted nodes;
Thu, 11 Nov 2010 18:55:17 +0100 wenzelm tuned error message;
Thu, 11 Nov 2010 17:07:05 +0100 wenzelm unified type Document.Edit;
Thu, 11 Nov 2010 16:48:46 +0100 wenzelm replaced Document.Node_Text_Edit by Document.Text_Edit, with treatment of deleted nodes;
Thu, 11 Nov 2010 13:23:39 +0100 wenzelm tuned;
Thu, 11 Nov 2010 13:07:41 +0100 wenzelm reduced danger of line breaks within minipage;
Wed, 10 Nov 2010 20:43:22 +0100 wenzelm Sidekick block asset: show first line only;
Wed, 10 Nov 2010 20:21:55 +0100 wenzelm added buffer_text convenience, with explicit locking;
Wed, 10 Nov 2010 17:53:41 +0100 wenzelm use official/portable Multithreading.max_threads_value, which is also subject to user preferences (NB: Thread.numProcessors is apt to lead to surprises like very high numbers for systems with hyperthreading);
Wed, 10 Nov 2010 16:05:15 +0100 wenzelm merged
Wed, 10 Nov 2010 09:03:07 +0100 blanchet make SML/NJ happy
Tue, 09 Nov 2010 16:18:40 +0100 haftmann merged
Tue, 09 Nov 2010 14:02:14 +0100 haftmann slightly changed fun_map_def
Tue, 09 Nov 2010 14:02:14 +0100 haftmann fun_rel_def is no simp rule by default
Tue, 09 Nov 2010 14:02:13 +0100 haftmann more appropriate specification packages; fun_rel_def is no simp rule by default
Tue, 09 Nov 2010 14:02:13 +0100 haftmann type annotations in specifications; fun_rel_def is no simp rule by default; slightly changed fun_map_def; more on predicates on relation functions; proper HOL equations in definitions
Tue, 09 Nov 2010 14:02:13 +0100 haftmann more appropriate specification packages; fun_rel_def is no simp rule by default
Tue, 09 Nov 2010 14:02:12 +0100 haftmann type annotations in specifications; fun_rel_def is no simp rule by default
Tue, 09 Nov 2010 14:02:12 +0100 haftmann fun_rel_def is no simp rule by default
Tue, 09 Nov 2010 14:00:10 +0000 paulson merged
Tue, 09 Nov 2010 13:59:37 +0000 paulson tidied using metis
Wed, 10 Nov 2010 15:59:23 +0100 wenzelm manage folding via sidekick by default;
Wed, 10 Nov 2010 15:47:56 +0100 wenzelm eliminated obsolete heading category -- superseded by heading_level;
Wed, 10 Nov 2010 15:43:06 +0100 wenzelm treat main theory commands like headings, and nest anything else inside;
Wed, 10 Nov 2010 15:42:20 +0100 wenzelm proper treatment of equal heading level;
Wed, 10 Nov 2010 15:41:29 +0100 wenzelm added missing Keyword.THY_SCHEMATIC_GOAL;
Wed, 10 Nov 2010 15:17:25 +0100 wenzelm default Sidekick parser based on section headings;
Wed, 10 Nov 2010 15:00:40 +0100 wenzelm some support for nested source structure, based on section headings;
Wed, 10 Nov 2010 11:44:35 +0100 wenzelm tuned;
Tue, 09 Nov 2010 23:24:46 +0100 wenzelm misc tuning and simplification, using Isabelle_Sidekick.Asset (not sidekick.Asset, which is dynamically dispatched to slightly different semantics);
Tue, 09 Nov 2010 22:37:10 +0100 wenzelm updated version;
Tue, 09 Nov 2010 21:52:05 +0100 wenzelm private counter, to keep externalized ids a bit smaller;
Tue, 09 Nov 2010 21:44:19 +0100 wenzelm added general Synchronized.counter convenience;
Tue, 09 Nov 2010 21:13:06 +0100 wenzelm explicitly identify forked/joined tasks;
Tue, 09 Nov 2010 11:27:58 +0100 wenzelm accomodate old manuals that include pdfsetup.sty without isabelle.sty;
Tue, 09 Nov 2010 11:17:15 +0100 wenzelm merged
Mon, 08 Nov 2010 23:02:20 +0100 krauss removed type-inference-like behaviour from relation_tac completely; tuned
Mon, 08 Nov 2010 20:55:27 +0100 wenzelm avoid clash of \<upharpoonright> vs. \<restriction> (cf. 666ea7e62384 and 3c49dbece0a8);
Mon, 08 Nov 2010 20:50:56 +0100 wenzelm explicitly check uniqueness of symbol recoding;
Mon, 08 Nov 2010 17:44:47 +0100 wenzelm more hints on building and running Isabelle/jEdit from command line;
Mon, 08 Nov 2010 14:41:11 +0100 wenzelm merged
Mon, 08 Nov 2010 14:33:54 +0100 blanchet merge
Mon, 08 Nov 2010 14:33:30 +0100 blanchet reduce the number of monomorphization iterations from 10 (the default) to 4, in the interest of faster SMT solving
Mon, 08 Nov 2010 05:07:18 -0800 huffman merged
Sat, 06 Nov 2010 10:01:00 -0700 huffman merged
Fri, 05 Nov 2010 15:15:28 -0700 huffman (infixl "<<" 55) -> (infix "<<" 50)
Wed, 03 Nov 2010 17:22:25 -0700 huffman simplify some proofs
Wed, 03 Nov 2010 17:06:21 -0700 huffman remove unnecessary stuff from Discrete.thy
Wed, 03 Nov 2010 16:39:23 -0700 huffman remove some unnecessary lemmas; move monofun_LAM to Cfun.thy
Wed, 03 Nov 2010 15:57:39 -0700 huffman add lemma eq_imp_below
Wed, 03 Nov 2010 15:47:46 -0700 huffman discontinue a bunch of legacy theorem names
Wed, 03 Nov 2010 15:31:24 -0700 huffman move a few admissibility lemmas into FOCUS/Stream_adm.thy
Wed, 03 Nov 2010 15:03:16 -0700 huffman simplify some proofs
Mon, 08 Nov 2010 13:53:18 +0100 blanchet compile -- 7550b2cba1cb broke the build
Mon, 08 Nov 2010 13:25:00 +0100 blanchet merge
Mon, 08 Nov 2010 09:10:44 +0100 blanchet recognize Vampire error
Mon, 08 Nov 2010 12:13:51 +0100 boehmes return the process return code along with the process outputs
Mon, 08 Nov 2010 12:13:44 +0100 boehmes better modularization: moved SMT configuration options and diagnostics as well as SMT failure and exception into separate structures (both of which are loaded first and consequently are available to other SMT structures)
Mon, 08 Nov 2010 11:49:28 +0100 haftmann merged
Mon, 08 Nov 2010 10:56:48 +0100 haftmann corrected slip: must keep constant map, not type map; tuned code
Mon, 08 Nov 2010 10:43:24 +0100 haftmann constructors to datatypes in code_reflect can be globbed; dropped unused code
Mon, 08 Nov 2010 09:25:43 +0100 bulwahn adding code and theory for smallvalue generators, but do not setup the interpretation yet
Mon, 08 Nov 2010 02:33:48 +0100 blanchet make sure the SMT solver runs several iterations by lowering the timeout at each iteration -- yields better results in practice
Mon, 08 Nov 2010 02:32:27 +0100 blanchet better detection of completely irrelevant facts
Sun, 07 Nov 2010 18:19:04 +0100 blanchet always use a hard timeout in Mirabelle
Sun, 07 Nov 2010 18:15:13 +0100 blanchet use "smt" (rather than "metis") to reconstruct SMT proofs
Sun, 07 Nov 2010 18:03:24 +0100 blanchet don't pass too many facts on the first iteration of the SMT solver
Sun, 07 Nov 2010 18:02:02 +0100 blanchet catch TimeOut exception
Sun, 07 Nov 2010 17:56:07 +0100 blanchet ensure the SMT solver respects the timeout -- Mirabelle revealed cases where "smt_filter" apparently never returns
(0) -30000 -10000 -3000 -1000 -120 +120 +1000 +3000 +10000 +30000 tip