Wed, 21 Jul 2010 16:14:16 +0200 wenzelm eliminated old time_use/time_use_thy variants -- timing is implicitly controlled via Output.timing;
Wed, 21 Jul 2010 15:44:36 +0200 wenzelm moved src/Tools/Compute_Oracle to src/HOL/Matrix/Compute_Oracle -- it actually depends on HOL anyway;
Wed, 21 Jul 2010 15:31:38 +0200 wenzelm replaced Thy_Info.the_theory by Context.this_theory -- avoid referring to accidental theory loader state;
Wed, 21 Jul 2010 15:23:46 +0200 wenzelm thm_deps/unused_thms: Context.get_theory based on proper theory ancestry, not accidental theory loader state;
Wed, 21 Jul 2010 15:13:36 +0200 wenzelm explicit dependency on theory HOL;
Wed, 21 Jul 2010 15:02:51 +0200 wenzelm ML antiquotations @{theory} and @{theory_ref} refer to the theory ancestry, not any accidental theory loader state;
Wed, 21 Jul 2010 14:27:05 +0200 wenzelm added Context.get_theory -- avoid referring to accidental theory loader state (cf. Thy_Info.get_theory);
Wed, 21 Jul 2010 13:55:44 +0200 wenzelm thy_deps: more direct comparison of sessions, which is presumably what "unfold" is meant to indicate here -- also avoid referring to accidental theory loader state;
Wed, 21 Jul 2010 13:25:14 +0200 wenzelm clarified/exported Future.worker_subgroup, which is already the default for Future.fork;
Tue, 20 Jul 2010 23:16:21 +0200 wenzelm qualified Thy_Info.get_theory;
Tue, 20 Jul 2010 23:09:49 +0200 wenzelm discontinued pervasive val theory = Thy_Info.get_theory -- prefer antiquotations in most situations;
Tue, 20 Jul 2010 22:03:37 +0200 wenzelm further Mac OS X deviations;
Tue, 20 Jul 2010 21:57:26 +0200 wenzelm warning in proper transaction context;
Tue, 20 Jul 2010 21:49:39 +0200 wenzelm SML/NJ: refrain from modifying toplevel pp for type string -- unclear if it could work here;
Tue, 20 Jul 2010 21:07:23 +0200 wenzelm avoid duplicate printing of 'theory' state (cf. 173974e07dea);
Tue, 20 Jul 2010 20:56:28 +0200 wenzelm toplevel pp for Proof.state and Toplevel.state;
Tue, 20 Jul 2010 20:10:27 +0200 wenzelm execute document version at high priority;
Tue, 20 Jul 2010 18:33:19 +0200 wenzelm Topelevel.run_command: interactive mode for initial 'theory' ensures that Thy_Info.begin_theory loads parent theories;
Tue, 20 Jul 2010 18:19:50 +0200 wenzelm edit_document: join parent execution in synchronous/uninterruptible mode, to prevent spurious interrupts when cascaded executions run into each other;
Tue, 20 Jul 2010 17:35:42 +0200 wenzelm back to more strict dependencies, even for canceled groups (reverting parts of 02936e77a07c);
Tue, 20 Jul 2010 16:42:48 +0200 wenzelm export Graph.get_entry for convenience;
Tue, 20 Jul 2010 14:44:33 +0200 wenzelm eliminated old-style sys_error/SYS_ERROR in favour of exception Fail -- after careful checking that there is no overlap with existing handling of that;
Tue, 20 Jul 2010 14:41:13 +0200 wenzelm tuned;
Tue, 20 Jul 2010 11:11:15 +0200 wenzelm observe follow_caret (again);
Mon, 19 Jul 2010 22:19:18 +0200 wenzelm Session: predefined real time parameters;
Mon, 19 Jul 2010 08:59:43 +0200 haftmann bind and then latex symbols
Sun, 18 Jul 2010 17:56:04 +0200 wenzelm minor update of dependencies;
Fri, 16 Jul 2010 15:28:23 +0200 haftmann corrected range chec
Fri, 16 Jul 2010 15:28:22 +0200 haftmann first roughly working version of Imperative HOL for Scala
Fri, 16 Jul 2010 14:11:08 +0200 haftmann tuned
Fri, 16 Jul 2010 13:58:37 +0200 haftmann merged
Fri, 16 Jul 2010 13:58:29 +0200 haftmann a first sketch for Imperative HOL witht Scala
Fri, 16 Jul 2010 13:57:46 +0200 haftmann don't fail gracefully
Fri, 16 Jul 2010 13:57:29 +0200 haftmann restored long-broken syntax sanity checks
Fri, 16 Jul 2010 13:57:29 +0200 haftmann tuned interpunctation
Fri, 16 Jul 2010 10:23:21 +0200 haftmann fragments of Scala
Thu, 15 Jul 2010 10:16:17 +0200 haftmann merged
Thu, 15 Jul 2010 10:12:49 +0200 haftmann adjusted; fixed typo
Thu, 15 Jul 2010 08:14:05 +0200 haftmann dropped spurious export_code
Wed, 14 Jul 2010 19:10:23 +0100 kleing use different log server (macbroy23 down)
Wed, 14 Jul 2010 17:27:54 +0200 haftmann more consistent spacing in generated monadic code
Wed, 14 Jul 2010 17:16:02 +0200 haftmann braced needed in layout-insensitive syntax
Wed, 14 Jul 2010 17:15:58 +0200 haftmann repaired some implementations of imperative operations
Wed, 14 Jul 2010 16:45:30 +0200 haftmann repaired reference implementation for OCaml
Wed, 14 Jul 2010 16:45:30 +0200 haftmann part of pervasive test
Wed, 14 Jul 2010 16:45:30 +0200 haftmann avoid ambiguities; tuned
Wed, 14 Jul 2010 16:45:29 +0200 haftmann repaired of_list implementation for SML, OCaml
Wed, 14 Jul 2010 16:13:14 +0200 haftmann avoid export_code ... file -
Wed, 14 Jul 2010 16:02:50 +0200 haftmann explicit optional checking
Wed, 14 Jul 2010 15:49:29 +0200 haftmann added Isar syntax for code checking
Wed, 14 Jul 2010 15:49:29 +0200 haftmann corrected import
Wed, 14 Jul 2010 15:08:02 +0200 haftmann use generic description slot for formal code checking
Wed, 14 Jul 2010 14:53:44 +0200 haftmann formal slot for code checker
Wed, 14 Jul 2010 14:53:44 +0200 haftmann export_code without file prints to standard output
Wed, 14 Jul 2010 14:20:47 +0200 haftmann check without explicit path
Wed, 14 Jul 2010 14:16:12 +0200 haftmann load cache_io before code generator; moved adhoc-overloading to generic tools
Wed, 14 Jul 2010 12:27:44 +0200 haftmann tuned infix syntax
Wed, 14 Jul 2010 12:27:44 +0200 haftmann dropped M suffix; added predicate monad bind
Wed, 14 Jul 2010 12:27:43 +0200 haftmann self-built symbol for part of bind operator
Wed, 14 Jul 2010 09:42:44 +0200 haftmann redirect stderr to stdout
Tue, 13 Jul 2010 21:07:12 +0100 paulson merged
Tue, 13 Jul 2010 11:27:19 +0100 paulson merged
Tue, 13 Jul 2010 11:26:16 +0100 paulson corrected mixfix declarations and tidied proofs
Tue, 13 Jul 2010 17:19:35 +0100 paulson merged
Tue, 13 Jul 2010 17:19:08 +0100 paulson Fixed syntax and tidied some proofs
Tue, 13 Jul 2010 18:01:42 +0200 bulwahn correcting function name of generator for products of traditional code generator (introduced in 0040bafffdef)
Tue, 13 Jul 2010 16:30:13 +0200 haftmann consolidated names of theorems
Tue, 13 Jul 2010 16:21:49 +0200 haftmann qualified names for (really) all array operations
Tue, 13 Jul 2010 16:12:40 +0200 haftmann canonical argument order for get
Tue, 13 Jul 2010 16:00:56 +0200 haftmann qualified names for (almost) all array operations
Tue, 13 Jul 2010 15:37:31 +0200 haftmann canonical argument order for present
Tue, 13 Jul 2010 15:34:02 +0200 haftmann canonical argument order for length
Tue, 13 Jul 2010 11:23:21 +0100 kleing merged
Tue, 13 Jul 2010 11:21:22 +0100 kleing new crontab
Tue, 13 Jul 2010 12:20:23 +0200 haftmann merged
Tue, 13 Jul 2010 12:16:24 +0200 haftmann proper merge of operation changes and generic do-syntax
Tue, 13 Jul 2010 12:05:20 +0200 haftmann merged
Tue, 13 Jul 2010 12:01:34 +0200 haftmann hide_const; update replaces change
Tue, 13 Jul 2010 11:17:13 +0100 kleing remove separate afp settings again, use plain mac-poly64-M4 instead.
Tue, 13 Jul 2010 11:01:12 +0100 kleing merged
Tue, 13 Jul 2010 11:00:20 +0100 kleing new settings for afp test
Tue, 13 Jul 2010 12:00:11 +0200 krauss Heap_Monad uses Monad_Syntax
Tue, 13 Jul 2010 11:50:22 +0200 krauss State_Monad uses Monad_Syntax
Tue, 13 Jul 2010 00:15:37 +0200 krauss uniform do notation for monads
Tue, 13 Jul 2010 00:15:37 +0200 krauss generic ad-hoc overloading via check/uncheck
Tue, 13 Jul 2010 11:38:04 +0200 haftmann corrected title
Tue, 13 Jul 2010 11:38:03 +0200 haftmann theorem collections do not contain default rules any longer
Tue, 13 Jul 2010 02:29:05 +0200 boehmes fixed handling of Ball/Bex: turn equalities into meta-equalities for the rewriting conversions;
Mon, 12 Jul 2010 22:35:41 +0200 wenzelm removed unused/untested IOA 'automaton' package;
Mon, 12 Jul 2010 22:17:31 +0200 wenzelm removed impractical tolerate_legacy_features flag;
Mon, 12 Jul 2010 22:14:11 +0200 wenzelm tuned comment;
Mon, 12 Jul 2010 22:07:36 +0200 wenzelm removed legacy aliases;
Mon, 12 Jul 2010 21:38:37 +0200 wenzelm moved misc legacy stuff from OldGoals to Misc_Legacy;
Mon, 12 Jul 2010 21:12:18 +0200 wenzelm eliminated OldGoals.strip_context;
Mon, 12 Jul 2010 20:35:10 +0200 wenzelm removed old HOL/HOLCF-Modelcheck setup, which has been unused/untested for many years;
Mon, 12 Jul 2010 20:21:39 +0200 wenzelm do not intercept ML exceptions -- printing exception positions/text is the job of the Isar/ML toplevel;
Mon, 12 Jul 2010 18:59:38 +0200 wenzelm some modernization of really ancient Meson experiments;
Mon, 12 Jul 2010 16:40:48 +0200 haftmann dropped empty theory
Mon, 12 Jul 2010 16:38:20 +0200 haftmann moved auxiliary lemma
Mon, 12 Jul 2010 16:26:48 +0200 haftmann dropped unused lemmas of dubious value
Mon, 12 Jul 2010 16:23:30 +0200 haftmann dropped unused lemmas of dubious value
Mon, 12 Jul 2010 16:19:15 +0200 haftmann split off mrec into separate theory
Mon, 12 Jul 2010 16:05:08 +0200 haftmann spelt out relational framework in a consistent way
Mon, 12 Jul 2010 11:39:27 +0200 haftmann avoid explicit mandatory prefix markers when prefixes are mandatory implicitly
Mon, 12 Jul 2010 11:21:56 +0200 haftmann merged
Mon, 12 Jul 2010 11:21:27 +0200 haftmann moved co-regularity to class section; avoid duplicated class_deps
Mon, 12 Jul 2010 10:48:37 +0200 haftmann dropped superfluous [code del]s
Mon, 12 Jul 2010 08:58:27 +0200 haftmann merged
Mon, 12 Jul 2010 08:58:13 +0200 haftmann dropped superfluous [code del]s
Mon, 12 Jul 2010 08:58:12 +0200 haftmann more regular session structure
Sat, 10 Jul 2010 22:39:16 +0200 wenzelm regular image setup for HOL-Library (cf. 4915de09b4d3 and ccae4ecd67f4) -- note that document preparation requires a separate session directory, and library.ML is a bit too generic as a file in the default load path;
Sat, 10 Jul 2010 21:38:16 +0200 wenzelm merged
Fri, 09 Jul 2010 16:44:05 +0100 kleing Added current crontab of macbroy28
Fri, 09 Jul 2010 17:15:03 +0200 krauss moved example to its own file in HOL/ex
Fri, 09 Jul 2010 17:00:42 +0200 haftmann merged
Fri, 09 Jul 2010 16:58:44 +0200 haftmann pervasive success combinator
Fri, 09 Jul 2010 16:32:25 +0200 krauss added "while_option", which needs no well-foundedness; defined "while" in terms of "while_option"
Fri, 09 Jul 2010 10:08:10 +0200 haftmann avoid slightly odd "M" suffix; rename mapM to fold_map (fold_map_abort would be more correct, though)
Fri, 09 Jul 2010 09:48:54 +0200 haftmann adapted to changes
Fri, 09 Jul 2010 09:48:53 +0200 haftmann guard combinator
Fri, 09 Jul 2010 09:48:53 +0200 haftmann tuned reference theory
Fri, 09 Jul 2010 09:48:52 +0200 haftmann tuned array theory
Fri, 09 Jul 2010 08:11:10 +0200 haftmann nicer xsymbol syntax for fcomp and scomp
Thu, 08 Jul 2010 17:23:05 +0200 haftmann dropped ancient in-place compilation of SML; more tests
Thu, 08 Jul 2010 16:48:33 +0200 haftmann updated documentation
Thu, 08 Jul 2010 16:41:57 +0200 haftmann dropped ancient in-place compilation of SML
Thu, 08 Jul 2010 16:28:18 +0200 haftmann more accurate dependencies
Thu, 08 Jul 2010 16:20:03 +0200 haftmann empty default
Thu, 08 Jul 2010 16:19:24 +0200 haftmann checking generated code for various target languages
Thu, 08 Jul 2010 16:19:24 +0200 haftmann tuned titles
Thu, 08 Jul 2010 16:19:23 +0200 haftmann tuned module names
Thu, 08 Jul 2010 16:17:44 +0200 haftmann tuned tabs
Thu, 08 Jul 2010 16:17:44 +0200 haftmann tuned script
Thu, 08 Jul 2010 09:36:23 +0200 haftmann combinator with_tmp_dir
Thu, 08 Jul 2010 09:36:22 +0200 haftmann rm_tree: remove entire file system trees
Wed, 07 Jul 2010 18:17:23 +0200 berghofe Boxes may now have different widths.
Wed, 07 Jul 2010 09:26:54 +0200 hoelzl tuned
Wed, 07 Jul 2010 08:25:23 +0200 bulwahn replaced manual derivation of equations for inductive predicates by automatic derivation by inductive_simps
Wed, 07 Jul 2010 08:25:22 +0200 bulwahn added NEWS entry
Wed, 07 Jul 2010 08:25:21 +0200 bulwahn added the new command inductive_cases to derive simplification equations for inductive predicates; added binding simps for general simplification equation
Tue, 06 Jul 2010 08:08:35 -0700 huffman merged
Mon, 05 Jul 2010 09:14:51 -0700 huffman generalize type of is_interval to class euclidean_space
Mon, 05 Jul 2010 09:12:35 -0700 huffman section -> subsection
Sun, 04 Jul 2010 09:26:30 -0700 huffman generalize some lemmas about derivatives
Sun, 04 Jul 2010 09:25:17 -0700 huffman uniqueness of Frechet derivative
Tue, 06 Jul 2010 21:33:14 +0200 wenzelm implode pseudo utf8, i.e. decode byte-stuffed low ASCII characters;
Tue, 06 Jul 2010 10:02:24 +0200 wenzelm merged
Tue, 06 Jul 2010 09:27:49 +0200 haftmann even more fun with primrec
Tue, 06 Jul 2010 09:21:15 +0200 haftmann refactored reference operations
Tue, 06 Jul 2010 09:21:13 +0200 haftmann tuned
Tue, 06 Jul 2010 09:21:13 +0200 haftmann tuned empty heap
Mon, 05 Jul 2010 16:43:08 +0100 paulson merged
Mon, 05 Jul 2010 14:21:53 +0100 paulson merged
Mon, 05 Jul 2010 14:21:30 +0100 paulson Unification (flexflex) bug fix; making "auto" deterministic
Mon, 05 Jul 2010 16:46:23 +0200 haftmann moved "open" operations from Heap.thy to Array.thy and Ref.thy
Mon, 05 Jul 2010 15:36:37 +0200 haftmann only definite assignment
Mon, 05 Jul 2010 15:25:42 +0200 haftmann moved special operation array_ran here
Mon, 05 Jul 2010 15:25:42 +0200 haftmann remove primitive operation Heap.array in favour of Heap.array_of_list
Mon, 05 Jul 2010 15:12:20 +0200 haftmann tuned proof
Mon, 05 Jul 2010 15:12:20 +0200 haftmann tuned
Mon, 05 Jul 2010 23:07:36 +0200 wenzelm Outer_Syntax.prepare_command: disallow control commands here, and consequently in Isar documents;
Mon, 05 Jul 2010 22:26:20 +0200 wenzelm specific ML_val vs. ML_command;
Mon, 05 Jul 2010 20:36:39 +0200 wenzelm async_state: report within proper transaction context;
Mon, 05 Jul 2010 14:35:00 +0200 haftmann merged
Mon, 05 Jul 2010 14:34:28 +0200 haftmann simplified representation of monad type
Mon, 05 Jul 2010 11:25:06 +0200 wenzelm attempt to reconstruct missing HOL/Codegenerator_Test/ROOT.ML;
Mon, 05 Jul 2010 10:47:39 +0200 wenzelm merged
Mon, 05 Jul 2010 10:42:27 +0200 haftmann updated document
Mon, 05 Jul 2010 10:39:49 +0200 haftmann dropped passed irregular names
Sat, 03 Jul 2010 00:50:35 +0200 blanchet adapt Nitpick to "prod_case" and "*" -> "sum" renaming;
Sat, 03 Jul 2010 00:49:12 +0200 blanchet remove needless signature entry
Fri, 02 Jul 2010 17:27:44 +0200 haftmann references to ghc and ocaml
Fri, 02 Jul 2010 17:27:44 +0200 haftmann explicit code_datatype declaration prevents multiple instantiations later on
Fri, 02 Jul 2010 16:50:53 +0200 haftmann refrain from using datatype declaration -- opens chance for quickcheck later on
Fri, 02 Jul 2010 16:50:52 +0200 haftmann tuned proof
Fri, 02 Jul 2010 16:20:56 +0200 haftmann reverted to verion from fc27be4c6b1c
Fri, 02 Jul 2010 16:15:49 +0200 haftmann traceback for error messages
Fri, 02 Jul 2010 16:10:59 +0200 haftmann accomodate for different behvaiour of nitpick (c.f. also 180e80b4eac1)
Fri, 02 Jul 2010 14:23:18 +0200 haftmann introduced distinct session HOL-Codegenerator_Test
Fri, 02 Jul 2010 14:23:17 +0200 haftmann tuned bootstrap files
Fri, 02 Jul 2010 14:23:17 +0200 haftmann remove codegeneration-related theories from big library theory
Fri, 02 Jul 2010 14:23:17 +0200 haftmann drop unconvenient code declarations
Fri, 02 Jul 2010 14:23:16 +0200 haftmann build image for session HOL-Library; introduced distinct session HOL-Codegenerator_Test
Sun, 04 Jul 2010 21:01:22 +0200 wenzelm general Future.report -- also for Toplevel.async_state;
Sun, 04 Jul 2010 00:05:32 +0200 wenzelm simplified Isabelle_Process.Result: use markup directly;
Sat, 03 Jul 2010 23:24:36 +0200 wenzelm run_command: actually observe "print" flag;
Sat, 03 Jul 2010 22:33:10 +0200 wenzelm Toplevel.run_command: asynchronous state output, as an attempt to address potentially slow pretty printing (e.g. in HOL/Bali);
Sat, 03 Jul 2010 20:36:30 +0200 wenzelm more precise timing;
Sat, 03 Jul 2010 20:20:13 +0200 wenzelm more efficient document model/view -- avoid repeated iteration over commands from start, prefer bulk operations;
Fri, 02 Jul 2010 21:48:54 +0200 wenzelm standard argument order;
Fri, 02 Jul 2010 21:41:06 +0200 wenzelm do not open auxiliary ML structures;
Fri, 02 Jul 2010 20:44:17 +0200 wenzelm tuned white space;
(0) -30000 -10000 -3000 -1000 -192 +192 +1000 +3000 +10000 +30000 tip