src/HOL/Mirabelle/Tools/mirabelle.ML
Thu, 03 Mar 2016 15:23:02 +0100 wenzelm clarified modules;
Sun, 13 Dec 2015 21:56:15 +0100 wenzelm more general types Proof.method / context_tactic;
Tue, 02 Jun 2015 10:12:46 +0200 wenzelm clarified context;
Sat, 15 Mar 2014 11:59:18 +0100 wenzelm tuned signature;
Wed, 02 May 2012 11:47:45 +0200 wenzelm updated headers;
Tue, 24 Apr 2012 13:59:29 +0100 sultana reversed Tools to Actions Mirabelle renaming;
Fri, 08 Jul 2011 17:04:38 +0200 wenzelm discontinued odd Position.column -- left-over from attempts at PGIP implementation;
Mon, 02 May 2011 16:33:21 +0200 wenzelm added Attrib.setup_config_XXX conveniences, with implicit setup of the background theory;
Sun, 20 Mar 2011 22:08:12 +0100 wenzelm simplified various cpu_time clones (!): eliminated odd Exn.capture/Exn.release (no need to "stop" timing);
Sun, 20 Mar 2011 21:28:11 +0100 wenzelm structure Timing: covers former start_timing/end_timing and Output.timeit etc;
Sun, 09 Jan 2011 12:56:00 +0100 wenzelm refined comment (again);
Sat, 08 Jan 2011 17:14:48 +0100 wenzelm misc tuning and comments based on review of Theory_Data, Proof_Data, Generic_Data usage;
Mon, 20 Sep 2010 16:05:25 +0200 wenzelm renamed structure PureThy to Pure_Thy and moved most content to Global_Theory, to emphasize that this is global-only;
Thu, 16 Sep 2010 09:59:32 +0200 blanchet prevent exception when calling "Mirabelle.can_apply" on empty proof sequence;
Tue, 14 Sep 2010 23:38:36 +0200 blanchet tuning
Thu, 09 Sep 2010 17:20:27 +0200 wenzelm more abstract treatment of interrupts in structure Exn -- hardly ever need to mention Interrupt literally;
Mon, 10 May 2010 20:53:06 +0200 wenzelm renamed Config.get_thy to Config.get_global etc. to indicate that this is not the real thing;
Sun, 28 Mar 2010 16:59:06 +0200 wenzelm static defaults for configuration options;
Fri, 05 Mar 2010 23:51:32 +0100 wenzelm use regular Proof.goal (which is what methods usually see) and prevent sledgehammer from crashing;
Thu, 10 Dec 2009 18:10:59 +0100 boehmes only invoke metisFT if metis failed
Tue, 08 Dec 2009 23:05:23 +0100 boehmes also consider the fully-typed version of metis for Mirabelle measurements
Sun, 08 Nov 2009 18:43:42 +0100 wenzelm adapted Theory_Data;
Wed, 28 Oct 2009 22:18:00 +0100 wenzelm renamed raw Proof.get_goal to Proof.raw_goal;
Tue, 27 Oct 2009 17:34:00 +0100 wenzelm normalized basic type abbreviations;
Thu, 24 Sep 2009 17:25:42 +0200 nipkow record how many "proof"s are solved by s/h
Sun, 13 Sep 2009 02:10:41 +0200 wenzelm explicitly export type abbreviations (as usual in SML97);
Sat, 12 Sep 2009 16:30:48 +0200 wenzelm standard headers and text sections;
Thu, 10 Sep 2009 15:57:55 +0200 nipkow position information is now passed to all actions;
Sat, 05 Sep 2009 11:45:57 +0200 boehmes added initialization and cleanup of actions,
Thu, 03 Sep 2009 22:47:31 +0200 boehmes Mirabelle: actions are responsible for catching exceptions and producing suitable log messages (makes log message uniform),
Thu, 03 Sep 2009 14:31:04 +0200 boehmes replaced backlist by whitelist
Thu, 03 Sep 2009 14:05:13 +0200 boehmes Mirabelle: logging of exceptions (works only for PolyML)
Wed, 02 Sep 2009 21:31:58 +0200 boehmes Mirabelle: actions are responsible for handling exceptions,
Wed, 02 Sep 2009 16:29:50 +0200 boehmes removed errors overseen in previous changes
Wed, 02 Sep 2009 16:23:53 +0200 boehmes moved Mirabelle from HOL/Tools to HOL,
less more (0) tip