src/HOL/Tools/Sledgehammer/sledgehammer_atp_translate.ML
Sun, 22 May 2011 14:51:01 +0200 blanchet added support for remote Waldmeister
Fri, 20 May 2011 18:01:46 +0200 blanchet name tuning
Fri, 20 May 2011 17:16:13 +0200 blanchet further improvements to "poly_{preds,tags}_{bang,query}" -- better solution to the combinator problem + make sure type assumptions can be discharged
Fri, 20 May 2011 17:16:13 +0200 blanchet prevent unsound combinator proofs in partially typed polymorphic type systems
Fri, 20 May 2011 12:47:59 +0200 blanchet improved "poly_preds_{bang,query}" by picking up good witnesses for the possible infinity of common type classes and ensuring that "?'a::type" doesn't ruin everything
Fri, 20 May 2011 12:47:59 +0200 blanchet reintroduced type encodings "poly_preds_{bang,query}", but this time being more liberal about type variables of known safe sorts
Fri, 20 May 2011 12:47:59 +0200 blanchet automatically use "metisFT" when typed helpers are necessary
Fri, 20 May 2011 12:47:58 +0200 blanchet generate useful information for type axioms
Fri, 20 May 2011 12:47:58 +0200 blanchet slightly fewer type predicates introduced in the lightweight encoding, based on the observation that only universal positive equalities are dangerous
Thu, 19 May 2011 10:24:13 +0200 blanchet renamed "simple_types" to "simple"
Thu, 19 May 2011 10:24:13 +0200 blanchet since we always default on the "_light" encoding (for good reasons, according to Judgment Day), get rid of that suffix
Thu, 19 May 2011 10:24:13 +0200 blanchet honor "conj_sym_kind" also for tag symbol declarations
Thu, 19 May 2011 10:24:13 +0200 blanchet removed "poly_tags_light_bang" since highly unsound
Tue, 17 May 2011 15:11:36 +0200 blanchet renamed thin to light, fat to heavy
Tue, 17 May 2011 15:11:36 +0200 blanchet code cleanup, better handling of corner cases
Tue, 17 May 2011 15:11:36 +0200 blanchet implemented thin versions of "preds" type systems + fixed various issues with type args
Tue, 17 May 2011 15:11:36 +0200 blanchet renamed "shallow" to "thin" and make it the default
Tue, 17 May 2011 15:11:36 +0200 blanchet more work on "shallow" encoding + adjustments to other encodings
Tue, 17 May 2011 15:11:36 +0200 blanchet generate type classes predicates in new "shallow" encoding
Tue, 17 May 2011 15:11:36 +0200 blanchet started implementing "shallow" type systems, based on ideas by Claessen et al.
Tue, 17 May 2011 15:11:36 +0200 blanchet added syntax for "shallow" encodings
Fri, 13 May 2011 10:10:43 +0200 blanchet optimized a common case
Fri, 13 May 2011 10:10:43 +0200 blanchet avoid "UnequalLengths" exception for special constant "fequal" -- and optimize code in the common case where no type arguments are needed
Fri, 13 May 2011 10:10:43 +0200 blanchet make SML/NJ happy
Thu, 12 May 2011 15:29:19 +0200 blanchet fixed several bugs in Isar proof reconstruction, in particular w.r.t. mangled types and hAPP
Thu, 12 May 2011 15:29:19 +0200 blanchet robustly detect how many type args were passed to the ATP, even if some of them were omitted
Thu, 12 May 2011 15:29:19 +0200 blanchet make sure "simple_types_query" and "simple_types_bang" symbols are declared with the proper types
Thu, 12 May 2011 15:29:19 +0200 blanchet drop some type arguments to constants in unsound type systems + remove a few type systems that make no sense from the circulation
Thu, 12 May 2011 15:29:19 +0200 blanchet ensure Set.member isn't introduced by Meson's preprocessing if it's supposed to be unfolded
Thu, 12 May 2011 15:29:19 +0200 blanchet use the same code for extensionalization in Metis and Sledgehammer and generalize that code so that it gracefully handles negations (e.g. negated conjecture), formulas of the form (%x. t) = u, etc.
Thu, 12 May 2011 15:29:19 +0200 blanchet unfold set constants in Sledgehammer/ATP as well if Metis does it too
Thu, 12 May 2011 15:29:19 +0200 blanchet don't give weights to built-in symbols
Thu, 12 May 2011 15:29:19 +0200 blanchet gracefully declare fTrue and fFalse proxies' types if the constants only appear in the helpers
Thu, 12 May 2011 15:29:19 +0200 blanchet improve detection of quantifications over dangerous types by leveraging "is_type_surely_finite" predicate and added "prop" to the list of surely finite types
Thu, 12 May 2011 15:29:19 +0200 blanchet ensure type class predicates are generated in symbol declarations (for "poly_preds" and similar)
Thu, 12 May 2011 15:29:18 +0200 blanchet avoid "Empty" exception by making sure that a certain optimization only is attempted when it makes sense
Thu, 12 May 2011 15:29:18 +0200 blanchet renamed type systems for more consistency
Fri, 06 May 2011 13:34:59 +0200 blanchet allow each prover to specify its own formula kind for symbols occurring in the conjecture
Thu, 05 May 2011 14:04:40 +0200 blanchet reintroduce unsoundnesses taken out in 4d29b4785f43 and 3c2baf9b3c61 but only for unsound type systems
Thu, 05 May 2011 12:40:48 +0200 blanchet added FIXME
Thu, 05 May 2011 12:40:48 +0200 blanchet help SOS by ensuring that typing information is marked as part of the conjecture + be more precise w.r.t. typedefs in monotonicity check
Thu, 05 May 2011 12:40:48 +0200 blanchet query typedefs as well for monotonicity
Thu, 05 May 2011 10:24:12 +0200 blanchet hopefully this will help the SML/NJ type inference
Thu, 05 May 2011 10:16:14 +0200 blanchet reverted 6efda6167e5d because unsound -- Vampire found a counterexample
Thu, 05 May 2011 08:03:28 +0200 blanchet I have an intuition that it's sound to omit the first type arg of an hAPP -- and this reduces the size of monomorphized problems quite a bit
Thu, 05 May 2011 02:27:02 +0200 blanchet removed unsound hAPP optimization
Thu, 05 May 2011 00:51:56 +0200 blanchet versions of ! and ? for the ASCII-challenged Mirabelle
Thu, 05 May 2011 00:22:37 +0200 blanchet smoother handling of ! and ? in type system names
Wed, 04 May 2011 23:26:20 +0200 blanchet tuning
Wed, 04 May 2011 23:18:28 +0200 blanchet documentation tuning
Wed, 04 May 2011 22:56:33 +0200 blanchet renamed "many_typed" to "simple" (as in simple types)
Wed, 04 May 2011 22:47:13 +0200 blanchet added type homogenization, whereby all (isomorphic) infinite types are mapped to the same type (to reduce the number of different predicates/TFF-types)
Wed, 04 May 2011 19:35:48 +0200 blanchet exploit inferred monotonicity
Wed, 04 May 2011 15:35:05 +0200 blanchet monotonic type inference in ATP Sledgehammer problems -- based on Claessen & al.'s CADE 2011 paper, Sect. 2.3.
Wed, 04 May 2011 11:49:46 +0200 blanchet added type annotation for SML/NJ
Wed, 04 May 2011 10:12:44 +0200 blanchet eta-expansion for SML/NJ
Tue, 03 May 2011 21:46:05 +0200 blanchet cosmetics
Tue, 03 May 2011 01:04:03 +0200 blanchet no need to generate fact numbers for polymorphic type systems -- this confuses the TPTP exporter
Tue, 03 May 2011 00:10:22 +0200 blanchet replaced some Unsynchronized.refs with Config.Ts
Mon, 02 May 2011 23:01:22 +0200 blanchet do not declare TPTP built-ins, e.g. $true
less more (0) -100 -60 tip