Sat, 16 Nov 2013 19:23:16 +0100 wenzelm tuned;
Sat, 16 Nov 2013 18:34:11 +0100 wenzelm merged
Sat, 16 Nov 2013 18:31:30 +0100 wenzelm tuned proofs;
Sat, 16 Nov 2013 18:08:57 +0100 wenzelm tuned signature;
Sat, 16 Nov 2013 17:52:01 +0100 wenzelm tuned signature -- clarified Proof General legacy;
Sat, 16 Nov 2013 17:39:11 +0100 wenzelm toplevel function "use" refers to raw ML bootstrap environment;
Sat, 16 Nov 2013 17:04:17 +0100 wenzelm obsolete;
Sat, 16 Nov 2013 16:57:09 +0100 wenzelm proper thy_load command 'boogie_file' -- avoid direct access to file-system;
Sat, 16 Nov 2013 13:12:02 +0100 wenzelm tuned signature;
Sat, 16 Nov 2013 13:07:38 +0100 wenzelm updated example;
Sat, 16 Nov 2013 12:41:16 +0100 wenzelm prefer UTF8.decode_permissive;
Sat, 16 Nov 2013 12:29:10 +0100 wenzelm more distinctive Isabelle_Process.Output vs. Isabelle_Process.Protocol_Output;
Fri, 15 Nov 2013 19:31:10 +0100 wenzelm more specific Protocol_Output: empty message.body, main content via bytes/text;
Thu, 14 Nov 2013 17:39:32 +0100 wenzelm tuned imports;
Thu, 14 Nov 2013 17:17:57 +0100 wenzelm tuned signature;
Thu, 14 Nov 2013 16:55:32 +0100 wenzelm immutable byte vectors versus UTF8 strings;
Fri, 15 Nov 2013 22:02:05 +0100 haftmann dropped duplicate of of_bool
Fri, 15 Nov 2013 22:02:01 +0100 haftmann proper code equations for Gcd and Lcm on nat and int
Sat, 16 Nov 2013 07:45:53 +0100 nipkow tuned
Thu, 14 Nov 2013 20:55:09 +0100 blanchet fixed type variable confusion in 'datatype_new_compat'
Thu, 14 Nov 2013 19:54:10 +0100 blanchet implemented 'tptp_translate'
Thu, 14 Nov 2013 16:10:31 +0100 blanchet reintroduced (unimplemented) 'tptp_translate' tool
Thu, 14 Nov 2013 15:57:48 +0100 blanchet have MaSh support nameless facts (i.e. proofs) and use that support
Thu, 14 Nov 2013 15:40:06 +0100 blanchet made SML/NJ happy
Thu, 14 Nov 2013 15:40:06 +0100 blanchet renamed thm
Thu, 14 Nov 2013 13:03:09 +0100 haftmann explicit inclusion of data refinement theory into HOL-Library session
Thu, 14 Nov 2013 10:59:22 +0100 nipkow tuned to improve automation (for REPEAT)
Wed, 13 Nov 2013 19:12:15 +0100 haftmann separated comparision on bit operations into separate theory
Wed, 13 Nov 2013 15:36:32 +0100 traytel prohibit locally fixed type variables in bnf definitions
Wed, 13 Nov 2013 15:36:32 +0100 traytel tuned
Wed, 13 Nov 2013 15:36:32 +0100 traytel standard relator for list bnf
Wed, 13 Nov 2013 11:23:25 +0100 traytel tuned example
Wed, 13 Nov 2013 12:32:26 +0100 blanchet shortened generated property name
Wed, 13 Nov 2013 10:53:36 +0100 traytel more explicit syntax for defining a bnf
Wed, 13 Nov 2013 09:37:00 +0100 hoelzl fix document generation for HOL-Probability
Tue, 12 Nov 2013 20:08:29 +0100 hoelzl fix document generation for Extended_Nat
Tue, 12 Nov 2013 19:28:56 +0100 hoelzl measure of a countable union
Tue, 12 Nov 2013 19:28:56 +0100 hoelzl add restrict_space measure
Tue, 12 Nov 2013 19:28:55 +0100 hoelzl better support for enat and ereal conversions
Tue, 12 Nov 2013 19:28:55 +0100 hoelzl enat is countable
Tue, 12 Nov 2013 19:28:54 +0100 hoelzl add equalities for SUP and INF over constant functions
Tue, 12 Nov 2013 19:28:54 +0100 hoelzl add finite_select_induct; move generic lemmas from MV_Analysis/Linear_Algebra to the HOL image
Tue, 12 Nov 2013 19:28:53 +0100 hoelzl add acyclicI_order
Tue, 12 Nov 2013 19:28:52 +0100 hoelzl stronger inc_induct and dec_induct
Tue, 12 Nov 2013 19:28:51 +0100 hoelzl countability of the image of a reflexive transitive closure
Tue, 12 Nov 2013 19:28:51 +0100 hoelzl support of_rat with 0 or 1 on order relations
Tue, 12 Nov 2013 19:28:50 +0100 hoelzl equation when indicator function equals 0 or 1
Tue, 12 Nov 2013 14:24:34 +0100 blanchet ported part of function package to new 'Ctr_Sugar' abstraction
Tue, 12 Nov 2013 14:00:56 +0100 blanchet undid copy-paste
Tue, 12 Nov 2013 13:47:24 +0100 blanchet ported 'partial_function' to 'Ctr_Sugar' abstraction
Tue, 12 Nov 2013 13:47:24 +0100 blanchet port list comprehension simproc to 'Ctr_Sugar' abstraction
Tue, 12 Nov 2013 13:47:24 +0100 blanchet added convenience function
Tue, 12 Nov 2013 13:47:24 +0100 blanchet document idiomatic use of 'simps_of_case'
Tue, 12 Nov 2013 13:47:24 +0100 blanchet ported 'Simps_Case_Conv' to use new 'Ctr_Sugar' abstraction
Tue, 12 Nov 2013 13:47:24 +0100 blanchet register old-style datatypes as 'Ctr_Sugar'
Tue, 12 Nov 2013 13:47:24 +0100 blanchet export useful ML function
Tue, 12 Nov 2013 13:47:24 +0100 blanchet moved 'Ctr_Sugar' further up the theory hierarchy, so that 'Datatype' can use it
Tue, 12 Nov 2013 13:47:24 +0100 blanchet tuned headers
Tue, 12 Nov 2013 13:47:24 +0100 blanchet moved 'Ctr_Sugar' files out of BNF, so that it can become a general-purpose abstraction
Tue, 12 Nov 2013 12:04:17 +0100 wenzelm updated sessions;
Tue, 12 Nov 2013 11:52:42 +0100 wenzelm proper latex -- NB: cannot use antiquotation here;
Mon, 11 Nov 2013 22:00:57 +0100 wenzelm merged
Mon, 11 Nov 2013 21:28:08 +0100 wenzelm simplified App template;
Mon, 11 Nov 2013 21:20:51 +0100 wenzelm obsolete;
Mon, 11 Nov 2013 21:16:23 +0100 wenzelm obsolete;
Mon, 11 Nov 2013 21:04:30 +0100 wenzelm tuned message;
Mon, 11 Nov 2013 20:50:12 +0100 wenzelm tuned signature -- removed obsolete Addsimprocs, Delsimprocs;
Mon, 11 Nov 2013 20:00:53 +0100 wenzelm tuned signature;
Mon, 11 Nov 2013 20:51:00 +0100 blanchet minor doc fix
Mon, 11 Nov 2013 18:37:56 +0100 wenzelm merged
Mon, 11 Nov 2013 17:44:21 +0100 wenzelm merged, using src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML and src/HOL/Tools/Sledgehammer/sledgehammer_run.ML from 347c3b0cab44;
Mon, 11 Nov 2013 17:34:44 +0100 wenzelm removed obsolete RC tags;
Mon, 11 Nov 2013 16:40:07 +0100 wenzelm Added tag Isabelle2013-1 for changeset 9c1f21365326
Sat, 09 Nov 2013 18:00:36 +0100 wenzelm tuned; Isabelle2013-1
Sat, 09 Nov 2013 12:47:32 +0100 wenzelm more on completion;
Sat, 09 Nov 2013 11:41:32 +0100 wenzelm adjust modules for Admin/build jars_test;
Sat, 09 Nov 2013 11:24:21 +0100 wenzelm tuned whitespace;
Fri, 08 Nov 2013 17:34:37 +0100 wenzelm added jedit_completion_dismiss_delay for hide_popup, which helps to avoid loosing key events on old popup (no change of default behavior);
Fri, 08 Nov 2013 15:10:16 +0100 wenzelm transfer focus before closing old component -- avoid intermediate focus switch to root component, which is actually visible e.g. on Windows;
Thu, 07 Nov 2013 19:35:57 +0100 wenzelm Added tag Isabelle2013-1-RC4 for changeset 594628261376
Thu, 07 Nov 2013 19:17:53 +0100 wenzelm updated to polyml-5.5.1-1 (fixes-5.5.1 version 1875);
Thu, 07 Nov 2013 13:38:44 +0100 wenzelm tuned;
Thu, 07 Nov 2013 13:34:04 +0100 wenzelm misc tuning;
Wed, 06 Nov 2013 21:20:20 +0100 wenzelm updated to jedit_build-20131106 (Console.jar 5.1.3);
Wed, 06 Nov 2013 20:58:11 +0100 wenzelm join all theory body forks, notably Toplevel.atom_result (diagnostic commands), before peeking at full status;
Wed, 06 Nov 2013 20:46:00 +0100 wenzelm tuned signature;
Wed, 06 Nov 2013 18:15:25 +0100 wenzelm less tiny font for search criteria;
Wed, 06 Nov 2013 18:04:36 +0100 wenzelm tuned tooltips;
Thu, 17 Oct 2013 17:14:06 +0200 Andreas Lochbihler swap equations and premises in the coinductive step for better proof automation
Tue, 05 Nov 2013 18:16:16 +0100 wenzelm no default shortcut for isabelle.reset-font-size -- avoid conflict with unsplit-current;
Tue, 05 Nov 2013 16:41:19 +0100 wenzelm tuned;
Mon, 28 Oct 2013 11:27:14 +0100 noschinl CONTRIBUTORS
Sun, 03 Nov 2013 18:12:23 +0100 wenzelm more on text completion;
Sun, 03 Nov 2013 16:49:52 +0100 wenzelm tuned;
Sun, 03 Nov 2013 16:37:54 +0100 wenzelm more on Monitor panel;
Sun, 03 Nov 2013 16:22:57 +0100 wenzelm more on Timing;
Fri, 01 Nov 2013 17:26:47 +0100 wenzelm more on miscellaneous tools;
Thu, 31 Oct 2013 17:37:08 +0100 wenzelm more screenshots;
Thu, 31 Oct 2013 17:13:39 +0100 wenzelm more screenshots;
Thu, 31 Oct 2013 16:47:36 +0100 wenzelm more on Sledgehammer;
Thu, 31 Oct 2013 16:10:35 +0100 wenzelm more on automatically tried tools;
Wed, 30 Oct 2013 21:23:47 +0100 wenzelm more on prover output;
Wed, 30 Oct 2013 18:47:09 +0100 wenzelm misc tuning and clarification;
Wed, 30 Oct 2013 17:05:23 +0100 wenzelm more on file-system access;
Tue, 29 Oct 2013 21:00:37 +0100 wenzelm tuned;
Tue, 29 Oct 2013 19:45:55 +0100 wenzelm more on problems and workarounds;
Tue, 29 Oct 2013 18:20:20 +0100 wenzelm tuned;
Tue, 29 Oct 2013 16:52:25 +0100 wenzelm clarified isabelle options -l;
Tue, 29 Oct 2013 15:34:29 +0100 wenzelm tuned;
Wed, 16 Oct 2013 18:48:37 +0200 wenzelm clarified workaround: problem is potential blocking of vacuous input (see also Poly/ML SVN 1874);
Mon, 14 Oct 2013 19:50:36 +0200 wenzelm removed dead code (see also db4bf4fb5492);
Wed, 16 Oct 2013 13:02:35 +0200 wenzelm Added tag Isabelle2013-1-RC3 for changeset fbcaa9f08879
Wed, 16 Oct 2013 12:14:35 +0200 wenzelm avoid non-portable int constant -- make SML/NJ happy;
Wed, 16 Oct 2013 12:04:38 +0200 wenzelm avoid empty input and its adverse effect on socket communication, e.g. output message getting "stuck" after vacuous update due to Session.update_options;
Wed, 16 Oct 2013 11:48:42 +0200 wenzelm prefer TCP_NODELAY -- avoid extra buffering due to Nagle's algorithm;
Wed, 16 Oct 2013 11:35:04 +0200 wenzelm basic IO buffer size like for fifo -- imitate implicit flushing behaviour more closely;
Mon, 14 Oct 2013 15:46:35 +0200 wenzelm removed junk (cf. 409d7f7247f4);
Mon, 14 Oct 2013 15:13:11 +0200 kuncar fix a citation
Mon, 14 Oct 2013 15:01:41 +0200 kuncar declare Quotient_Examples/FSet.thy as almost obsolete
Mon, 14 Oct 2013 15:01:41 +0200 kuncar update documentation of important public ML functions in Lifting
Mon, 14 Oct 2013 15:01:37 +0200 kuncar update documentation of Lifting/Transfer and Quotient
Fri, 11 Oct 2013 18:36:51 +0200 kuncar don't allow parametricity theorem for typedefs in setup_lifting. The theorem is not used.
Mon, 14 Oct 2013 15:21:45 +0200 wenzelm tuned;
Sat, 12 Oct 2013 19:41:59 +0200 wenzelm more screenshots;
Sat, 12 Oct 2013 19:00:59 +0200 wenzelm tuned;
Sat, 12 Oct 2013 14:37:45 +0200 wenzelm misc tuning;
Sat, 12 Oct 2013 00:10:07 +0200 wenzelm more strict find_command -- avoid invalid hyperlink_command;
Fri, 11 Oct 2013 23:12:04 +0200 wenzelm more consistent state and GUI update, e.g. relevant for full-screen mode switch with its exit/init side-effect;
Fri, 11 Oct 2013 22:11:07 +0200 wenzelm obsolete;
Fri, 11 Oct 2013 20:45:21 +0200 wenzelm clarified Editor.current_command: allow outdated snapshot;
Fri, 11 Oct 2013 12:06:26 +0200 wenzelm make double sure that AWT/Swing antialiasing is enabled (see also http://www.jedit.org/users-guide/jvm-options.html and jdk/src/share/classes/sun/awt/SunToolkit.java);
Thu, 10 Oct 2013 18:02:08 +0200 wenzelm more documentation;
Thu, 10 Oct 2013 15:46:05 +0200 wenzelm more documentation;
Thu, 10 Oct 2013 14:29:21 +0200 wenzelm more documentation;
Thu, 10 Oct 2013 12:02:12 +0200 wenzelm tuned;
Wed, 09 Oct 2013 23:11:56 +0200 wenzelm NEWS;
Wed, 09 Oct 2013 23:06:23 +0200 wenzelm avoid confusion of isabelle.complete vs. menu item complete-word (NB: alternative shortcuts not shown in menus);
Wed, 09 Oct 2013 15:33:20 +0200 Andreas Lochbihler add congruence rule to prevent code_simp from looping
Wed, 09 Oct 2013 13:40:14 +0200 wenzelm Added tag Isabelle2013-1-RC2 for changeset 782e430e6a83
Mon, 07 Oct 2013 22:19:08 +0200 wenzelm native executable for Linux (see Admin/Linux);
Mon, 07 Oct 2013 22:02:46 +0200 wenzelm proper NULL termination;
Mon, 07 Oct 2013 21:24:44 +0200 wenzelm native executable even for Linux, to avoid surprises with file managers opening executable script as text file;
Mon, 07 Oct 2013 17:55:01 +0200 wenzelm proper warning at run time, not in the parser;
Mon, 07 Oct 2013 13:42:33 +0200 wenzelm prefer "fresh" open -- requires Lion / Mountain Lion;
Mon, 07 Oct 2013 12:28:19 +0200 wenzelm clarified remove_overlay: always flush in order to make sure that apply_query can make a fresh start with the same arguments (see also 6e69f9ca8f1c) -- NB: print functions are idempotent;
Fri, 04 Oct 2013 14:35:00 +0200 blanchet prevent explosion in monomorphizer (e.g. when the facts typerep_int_def typerep_num_def typerep_option_def typerep_node_def are selected)
Fri, 04 Oct 2013 11:12:28 +0200 blanchet more parallelism in blocking mode
Fri, 04 Oct 2013 11:28:28 +0200 blanchet count remote threads as well when balancing CPU usage -- otherwise jEdit users and other users of the "blocking" mode may have to wait for 2 * timeout if they e.g. have 4 cores and 5 provers (the typical situation)
Fri, 04 Oct 2013 18:51:47 +0200 wenzelm another shortcut alias;
Fri, 04 Oct 2013 13:17:49 +0200 wenzelm NEWS;
Thu, 03 Oct 2013 17:03:20 +0200 wenzelm Added tag Isabelle2013-1-RC1 for changeset c37100233af7
Mon, 11 Nov 2013 18:25:13 +0100 blanchet reintroduced check from bd36da55d825 after all, due to hard-to-solve issues outside the N2M code
Mon, 11 Nov 2013 18:13:17 +0100 blanchet removed dead code
Mon, 11 Nov 2013 17:59:41 +0100 blanchet added check to avoid odd situations the N2M code cannot handle
Mon, 11 Nov 2013 17:40:55 +0100 blanchet reverted check introduced in ce58fb149ff6, now that independent functions are allowed (cf. 347c3b0cab44)
Mon, 11 Nov 2013 17:38:53 +0100 blanchet tuned signature
Mon, 11 Nov 2013 16:41:08 +0100 traytel handle independent functions defined in parallel in N2M (in presence of type variables, see ce58fb149ff6)
Mon, 11 Nov 2013 10:23:01 +0100 nipkow tuned
Mon, 11 Nov 2013 10:10:28 +0100 nipkow tuned
Sun, 10 Nov 2013 15:05:06 +0100 haftmann qualifed popular user space names
Sun, 10 Nov 2013 10:02:34 +0100 haftmann dropped obsolete check: dest_num always yields positive number
Sun, 10 Nov 2013 10:02:34 +0100 haftmann simplified: negative number is trivially smaller than 2, and SMT_Builtin.is_builtin_num implies that its argument is a number
Fri, 08 Nov 2013 21:40:07 +0100 nipkow more exercises
Fri, 08 Nov 2013 19:03:14 +0100 blanchet by (auto ...)[1] not by (auto [1])
Fri, 08 Nov 2013 08:59:54 +0100 nipkow added exercise
Thu, 07 Nov 2013 16:08:19 +1100 kleing Add output translation for <a := .., b := .., ..> state notation.
Thu, 07 Nov 2013 02:42:20 +0100 blanchet reintroduce mutually (co)rec check, since the underlying N2M code doesn't quite handle the general case (esp. in presence of type variables)
Thu, 07 Nov 2013 01:01:04 +0100 blanchet more docs
Thu, 07 Nov 2013 00:37:18 +0100 blanchet properly detect when to perform n2m -- e.g. handle the case of two independent functions on irrelevant types being defined in parallel
Wed, 06 Nov 2013 23:05:44 +0100 blanchet reverted 3e1d230f1c00 -- pervasiveness is useful, cf. Coinductive_Nat in the AFP
Wed, 06 Nov 2013 22:50:12 +0100 blanchet simplified code
Wed, 06 Nov 2013 22:42:54 +0100 blanchet fourth attempt at generalizing N2M types (to leverage caching)
Wed, 06 Nov 2013 21:40:41 +0100 blanchet tuning
Tue, 05 Nov 2013 21:23:42 +0100 hoelzl int and nat are conditionally_complete_lattices
Wed, 06 Nov 2013 14:50:50 +0100 blanchet be more open-minded and allow needless mutual recursion for 'prim(co)rec', since we allow it for '(co)datatype' -- eventual warnings (or errors) should be centralized in 'fp_bnf'
Wed, 06 Nov 2013 13:00:45 +0100 blanchet removed dead code
Wed, 06 Nov 2013 13:00:16 +0100 blanchet update docs
Wed, 06 Nov 2013 12:47:50 +0100 blanchet take out possibility of moving corecursive calls past constructors -- this doesn't work in the general case
Wed, 06 Nov 2013 12:01:48 +0100 blanchet took out loopy code
Wed, 06 Nov 2013 10:35:30 +0100 blanchet take out even less aggressive generalization -- it's still too aggressive
Wed, 06 Nov 2013 01:57:22 +0100 blanchet reverted too aggressive 7cb8442298f0
Wed, 06 Nov 2013 01:06:01 +0100 blanchet generalize more aggressively
Tue, 05 Nov 2013 16:53:40 +0100 blanchet avoid subtle failure in the presence of top sort
Tue, 05 Nov 2013 16:47:10 +0100 blanchet tuning
Tue, 05 Nov 2013 16:47:10 +0100 blanchet get mutually recursive maps as well
Tue, 05 Nov 2013 15:10:59 +0100 hoelzl tuned proofs in Approximation
Tue, 05 Nov 2013 13:23:27 +0100 blanchet fixed subtle name shadowing bug
Tue, 05 Nov 2013 12:40:58 +0100 blanchet use right permutation in 'map2'
Tue, 05 Nov 2013 11:55:45 +0100 blanchet stronger normalization, to increase n2m cache effectiveness
Tue, 05 Nov 2013 11:17:42 +0100 blanchet make local theory operations non-pervasive (makes more intuitive sense)
Tue, 05 Nov 2013 09:45:03 +0100 hoelzl NEWS
Tue, 05 Nov 2013 09:45:02 +0100 hoelzl move Lubs from HOL to HOL-Library (replaced by conditionally complete lattices)
Tue, 05 Nov 2013 09:45:00 +0100 hoelzl generalize bdd_above/below_uminus to ordered_ab_group_add
Tue, 05 Nov 2013 09:45:00 +0100 hoelzl restrict Limsup and Liminf to complete lattices
Tue, 05 Nov 2013 09:44:59 +0100 hoelzl use INF and SUP on conditionally complete lattices in multivariate analysis
Tue, 05 Nov 2013 09:44:59 +0100 hoelzl add SUP and INF for conditionally complete lattices
Tue, 05 Nov 2013 09:44:58 +0100 hoelzl use bdd_above and bdd_below for conditionally complete lattices
Tue, 05 Nov 2013 09:44:57 +0100 hoelzl generalize SUP and INF to the syntactic type classes Sup and Inf
Tue, 05 Nov 2013 05:48:08 +0100 blanchet added some N2M caching
Tue, 05 Nov 2013 05:48:08 +0100 blanchet also generalize fixed types
Tue, 05 Nov 2013 05:48:08 +0100 blanchet generalize types when synthetizing n2m (co)recursors, to facilitate reuse
Tue, 05 Nov 2013 05:48:08 +0100 blanchet nicer error message in case of duplicates
Tue, 05 Nov 2013 15:30:53 +1100 kleing use int example like in the rest of IMP (instead of nat)
Mon, 04 Nov 2013 20:10:10 +0100 haftmann dropped dead code
Mon, 04 Nov 2013 20:10:09 +0100 haftmann fact generalization and name consolidation
Mon, 04 Nov 2013 20:10:06 +0100 haftmann streamlined setup of linear arithmetic
Mon, 04 Nov 2013 18:08:47 +0100 blanchet make 'try0' return faster when invoked as part of 'try'
Mon, 04 Nov 2013 17:25:36 +0100 blanchet careful with lists of different lengths
Mon, 04 Nov 2013 16:53:43 +0100 blanchet split 'primrec_new' and 'primcorec' code (to ease bootstrapping, e.g. dependency on datatype 'String' in 'primcorec')
Mon, 04 Nov 2013 15:44:43 +0100 blanchet better error handling
Mon, 04 Nov 2013 14:54:29 +0100 traytel more robust treatment of dead variables in n2m
Mon, 04 Nov 2013 14:46:38 +0100 blanchet more robust n2m w.r.t. 'let's
Mon, 04 Nov 2013 12:40:28 +0100 blanchet tuning
Mon, 04 Nov 2013 11:59:08 +0100 blanchet strengthened tactic
Mon, 04 Nov 2013 11:03:13 +0100 blanchet made n2m code more robust w.r.t. advanced constructs (e.g. lambdas)
Mon, 04 Nov 2013 10:52:41 +0100 blanchet handle constructor syntax in n2m primcorec
Mon, 04 Nov 2013 10:52:41 +0100 blanchet typo
Mon, 04 Nov 2013 10:52:41 +0100 blanchet made sugared 'coinduct' theorem construction n2m-proof
Mon, 04 Nov 2013 10:52:41 +0100 blanchet moved code around
Mon, 04 Nov 2013 10:52:41 +0100 blanchet tuning
Mon, 04 Nov 2013 10:52:41 +0100 blanchet make code more robust w.r.t. applied/unapplied map (primrec vs. primcorec)
Mon, 04 Nov 2013 10:52:41 +0100 blanchet conceal definition
Sat, 02 Nov 2013 17:50:28 +0100 nipkow more exercises
Sat, 02 Nov 2013 17:19:34 +0100 nipkow more exercises
Fri, 01 Nov 2013 18:51:14 +0100 haftmann more simplification rules on unary and binary minus
Thu, 31 Oct 2013 16:54:22 +0100 blanchet generate stable names for axioms
Thu, 31 Oct 2013 11:44:20 +0100 haftmann purely algebraic foundation for even/odd
Thu, 31 Oct 2013 11:44:20 +0100 haftmann moving generic lemmas out of theory parity, disregarding some unused auxiliary lemmas;
Thu, 31 Oct 2013 11:44:20 +0100 haftmann explicit type class for modelling even/odd parity
Thu, 31 Oct 2013 11:44:20 +0100 haftmann generalized of_bool conversion
Thu, 31 Oct 2013 11:44:20 +0100 haftmann separated bit operations on type bit from generic syntactic bit operations
Thu, 31 Oct 2013 11:44:20 +0100 haftmann restructed
Thu, 31 Oct 2013 11:44:20 +0100 haftmann generalised lemma
Thu, 31 Oct 2013 11:44:20 +0100 haftmann more lemmas on division
Thu, 31 Oct 2013 11:44:20 +0100 haftmann more convenient place for a theory in solitariness
Thu, 31 Oct 2013 11:44:20 +0100 haftmann consolidated clone theory
Thu, 31 Oct 2013 11:48:45 +0100 nipkow more exercises
Wed, 30 Oct 2013 17:20:59 +0100 nipkow tuned text
Tue, 29 Oct 2013 13:48:18 +0100 berghofe inst_lift now fully instantiates context to avoid problems with loose bound variables
Tue, 29 Oct 2013 12:13:00 +0100 panny include corecursive functions' arguments in callssss
Tue, 29 Oct 2013 08:06:08 +0100 nipkow more exercises
Mon, 28 Oct 2013 10:29:56 +0100 nipkow merged
Mon, 28 Oct 2013 10:29:43 +0100 nipkow more exercises
Sun, 27 Oct 2013 19:02:26 +0100 blanchet commented out vaporware
Sat, 26 Oct 2013 23:06:40 +0200 nipkow more exercises
Sat, 26 Oct 2013 13:01:41 +0200 blanchet tuning
Sat, 26 Oct 2013 13:00:55 +0200 blanchet tuning
Sat, 26 Oct 2013 12:57:17 +0200 blanchet tuned names (to make them independent from temporary naming convention used in characteristic theorems)
Sat, 26 Oct 2013 12:54:57 +0200 blanchet align 'primrec_new' on 'primcorec' (+ got rid of one more 'dummyT')
Sat, 26 Oct 2013 12:54:39 +0200 blanchet convenience: handle composition gracefully in map in 'primcorec', analogously to 'primrec_new'
Sat, 26 Oct 2013 12:54:21 +0200 blanchet tuned error message
Fri, 25 Oct 2013 16:20:54 +0200 nipkow more exercises
Thu, 24 Oct 2013 19:43:21 +0200 blanchet handle applied ctor arguments gracefully when computing 'callssss' (for recursion through functions)
Thu, 24 Oct 2013 18:50:59 +0200 blanchet tuning
Thu, 24 Oct 2013 18:37:54 +0200 blanchet more correct (!) types for recursive calls
Thu, 24 Oct 2013 15:56:03 +0200 blanchet watch out for 'case' constant canditates whose general type is 'a (e.g. 'undefined')
Thu, 24 Oct 2013 15:32:34 +0200 blanchet got rid of annoying duplicate rewrite rule warnings
Thu, 24 Oct 2013 12:43:33 +0200 blanchet use definitions for LEO-II as well -- this simplifies the code and matches some users' expectations
Thu, 24 Oct 2013 10:03:20 +0200 traytel refactored rtrancl_while; prove termination for finite rtrancl
Wed, 23 Oct 2013 21:12:20 +0200 nipkow more exercises
Wed, 23 Oct 2013 18:04:43 +0200 nipkow added exercises
Wed, 23 Oct 2013 14:53:36 +0200 blanchet added 'primcorec' examples
Wed, 23 Oct 2013 09:58:30 +0200 nipkow tuned
Tue, 22 Oct 2013 16:07:09 +0200 traytel removed junk
Tue, 22 Oct 2013 14:22:06 +0200 traytel update doc according to c0186a0d8cb3
Tue, 22 Oct 2013 14:17:12 +0200 traytel define a trivial nonemptiness witness if none is provided
Mon, 21 Oct 2013 23:45:27 +0200 blanchet made lower-level function available
Mon, 21 Oct 2013 23:35:57 +0200 blanchet more doc -- feedback from Andrei P.
Mon, 21 Oct 2013 21:06:19 +0200 nipkow added exercise
Mon, 21 Oct 2013 10:49:02 +0200 blanchet more docs
Mon, 21 Oct 2013 10:38:21 +0200 blanchet more docs
Mon, 21 Oct 2013 10:31:31 +0200 blanchet more docs
Mon, 21 Oct 2013 10:19:57 +0200 blanchet expand doc a bit
Mon, 21 Oct 2013 09:35:18 +0200 blanchet updated doc
Mon, 21 Oct 2013 09:31:19 +0200 blanchet tuning
Mon, 21 Oct 2013 09:14:05 +0200 blanchet warn about incompatible recursor signature
Mon, 21 Oct 2013 08:27:51 +0200 blanchet more informative abort
Mon, 21 Oct 2013 07:50:32 +0200 blanchet tuning
Mon, 21 Oct 2013 07:24:18 +0200 blanchet systematically close derivations in BNF package
Sun, 20 Oct 2013 23:36:18 +0200 blanchet removed temporary error handling
Sun, 20 Oct 2013 23:29:49 +0200 blanchet strengthened tactic
Sun, 20 Oct 2013 22:51:21 +0200 blanchet tuning
Sun, 20 Oct 2013 22:39:40 +0200 blanchet reintroduced parts of 07a8145aaeba that a22ded8a7f7d wrongly took out
Sun, 20 Oct 2013 21:59:08 +0200 blanchet tuning
Sun, 20 Oct 2013 19:23:28 +0200 blanchet gracefully handle case where a nested recursive variable appears directly on the rhs of a primcorec equation
Sun, 20 Oct 2013 19:20:08 +0200 blanchet tuning
Sun, 20 Oct 2013 19:20:08 +0200 blanchet tuning
Sun, 20 Oct 2013 19:20:08 +0200 blanchet tuning
Sun, 20 Oct 2013 19:20:08 +0200 blanchet tuning
Sun, 20 Oct 2013 18:22:59 +0200 blanchet simplify code
Sun, 20 Oct 2013 17:45:54 +0200 blanchet avoid tactic failure for equations that contain an unapplied 'id'
Sat, 19 Oct 2013 00:00:50 +0200 blanchet improve support for recursion through functions
Fri, 18 Oct 2013 20:26:46 +0200 blanchet handle composition for multiple arguments correctly
Fri, 18 Oct 2013 19:18:32 +0200 panny merge
Fri, 18 Oct 2013 19:03:39 +0200 panny generate callssss
Fri, 18 Oct 2013 18:58:46 +0200 blanchet set stage for more flexible 'primrec' syntax for recursion through functions
Fri, 18 Oct 2013 17:47:25 +0200 blanchet don't print BNF constants
Fri, 18 Oct 2013 16:02:07 +0200 blanchet tuning
Fri, 18 Oct 2013 15:42:55 +0200 blanchet conceal even more ugly constructions
Fri, 18 Oct 2013 15:25:39 +0200 blanchet conceal more ugly constructions
Fri, 18 Oct 2013 15:19:21 +0200 blanchet conceal prim(co)rec definitions
Fri, 18 Oct 2013 15:12:04 +0200 blanchet avoid 'co_' prefix with underscore meaning 'co', since it is our only possible identifier representation of '(co)'
Fri, 18 Oct 2013 15:00:40 +0200 blanchet updated docs
Fri, 18 Oct 2013 14:58:02 +0200 blanchet set code attribute on discriminator equations
Fri, 18 Oct 2013 13:38:55 +0200 blanchet MaSh error handling
Fri, 18 Oct 2013 13:30:09 +0200 blanchet repair invariant in MaSh when learning new proofs
Fri, 18 Oct 2013 10:43:21 +0200 blanchet killed more "no_atp"s
Fri, 18 Oct 2013 10:43:20 +0200 blanchet killed most "no_atp", to make Sledgehammer more complete
Fri, 18 Oct 2013 10:35:57 +0200 blanchet doc fixes suggested by Andreas L.
Fri, 18 Oct 2013 10:35:56 +0200 blanchet make sure that registered code equations are actually equations
Fri, 18 Oct 2013 10:35:55 +0200 blanchet accept very long lines in MaSh
Fri, 18 Oct 2013 00:05:31 +0200 blanchet make sure add: doesn't add duplicates, and works for [no_atp] facts
Thu, 17 Oct 2013 23:41:00 +0200 blanchet no fact subsumption -- this only confuses later code, e.g. 'add:'
Thu, 17 Oct 2013 20:49:19 +0200 blanchet generate a comment storing the goal nickname in "learn_prover"
Thu, 17 Oct 2013 20:20:53 +0200 blanchet clarified message
Thu, 17 Oct 2013 20:03:37 +0200 blanchet added thread-safety warnings
Thu, 17 Oct 2013 18:53:00 +0200 blanchet avoid confusion between outer ifs and inner ifs, that caused tactic to go berserk
Thu, 17 Oct 2013 18:53:00 +0200 blanchet handle nested tuples in 'let's
Thu, 17 Oct 2013 16:45:54 +0200 nipkow more exercises
Thu, 17 Oct 2013 13:37:13 +0200 blanchet also unfold let (_, _) = ... syntax
Thu, 17 Oct 2013 11:27:53 +0200 blanchet added helper function (that solves chicken-and-egg problem w.r.t. "callssss")
Thu, 17 Oct 2013 10:29:28 +0200 blanchet graceful handling of abort
Thu, 17 Oct 2013 10:06:48 +0200 panny generalized interface
Thu, 17 Oct 2013 02:29:49 +0200 blanchet choose facts to reprove more randomly, to avoid getting stuck with impossible problems at first
Thu, 17 Oct 2013 02:22:54 +0200 blanchet thread the goal through instead of relying on unreliable (possibly fake) state
Thu, 17 Oct 2013 01:34:34 +0200 blanchet added comment
Thu, 17 Oct 2013 01:22:15 +0200 blanchet tuning
Thu, 17 Oct 2013 01:20:40 +0200 blanchet verbose minimization when learning from ATP proofs
Thu, 17 Oct 2013 01:10:08 +0200 blanchet if slicing is disabled, pick the maximum number of facts, not the number of facts in the last slice
Thu, 17 Oct 2013 01:04:00 +0200 blanchet if slicing is disabled, don't enforce last slice's "max_facts", but rather the maximum "max_facts"
Thu, 17 Oct 2013 01:03:59 +0200 blanchet fast track -- avoid domain error in 0 case
Thu, 17 Oct 2013 01:03:59 +0200 blanchet remove overloading of "max_facts" -- it already controls the number of facts passed to ATPs for 'learn_prover'
Wed, 16 Oct 2013 21:45:15 +0200 nipkow merged
Wed, 16 Oct 2013 21:44:56 +0200 nipkow tuned exercises
Wed, 16 Oct 2013 20:44:33 +0200 panny use Code.abort instead of undefined in auto-generated equations
Wed, 16 Oct 2013 19:55:23 +0200 blanchet have MaSh minimize
Tue, 15 Oct 2013 23:00:46 +0200 blanchet tweaked signature
Tue, 15 Oct 2013 22:55:01 +0200 blanchet strengthened tactic to deal with 'False ==> ...'
Tue, 15 Oct 2013 17:21:16 +0200 blanchet made theorem extraction code not delve too far when looking at local fact, by relying on 'strip_thm' instead of (wrongly) reverse-engineering proof terms
Tue, 15 Oct 2013 16:14:52 +0200 blanchet improved duplicate detection in "build_name_tables" by ensuring that the earliest occurrence of a duplicate (if it exists) gets picked as the canonical instance
Tue, 15 Oct 2013 15:31:32 +0200 blanchet updated S/H docs
Tue, 15 Oct 2013 15:31:18 +0200 blanchet use MePo with Auto Sledgehammer, because it's lighter than MaSh and always available
Tue, 15 Oct 2013 15:26:58 +0200 blanchet drop only real duplicates, not subsumed facts -- this confuses MaSh
Tue, 15 Oct 2013 11:49:39 +0100 paulson renamed relcomp_def to relcomp_unfold
Tue, 15 Oct 2013 12:25:45 +0200 nipkow fixed thm names
Tue, 15 Oct 2013 10:59:34 +0200 blanchet addressed rare case where the same symbol would be treated alternately as a function and as a predicate -- adding "top2I top_boolI" to a problem that didn't talk about "top" was a way to trigger the issue
Mon, 14 Oct 2013 11:14:14 +0200 blanchet added Nitpick limitations to docs
Mon, 14 Oct 2013 11:07:59 +0200 blanchet more defensive Nitpick setup -- exotic types of recursion are not supported yet in the model finder
Mon, 14 Oct 2013 10:55:49 +0200 blanchet keep temporary error handling in there until code equations are properly generated
Mon, 14 Oct 2013 10:50:44 +0200 blanchet tuning (simplified parts of 92c5bd3b342d)
Mon, 14 Oct 2013 10:27:16 +0200 blanchet tuning
Mon, 14 Oct 2013 10:06:03 +0200 blanchet stengthened tactic to cope with abort cases
Mon, 14 Oct 2013 09:31:42 +0200 blanchet tuned names
Mon, 14 Oct 2013 09:17:04 +0200 blanchet strengthened tactic w.r.t. "let"
Sun, 13 Oct 2013 21:36:26 +0200 blanchet more prominent MaSh errors
Fri, 11 Oct 2013 23:15:30 +0200 panny compile -- fix typo introduced in 07a8145aaeba
Fri, 11 Oct 2013 20:47:37 +0200 panny pass the right theorems to tactic
Fri, 11 Oct 2013 16:31:23 +0200 panny prove user-supplied equations for ctr and code reductions, preserving "let"s, "case"s etc.;
Thu, 10 Oct 2013 08:23:57 +0200 blanchet repaired confusion between the stated and effective fact filter -- the mismatch could result in "Match" exceptions
Thu, 10 Oct 2013 01:17:37 +0200 blanchet simplify fudge factor code
Wed, 09 Oct 2013 17:21:28 +0200 blanchet cleanup SMT-related config options
Wed, 09 Oct 2013 16:40:03 +0200 blanchet no isar proofs if preplay was not attempted
Wed, 09 Oct 2013 16:38:48 +0200 blanchet normalize more equalities
Wed, 09 Oct 2013 16:07:33 +0200 blanchet parallelize MeSh
Wed, 09 Oct 2013 15:58:02 +0200 blanchet run relevance filter only once for ATPs and SMT solvers, since it should now yield the same results anyway
Wed, 09 Oct 2013 15:39:34 +0200 blanchet use same relevance filter for ATP and SMT solvers -- attempting to filter out certain ground instances of polymorphic symbols like + and 0 has unexpected side-effects that lead to incompletenesses (relevant facts not being selected)
Wed, 09 Oct 2013 10:47:43 +0200 blanchet minor performance tuning
Wed, 09 Oct 2013 09:53:18 +0200 blanchet use plain types instead of dedicated type pattern
Wed, 09 Oct 2013 09:51:24 +0200 blanchet duplicate term and type patterns
Wed, 09 Oct 2013 09:47:59 +0200 blanchet optimized built-in const check
Wed, 09 Oct 2013 08:28:36 +0200 blanchet added TODO
Wed, 09 Oct 2013 08:12:53 +0200 blanchet crank up limit a bit -- truly huge background theories are still nearly 3 times larger
Tue, 08 Oct 2013 22:33:05 +0200 blanchet higher minimum relevance threshold, to prevent Sledgehammer from taking too long on "lemma False"
Tue, 08 Oct 2013 21:19:46 +0200 blanchet minor fact filter speedups
Tue, 08 Oct 2013 20:56:35 +0200 blanchet more gracefully handle huge theories in relevance filters
Tue, 08 Oct 2013 20:53:37 +0200 blanchet handle huge MaSh requests gracefully
Tue, 08 Oct 2013 16:40:03 +0200 blanchet further optimization in relevance filter
Tue, 08 Oct 2013 14:53:33 +0200 blanchet further speed up duplicate elimination
Tue, 08 Oct 2013 14:41:25 +0200 blanchet more efficient theorem variable normalization
Mon, 07 Oct 2013 23:44:53 +0200 blanchet strengthened constructor-view tactic to deal with 'let's
Mon, 07 Oct 2013 23:38:57 +0200 blanchet allow 'let's around constructors in constructor view
Mon, 07 Oct 2013 20:54:55 +0200 blanchet reword abstract
Mon, 07 Oct 2013 20:34:16 +0200 blanchet more primcorec docs
Mon, 07 Oct 2013 20:34:14 +0200 blanchet minor doc fix
Mon, 07 Oct 2013 08:39:50 -0700 huffman new topological lemmas; tuned proofs
Sun, 06 Oct 2013 20:54:28 +0200 blanchet strengthen the tactics to bring them in sync with the simplifications taking place in the code (and weaken the simplifications a bit -- let's not deal with implies)
Sun, 06 Oct 2013 20:24:06 +0200 blanchet generate optimized DNF formula
Sun, 06 Oct 2013 20:24:05 +0200 blanchet rationalized negation code
Sat, 05 Oct 2013 11:06:07 +0200 blanchet honor externally set MASH_PORT
Fri, 04 Oct 2013 18:27:07 +0200 panny process code-style inputs
Fri, 04 Oct 2013 17:00:35 +0200 blanchet more tracing
Fri, 04 Oct 2013 16:51:26 +0200 blanchet more thorough spying
Fri, 04 Oct 2013 16:11:19 +0200 blanchet more Sledgehammer spying -- record fact indices
Fri, 04 Oct 2013 14:35:00 +0200 blanchet prevent explosion in monomorphizer (e.g. when the facts typerep_int_def typerep_num_def typerep_option_def typerep_node_def are selected)
Fri, 04 Oct 2013 12:59:18 +0200 blanchet removed pointless special case
Fri, 04 Oct 2013 11:52:10 +0200 blanchet run fewer provers in "try" mode
Fri, 04 Oct 2013 11:28:28 +0200 blanchet count remote threads as well when balancing CPU usage -- otherwise jEdit users and other users of the "blocking" mode may have to wait for 2 * timeout if they e.g. have 4 cores and 5 provers (the typical situation)
Fri, 04 Oct 2013 11:12:28 +0200 blanchet more parallelism in blocking mode
Fri, 04 Oct 2013 09:46:08 +0200 blanchet more robustness in MaSh
Thu, 03 Oct 2013 19:01:10 +0200 wenzelm back to post-release mode -- after fork point;
Thu, 03 Oct 2013 16:32:33 +0200 wenzelm tuned;
Thu, 03 Oct 2013 16:25:40 +0200 wenzelm tuned;
Thu, 03 Oct 2013 16:15:47 +0200 wenzelm more notes;
Thu, 03 Oct 2013 16:09:47 +0200 wenzelm tuned;
Thu, 03 Oct 2013 12:34:32 +0200 nipkow added and generalised lemmas
Thu, 03 Oct 2013 00:39:16 +0200 ballarin Streamlined locales reference material.
Wed, 02 Oct 2013 23:05:36 +0200 nipkow merged
Wed, 02 Oct 2013 22:32:50 +0200 nipkow tuned
Wed, 02 Oct 2013 22:59:54 +0200 traytel merged
Wed, 02 Oct 2013 22:59:19 +0200 traytel keep the qualification of bindings when noting bnf theorems
Wed, 02 Oct 2013 22:54:42 +0200 blanchet strengthened tactic (primcorec_sel_tac) + tuning
Wed, 02 Oct 2013 22:54:42 +0200 blanchet renamings
Wed, 02 Oct 2013 22:54:42 +0200 blanchet got rid of needless argument
Wed, 02 Oct 2013 22:54:42 +0200 blanchet make SMT integration slacker w.r.t. bad apples (facts)
Wed, 02 Oct 2013 22:54:42 +0200 blanchet strengthen top sort check
Wed, 02 Oct 2013 19:49:31 +0200 wenzelm tuned whitespace;
Wed, 02 Oct 2013 19:49:15 +0200 wenzelm tuned;
Wed, 02 Oct 2013 19:43:58 +0200 wenzelm unset XMODIFIERS by default, in order to prevent total loss of key events seen on Fedora 18/19;
Wed, 02 Oct 2013 19:27:12 +0200 wenzelm updated to scala-2.10.3;
Wed, 02 Oct 2013 17:10:01 +0200 wenzelm tuned;
Wed, 02 Oct 2013 17:09:12 +0200 wenzelm some highlights of Isabelle2013-1 based on NEWS;
Wed, 02 Oct 2013 17:08:39 +0200 wenzelm tuned;
Wed, 02 Oct 2013 16:56:02 +0200 wenzelm misc tuning for release;
Wed, 02 Oct 2013 16:29:41 +0200 blanchet more (co)data docs
Wed, 02 Oct 2013 16:29:40 +0200 blanchet don't register equations of the form 'f x = ...' as simp rules, even if they are safe (noncorecursive), because they unfold too aggresively concepts users are likely to want to stay folded
Wed, 02 Oct 2013 15:53:20 +0200 traytel NEWS and CONTRIBUTORS
Wed, 02 Oct 2013 15:13:41 +0200 traytel made SML/NJ happy
Wed, 02 Oct 2013 13:29:04 +0200 traytel use new coinduction method and primcorec in examples
Wed, 02 Oct 2013 11:57:52 +0200 traytel new coinduction method
Wed, 02 Oct 2013 10:53:15 +0200 blanchet tuned command descriptions
Wed, 02 Oct 2013 10:39:01 +0200 blanchet strengthen tactic w.r.t. let
Wed, 02 Oct 2013 10:34:13 +0200 blanchet minor doc fix (there is no guarantee that the equations for a given f_i are contiguous in the collection)
Wed, 02 Oct 2013 10:15:53 +0300 kuncar typo
Wed, 02 Oct 2013 10:13:54 +0300 kuncar NEWS and CONTRIBUTORS
Tue, 01 Oct 2013 23:51:15 +0200 blanchet merged
Tue, 01 Oct 2013 23:50:35 +0200 blanchet compile -- broken since 21dac9a60f0c
Tue, 01 Oct 2013 23:36:02 +0200 blanchet strengthened tactic for right-hand sides involving lambdas
Tue, 01 Oct 2013 23:46:46 +0200 krauss basic documentation for function elimination rules and fun_cases
Tue, 01 Oct 2013 22:50:42 +0200 blanchet allow uncurried lambda-abstractions on rhs of "primcorec"
Tue, 01 Oct 2013 19:58:31 +0200 blanchet tiny doc fix
Tue, 01 Oct 2013 17:06:35 +0200 traytel base the fset bnf on the new FSet theory
Tue, 01 Oct 2013 17:04:27 +0200 traytel improved backwards compatiblity of primrec_new (Isabelle/ML interface, attributes, etc.)
Tue, 01 Oct 2013 15:02:12 +0200 blanchet removed spurious save if nothing needs to bee learned
Tue, 01 Oct 2013 14:40:25 +0200 blanchet new version of MaSh that really honors the --port option and that checks for file name mismatches
Tue, 01 Oct 2013 14:29:27 +0200 blanchet minor textual changes
Tue, 01 Oct 2013 14:13:24 +0200 blanchet got rid of dead feature
Tue, 01 Oct 2013 14:05:25 +0200 blanchet refactoring -- splitting between constructor sugar dependencies and true BNF dependencies
Tue, 01 Oct 2013 14:05:25 +0200 blanchet renamed ML files
Tue, 01 Oct 2013 14:05:25 +0200 blanchet renamed theory file
Tue, 01 Oct 2013 12:53:24 +0200 wenzelm tuned signature -- facilitate experimentation with other processes;
Mon, 30 Sep 2013 22:01:46 +0900 Christian Sternagel preserve types during rewriting
Mon, 30 Sep 2013 22:36:43 +0200 blanchet made SML/NJ happy
Mon, 30 Sep 2013 18:08:35 +0200 blanchet made SML/NJ happy
Mon, 30 Sep 2013 17:53:44 +0200 blanchet made SML/NJ happier
Mon, 30 Sep 2013 17:47:50 +0200 blanchet added experimental configuration options to tune use of builtin symbols in SMT
Mon, 30 Sep 2013 16:28:54 +0200 blanchet added possibility to reset builtins (for experimentation)
Mon, 30 Sep 2013 16:07:56 +0200 blanchet just one data slot (record) per program unit
Mon, 30 Sep 2013 15:10:18 +0200 blanchet more "primrec_new" documentation
Mon, 30 Sep 2013 14:19:33 +0200 wenzelm merged
Mon, 30 Sep 2013 14:17:27 +0200 wenzelm tuned signature;
Mon, 30 Sep 2013 13:45:17 +0200 wenzelm eliminated clone of Inductive.mk_cases_tac;
Mon, 30 Sep 2013 13:35:05 +0200 wenzelm tuned signature;
Mon, 30 Sep 2013 13:29:09 +0200 wenzelm tuned whitespace;
Mon, 30 Sep 2013 13:20:44 +0200 wenzelm provide regular ML interface and use plain Syntax.read_prop/Syntax.check_prop (update by Manuel Eberl);
Mon, 30 Sep 2013 14:04:26 +0200 blanchet merge
Mon, 30 Sep 2013 13:59:07 +0200 blanchet minor tweak to error message
Mon, 30 Sep 2013 11:20:24 +0200 wenzelm tuned;
Sun, 29 Sep 2013 18:51:01 +0200 wenzelm explicit caret position after replacement;
Sun, 29 Sep 2013 16:01:22 +0200 haftmann tuned proofs
Sun, 29 Sep 2013 14:07:47 +0200 wenzelm observe user preferences;
Sun, 29 Sep 2013 13:53:16 +0200 wenzelm updated for release;
Sun, 29 Sep 2013 12:56:50 +0200 wenzelm tuned;
Sun, 29 Sep 2013 12:49:47 +0200 wenzelm tuned;
Sun, 29 Sep 2013 12:44:40 +0200 wenzelm more on text completion;
Sun, 29 Sep 2013 12:21:11 +0200 wenzelm made SML/NJ happy (NB: toplevel ML environment is unmanaged);
Sun, 29 Sep 2013 12:18:47 +0200 wenzelm updated for release;
Sun, 29 Sep 2013 12:17:02 +0200 wenzelm updated for release;
Sun, 29 Sep 2013 11:59:01 +0200 wenzelm updated to sumatra_pdf-2.3.2;
Sun, 29 Sep 2013 11:21:02 +0200 wenzelm low-priority print task is always asynchronous -- relevant for single-core machine and automatically tried tools;
Sun, 29 Sep 2013 00:15:05 +0200 wenzelm backout c6297fa1031a -- strange parsers are required to make this work;
(0) -30000 -10000 -3000 -1000 -480 +480 +1000 +3000 +10000 tip