src/HOL/Tools/Sledgehammer/sledgehammer_isar.ML
Fri, 25 Oct 2019 14:14:56 +0200 blanchet removed experimental encoding for Waldmeister
Fri, 04 Jan 2019 23:22:53 +0100 wenzelm isabelle update -u control_cartouches;
Tue, 30 Oct 2018 16:24:04 +0100 fleury add reconstruction by veriT in method smt
Fri, 20 Jul 2018 22:19:42 +0200 blanchet don't lose facts that were introduced to deal with a theory or some preprocessing in the prover (e.g. the definition of 'abs' in an SMT proof)
Thu, 01 Feb 2018 15:12:57 +0100 wenzelm tuned signature: more operations;
Sun, 14 Aug 2016 12:26:09 +0200 blanchet killed final stops in Sledgehammer and friends
Sat, 16 Jul 2016 19:35:27 +0200 wenzelm tuned signature;
Sat, 02 Apr 2016 23:29:05 +0200 wenzelm prefer infix operations;
Mon, 01 Feb 2016 20:55:23 +0100 blanchet avoid error in Isar proof reconstruction if no ATP proof is available
Mon, 29 Jun 2015 23:44:53 +0200 blanchet removed chained facts from preplaying -- and careful about extra chained facts when removing 'proof -' and 'qed' from one-line Isar proofs
Tue, 03 Mar 2015 16:37:45 +0100 blanchet SPASS-Pirate is now called Pirate
Fri, 31 Oct 2014 11:36:41 +0100 wenzelm discontinued obsolete Output.urgent_message;
Sun, 12 Oct 2014 21:52:45 +0200 blanchet improved handling of extensionality in Isar proofs generated from LEO-II and Satallax
Thu, 02 Oct 2014 18:10:09 +0200 blanchet more precise lemma insertion
Thu, 02 Oct 2014 17:40:46 +0200 blanchet insert lemmas closer to where they are needed, both for esthetics and (primarily) for correctness in case the lemma refers to a skolem
Thu, 02 Oct 2014 15:24:51 +0200 blanchet eliminate duplicate hypotheses (which can arise due to (un)clausification)
Thu, 02 Oct 2014 11:01:20 +0200 blanchet 'moura' method is also useful for reconstructing skolemization of lambda-lifting of formulas for other provers than Z3
Mon, 15 Sep 2014 14:31:32 +0200 blanchet tuning
Mon, 15 Sep 2014 12:30:06 +0200 blanchet removed accidental '@{print}'
Tue, 02 Sep 2014 16:38:26 +0200 steckerm Some work on the new waldmeister integration
Thu, 28 Aug 2014 23:57:26 +0200 blanchet renamed 'skolem' to 'moura' (to suggest Z3-style skolemization); reintroduced 'fastforce' to the mix of tested proof methods
Thu, 28 Aug 2014 16:58:27 +0200 blanchet removed show stuttering
Thu, 28 Aug 2014 16:58:27 +0200 blanchet try 'skolem' method first for Z3
Thu, 28 Aug 2014 16:58:27 +0200 blanchet added 'skolem' method, esp. for 'obtain's generated from Z3 proofs
Thu, 28 Aug 2014 00:40:38 +0200 blanchet renamed new SMT module from 'SMT2' to 'SMT'
Tue, 05 Aug 2014 10:59:40 +0200 blanchet rationalize Skolem names
Tue, 05 Aug 2014 10:17:15 +0200 blanchet tuning
Tue, 05 Aug 2014 09:20:00 +0200 blanchet tuning
Mon, 04 Aug 2014 16:53:09 +0200 blanchet deal with E definitions
Mon, 04 Aug 2014 15:02:02 +0200 blanchet cleaner 'compress' option
Mon, 04 Aug 2014 13:16:18 +0200 blanchet tuned terminology (cf. 'isar_proofs' option)
Mon, 04 Aug 2014 12:28:42 +0200 blanchet rationalized sorting of facts -- so that preplaying (almost always) coincides with the real thing, preventing odd failures
Sat, 02 Aug 2014 00:15:08 +0200 blanchet better duplicate detection
Fri, 01 Aug 2014 23:58:42 +0200 blanchet normalize conjectures vs. negated conjectures when comparing terms
Fri, 01 Aug 2014 23:33:43 +0200 blanchet tweaked 'clone' formula detection
Fri, 01 Aug 2014 23:29:50 +0200 blanchet fine-tuned Isar reconstruction, esp. boolean simplifications
Fri, 01 Aug 2014 23:29:49 +0200 blanchet centralized boolean simplification so that e.g. LEO-II benefits from it
Fri, 01 Aug 2014 20:44:29 +0200 blanchet better handling of variable names
Fri, 01 Aug 2014 20:08:50 +0200 blanchet nicer generated variable names
Fri, 01 Aug 2014 19:44:18 +0200 blanchet tuning
Fri, 01 Aug 2014 19:36:23 +0200 blanchet tuning
Fri, 01 Aug 2014 19:32:10 +0200 blanchet more precise handling of LEO-II skolemization
Fri, 01 Aug 2014 16:07:34 +0200 blanchet beware of 'skolem' rules that do not skolemize (e.g. LEO-II)
Fri, 01 Aug 2014 14:43:57 +0200 blanchet added appropriate method for skolemization of Z3 steps to the mix
Fri, 01 Aug 2014 14:43:57 +0200 blanchet tentatively took out 'fastforce' from the set of tried methods -- it seems to be largely subsumed and is hard to silence
Fri, 01 Aug 2014 14:43:57 +0200 blanchet tuning
Fri, 01 Aug 2014 14:43:57 +0200 blanchet eliminated Sledgehammer's "min" subcommand (and lots of complications in the code)
Wed, 30 Jul 2014 14:03:13 +0200 fleury Skolemization for tmp_ite_elim rule in the SMT solver veriT.
Wed, 30 Jul 2014 14:03:13 +0200 fleury Changing the role of rule "tmp_ite_elim" of the SMT solver veriT to Lemma.
Wed, 30 Jul 2014 14:03:13 +0200 fleury Whitespace and indentation correction.
Wed, 30 Jul 2014 14:03:12 +0200 fleury imported patch hilbert_choice_support
Wed, 30 Jul 2014 14:03:12 +0200 fleury veriT changes for lifted terms, and ite_elim rules.
Wed, 30 Jul 2014 14:03:12 +0200 fleury Subproofs for the SMT solver veriT.
Wed, 30 Jul 2014 14:03:12 +0200 fleury Basic support for the SMT prover veriT.
Wed, 30 Jul 2014 14:03:11 +0200 fleury Skolemization support for leo-II and Zipperposition.
Wed, 30 Jul 2014 00:50:41 +0200 blanchet also try 'metis' with 'full_types'
Thu, 24 Jul 2014 18:46:38 +0200 blanchet refined filter for ATP steps to avoid 'have True' steps in E proofs
Thu, 24 Jul 2014 18:46:38 +0200 blanchet 'shift_quantors' is not an E skolemization rule (cf. 3ab503b04bdb)
Tue, 24 Jun 2014 08:19:22 +0200 blanchet supports gradual skolemization (cf. Z3) by threading context through correctly
Tue, 24 Jun 2014 08:19:22 +0200 blanchet given two one-liners, only show the best of the two
less more (0) -300 -100 -60 tip