History log of /seL4-l4v-master/l4v/isabelle/src/HOL/Tools/Sledgehammer/sledgehammer_fact.ML
Revision Date Author Comments
# 44a31568 29-Nov-2019 wenzelm <none@none>

more informative spec rules: optional name;
clarified signature;
more thorough treatment of Thm.trim_context vs. Thm.transfer;


# 8349f97b 26-Mar-2019 wenzelm <none@none>

clarified signature: avoid direct comparison on type rough_classification;


# ed7a971e 05-Jan-2019 wenzelm <none@none>

isabelle update -u control_cartouches;


# a4bab154 04-Jan-2019 wenzelm <none@none>

isabelle update -u control_cartouches;


# 8aec7217 01-Feb-2018 wenzelm <none@none>

tuned signature: more operations;


# bf408fd1 07-Sep-2017 blanchet <none@none>

better duplicate detection


# 151b7ea2 10-Apr-2017 wenzelm <none@none>

tuned signature;


# 8aafd76b 26-Oct-2016 blanchet <none@none>

tuning


# d2aee004 21-Jun-2016 wenzelm <none@none>

position information for literal facts;
Markup.entry may have empty kind/name;


# c8a3ab07 05-Mar-2016 wenzelm <none@none>

tuned signature -- clarified modules;

--HG--
rename : src/Pure/Concurrent/time_limit.ML => src/Pure/Concurrent/timeout.ML


# 3115ef63 07-Jan-2016 wenzelm <none@none>

tuned signature;


# 4216bc36 07-Jan-2016 wenzelm <none@none>

more uniform treatment of package internals;


# 49773b00 20-Dec-2015 wenzelm <none@none>

renamed Pretty.str_of to Pretty.unformatted_string_of to emphasize its meaning;


# 91d2949f 12-Nov-2015 blanchet <none@none>

use cartouches instead of backquotes


# c3050b46 04-Oct-2015 blanchet <none@none>

speed up MaSh duplicate check


# 3b32ede6 30-Aug-2015 wenzelm <none@none>

trim context for persistent storage;


# 02f6d501 16-Aug-2015 wenzelm <none@none>

prefer theory_id operations;
tuned signature;


# a455fa51 16-Aug-2015 wenzelm <none@none>

clarified context;


# c05194cb 16-Aug-2015 wenzelm <none@none>

tuned signature;


# 1971a62a 13-Aug-2015 wenzelm <none@none>

tuned signature, in accordance to sortBy in Scala;


# 832cfa8b 11-Jun-2015 wenzelm <none@none>

support for 'consider' command;
allow full "fixes" for 'obtain' command;
tuned signature;


# 62dbb4e4 03-May-2015 blanchet <none@none>

improved one-line preplaying (don't rely on 'using x by simp' to mean 'by (simp add: x)' and beware of inaccessible '(local.)this')


# cff2e75b 08-Apr-2015 wenzelm <none@none>

proper context for Object_Logic operations;


# 4d247bc0 03-Apr-2015 wenzelm <none@none>

tuned;


# b19fa3e5 01-Apr-2015 wenzelm <none@none>

tuned signature;


# 4e1305ff 19-Mar-2015 wenzelm <none@none>

more position information;


# 34035ccd 04-Mar-2015 wenzelm <none@none>

tuned signature -- prefer qualified names;


# de3fa953 24-Jan-2015 wenzelm <none@none>

tuned signature;


# 13ddea91 26-Nov-2014 wenzelm <none@none>

renamed "pairself" to "apply2", in accordance to @{apply 2};


# c12ca051 07-Nov-2014 wenzelm <none@none>

plain value Keywords.keywords, which might be used outside theory for bootstrap purposes;
plain value Outer_Syntax within theory: parsing requires current theory context;
clarified name of Keyword.is_literal according to its semantics;
eliminated pointless type Keyword.T;
simplified @{command_spec};
clarified bootstrap keywords and syntax: take it as basis instead of side-branch;


# 514ac706 06-Nov-2014 wenzelm <none@none>

prefer explicit Keyword.keywords;


# f32dbf7c 08-Sep-2014 blanchet <none@none>

never include hidden names -- these cannot be referenced afterward


# 998f7f3a 28-Aug-2014 blanchet <none@none>

gracefully reconstruct Isar proofs in scenarios such as 'using f unfolding g', where backticks can't be used to refer to the unfolded version of 'f' (for some reason)


# d65030e5 19-Aug-2014 wenzelm <none@none>

tuned signature -- moved type src to Token, without aliases;


# 6fb4e52a 18-Aug-2014 blanchet <none@none>

reordered some (co)datatype property names for more consistency


# 244127cb 16-Aug-2014 wenzelm <none@none>

updated to named_theorems;


# 493ee8ab 01-Jul-2014 blanchet <none@none>

added hidden check to Sledgehammer fact filters, to avoid picking up facts like 'Nat.nat_induct0'


# 361b2791 01-Jul-2014 blanchet <none@none>

whitespace tuning


# 1721e8a7 01-Aug-2014 blanchet <none@none>

whitespace tuning


# d71c1002 01-Aug-2014 blanchet <none@none>

remove YXML formatting when parsing backquoted facts supplied manually to Sledgehammer


# 59521cea 01-Aug-2014 blanchet <none@none>

generate backquotes without markup, since this confuses preplay; bump up spying version identifier;


# 66fc1073 28-May-2014 blanchet <none@none>

more generous max number of suggestions, for more safety


# 2c8d6176 21-Mar-2014 wenzelm <none@none>

more qualified names;


# c99db3d6 15-Mar-2014 wenzelm <none@none>

more explicit treatment of verbose mode, which includes concealed entries;


# 51e19a6b 13-Mar-2014 wenzelm <none@none>

back to a form of hybrid facts, to reduce performance impact of ed92ce2ac88e;


# 7d65fe17 14-Mar-2014 wenzelm <none@none>

just one cumulative Proof_Context.facts, with uniform retrieval (including PIDE markup, completion etc.);
more thorough background_notes: distribute global notes to all contexts;


# f3fa700b 10-Mar-2014 wenzelm <none@none>

clarified Args.check_src: retain name space information for error output;
tuned signature;


# f1c9f8a2 10-Mar-2014 wenzelm <none@none>

prefer Name_Space.pretty with its builtin markup;


# e8872587 06-Mar-2014 wenzelm <none@none>

tuned signature;


# 70573b75 03-Feb-2014 blanchet <none@none>

tuning


# fed5d9bd 31-Jan-2014 blanchet <none@none>

tuning


# e423e659 26-Jan-2014 wenzelm <none@none>

tuned signature;


# b96e01d8 25-Jan-2014 wenzelm <none@none>

explicit eigen-context for attributes "where", "of", and corresponding read_instantiate, instantiate_tac;


# 8e00c5e5 02-Jan-2014 blanchet <none@none>

removed pointless warning (cf. http://stackoverflow.com/questions/20233463/isabelle-metis-proof-state-contains-the-universal-sort/20785045#20785045)


# 7ff3b5f2 19-Nov-2013 blanchet <none@none>

tuning


# fb3c73e4 17-Oct-2013 blanchet <none@none>

make sure add: doesn't add duplicates, and works for [no_atp] facts


# 8219bdec 17-Oct-2013 blanchet <none@none>

no fact subsumption -- this only confuses later code, e.g. 'add:'


# f3876dad 15-Oct-2013 blanchet <none@none>

drop only real duplicates, not subsumed facts -- this confuses MaSh


# 66c84939 09-Oct-2013 blanchet <none@none>

normalize more equalities


# ce476bdf 09-Oct-2013 blanchet <none@none>

added TODO


# ee0bcba1 09-Oct-2013 blanchet <none@none>

crank up limit a bit -- truly huge background theories are still nearly 3 times larger


# 3e582261 08-Oct-2013 blanchet <none@none>

minor fact filter speedups


# 63a3ad58 08-Oct-2013 blanchet <none@none>

more gracefully handle huge theories in relevance filters


# 3eedeca5 08-Oct-2013 blanchet <none@none>

further optimization in relevance filter


# 711bce40 08-Oct-2013 blanchet <none@none>

further speed up duplicate elimination


# aacc67c9 08-Oct-2013 blanchet <none@none>

more efficient theorem variable normalization


# b67710bb 02-Oct-2013 blanchet <none@none>

strengthen top sort check


# 5aada480 24-Sep-2013 blanchet <none@none>

encode goal digest in spying log (to detect duplicates)


# 26551d29 11-Sep-2013 blanchet <none@none>

reintroduced 8d8f72aa5c0b, which does make a small difference in practice, but implemented more efficiently


# fb4c22a6 11-Sep-2013 blanchet <none@none>

tuning


# 9d79372b 11-Sep-2013 blanchet <none@none>

disable some checks for huge background theories


# 37f4eea4 11-Sep-2013 blanchet <none@none>

tuning


# ee05c6f9 11-Sep-2013 blanchet <none@none>

reintroduced half of f99ee3adb81d -- that part definitely looks useless (and is inefficient)


# 9933ec9f 11-Sep-2013 blanchet <none@none>

reverted f99ee3adb81d -- that old logic seems to make a difference still today


# 1a93ebe1 10-Sep-2013 blanchet <none@none>

faster detection of tautologies


# f988c22b 10-Sep-2013 blanchet <none@none>

slight speed optimization


# bb8f38b1 10-Sep-2013 blanchet <none@none>

got rid of another slowdown factor in relevance filter


# 66959d0f 10-Sep-2013 blanchet <none@none>

removed completely needless, inefficient code


# 5dd6ca03 10-Sep-2013 blanchet <none@none>

minor speed optimization


# 0fff0bb1 10-Sep-2013 blanchet <none@none>

got rid of another taboo that appears to make no difference in practice (and that slows down the relevance filter)


# e733f861 10-Sep-2013 blanchet <none@none>

avoid double traversal of term


# b08aded7 10-Sep-2013 blanchet <none@none>

got rid of old, needless logic


# f03638fd 10-Sep-2013 blanchet <none@none>

faster uniquification


# aa30babb 10-Sep-2013 blanchet <none@none>

stronger fact normalization


# a6d539a9 10-Sep-2013 blanchet <none@none>

gracefully handle huge thys


# 46787ca7 10-Sep-2013 blanchet <none@none>

speed up detection of simp rules


# e232176f 16-May-2013 blanchet <none@none>

tuning -- renamed '_from_' to '_of_' in Sledgehammer


# 801d585a 15-May-2013 blanchet <none@none>

renamed Sledgehammer functions with 'for' in their names to 'of'


# 963a5558 15-Feb-2013 haftmann <none@none>

systematic conversions between nat and nibble/char;
more uniform approaches to execute operations on nibble/char

--HG--
extra : rebase_source : 982810ecce9e31070e2293715ed744c3b68ae21d


# 8e65386b 14-Feb-2013 haftmann <none@none>

reform of predicate compiler / quickcheck theories:
implement yieldn operations uniformly on the ML level -- predicate compiler uses negative integers as parameter to yieldn, whereas code_numeral represents natural numbers!
avoid odd New_ prefix by joining related theories;
avoid overcompact name DSequence;
separated predicate inside random monad into separate theory;
consolidated name of theory Quickcheck

--HG--
rename : src/HOL/DSequence.thy => src/HOL/Limited_Sequence.thy
rename : src/HOL/Quickcheck.thy => src/HOL/Quickcheck_Random.thy
extra : rebase_source : b6adaac1637d6d1cc809d2f937ae890fcc21969c


# 7cfd79bb 31-Jan-2013 blanchet <none@none>

distinguish raw and non-raw facts, using raw for 10 000s of facts and non-raw after selection of some hundreds


# ecec4e04 10-Jan-2013 blanchet <none@none>

make name table work the way it was intended to


# 4aa0a038 06-Jan-2013 blanchet <none@none>

put single-theorem names before multi-theorem ones (broken since 5d147d492792)


# 3535180a 05-Jan-2013 blanchet <none@none>

tuned blacklisting in relevance filter


# 8bc46745 04-Jan-2013 blanchet <none@none>

refined class handling, to prevent cycles in fact graph


# d8ad6642 04-Jan-2013 blanchet <none@none>

learn from low-level, inside-class facts


# 756a23f3 04-Jan-2013 blanchet <none@none>

tuning


# 67d06f43 17-Dec-2012 blanchet <none@none>

add a timeout in induction rule instantiation


# cb3ebf41 13-Dec-2012 blanchet <none@none>

get rid of some junk facts in the MaSh evaluation driver


# d2446a36 12-Dec-2012 blanchet <none@none>

tweaked which facts are included for MaSh evaluations


# 0ca072f5 12-Dec-2012 blanchet <none@none>

don't query blacklisted theorems in evaluation driver


# ca29b8f9 12-Dec-2012 blanchet <none@none>

export a pair of ML functions


# c919dab0 12-Dec-2012 blanchet <none@none>

further fix related to bd9a0028b063 -- that change was per se right, but it exposed a bug in the pattern for "all"


# 700a5cb2 12-Dec-2012 blanchet <none@none>

better tautology check -- don't reject "prod_cases3" for example


# ef9bd58c 12-Dec-2012 blanchet <none@none>

really all facts means really all facts (well, almost)


# d69c4158 11-Dec-2012 blanchet <none@none>

merge aliased theorems in MaSh dependencies, modulo symmetry of equality


# a0ee077f 11-Dec-2012 blanchet <none@none>

push normalization further -- avoid theorems that are duplicates of each other except for equality symmetry (esp. for "list.distinct(1)" vs. "(2)" etc.)


# 783dbf3f 08-Dec-2012 blanchet <none@none>

don't blacklist "case" theorems -- this causes problems in MaSh later


# 9336ad82 26-Nov-2012 wenzelm <none@none>

tuned signature;
tuned;


# cd384aa1 12-Nov-2012 blanchet <none@none>

fixed detection of tautologies -- things like "a = b" in a structured proof, where a and b are Frees, shouldn't be discarted as tautologies


# 559bb011 11-Nov-2012 blanchet <none@none>

avoid messing too much with output of "string_of_term", so that it doesn't break the yxml encoding for jEdit


# da40a1e3 12-Nov-2012 blanchet <none@none>

centralized term printing code


# d2ae4adc 12-Nov-2012 blanchet <none@none>

thread context correctly when printing backquoted facts


# 8029df66 31-Oct-2012 blanchet <none@none>

tuning


# ea994514 03-Aug-2012 blanchet <none@none>

rule out same "technical" theories for MePo as for MaSh


# 3da5b468 26-Jul-2012 blanchet <none@none>

repaired accessibility chains generated by MaSh exporter + tuned one function out


# 0495263b 23-Jul-2012 blanchet <none@none>

identified "evil" theories for MaSh -- this is rather ad hoc, but so is MaSh anyway


# f6a57450 23-Jul-2012 blanchet <none@none>

distinguish between recursive and nonrecursive definitions + clean up typedef dependencies in MaSh


# fd897859 23-Jul-2012 blanchet <none@none>

tuning


# 84aa75b1 20-Jul-2012 blanchet <none@none>

honor suggested MaSh weights


# caae738e 20-Jul-2012 blanchet <none@none>

minimal maxes + tuning


# 01cb6c78 20-Jul-2012 blanchet <none@none>

name tuning


# d2a5a3b6 20-Jul-2012 blanchet <none@none>

fixed various issues with MaSh's file handling + tune output + generate local facts again + handle nameless facts gracefully


# 8352d0ae 18-Jul-2012 blanchet <none@none>

optimize parent computation in MaSh + remove temporary files


# 7c2da977 18-Jul-2012 blanchet <none@none>

don't include hidden facts in relevance filter + tweak MaSh learning


# 09931ce3 18-Jul-2012 blanchet <none@none>

centrally construct expensive data structures


# b2783e64 18-Jul-2012 blanchet <none@none>

more work on MaSh


# c50c8e4f 18-Jul-2012 blanchet <none@none>

gracefully handle the case of empty theories when going up the accessibility chain


# 928cadab 18-Jul-2012 blanchet <none@none>

more code rationalization in relevance filter


# 6e993fb8 11-Jul-2012 blanchet <none@none>

moved most of MaSh exporter code to Sledgehammer


# a74b00cb 11-Jul-2012 blanchet <none@none>

further ML structure split to permit finer-grained loading/reordering (problem to solve: MaSh needs most of Sledgehammer)