History log of /seL4-l4v-10.1.1/l4v/isabelle/src/HOL/Nitpick.thy
Revision Date Author Comments
# a7ccdf43 10-Jan-2018 nipkow <none@none>

ran isabelle update_op on all sources


# c7cc1919 26-Nov-2017 wenzelm <none@none>

more symbols;


# 85b3e948 11-Nov-2017 haftmann <none@none>

dedicated definition for coprimality

--HG--
extra : rebase_source : 891168c98ce62efae6b7e72c7d3365fea12b33ae


# 00c37f50 05-Jun-2017 haftmann <none@none>

simplified setup

--HG--
extra : rebase_source : 3f48f5e2ae49ea17fb27eb23e2c7520bc75677a3


# 5f50f074 23-Apr-2017 haftmann <none@none>

include GCD as integral part of computational algebra in session HOL


# 351cc2e6 17-Oct-2016 nipkow <none@none>

setsum -> sum


# 131dfaff 15-Sep-2016 nipkow <none@none>

renamed listsum -> sum_list, listprod ~> prod_list


# 08cabf03 27-Dec-2015 wenzelm <none@none>

prefer symbols for "abs";


# 0df376fc 07-Dec-2015 wenzelm <none@none>

isabelle update_cartouches -c -t;


# 2ceb4cc9 14-Nov-2015 wenzelm <none@none>

option "inductive_defs" controls exposure of def and mono facts;


# 952abf53 06-Sep-2015 wenzelm <none@none>

do not expose low-level "_def" facts of 'function' definitions, to avoid potential confusion with the situation of plain 'definition';


# 85ed9565 01-Sep-2015 wenzelm <none@none>

eliminated \<Colon>;


# 1901affb 18-Jul-2015 wenzelm <none@none>

isabelle update_cartouches;


# 794edf80 02-Nov-2014 wenzelm <none@none>

modernized header uniformly as section;


# 1e04f9e5 16-Sep-2014 blanchet <none@none>

added 'extraction' plugins -- this might help 'HOL-Proofs'


# 6b777fb4 15-Sep-2014 blanchet <none@none>

generate 'code' attribute only if 'code' plugin is enabled


# 3c8247b0 14-Sep-2014 blanchet <none@none>

disable datatype 'plugins' for internal types


# 5fc26177 11-Sep-2014 blanchet <none@none>

updated news


# 1ba740de 02-Sep-2014 blanchet <none@none>

use 'datatype_new' in 'Main'


# 76d9c7e1 19-Aug-2014 blanchet <none@none>

tuning


# 2fde10a4 12-Jun-2014 blanchet <none@none>

tuned dependencies


# d4fd6e53 11-Jun-2014 blanchet <none@none>

reduces Sledgehammer dependencies


# 0811cf40 23-Apr-2014 blanchet <none@none>

move size hooks together, with new one preceding old one and sharing same theory data


# dd44ffb4 20-Feb-2014 blanchet <none@none>

adapted to renaming of datatype 'cases' and 'recs' to 'case' and 'rec'


# 8d680255 17-Feb-2014 blanchet <none@none>

simplified data structure by reducing the incidence of clumsy indices


# 40e0ba91 12-Feb-2014 blanchet <none@none>

renamed 'nat_{case,rec}' to '{case,rec}_nat'


# 63970edd 12-Feb-2014 blanchet <none@none>

renamed '{prod,sum,bool,unit}_case' to 'case_...'


# 67f491eb 31-Jan-2014 blanchet <none@none>

tuned ML file name

--HG--
rename : src/HOL/Tools/Nitpick/nitpick_isar.ML => src/HOL/Tools/Nitpick/nitpick_commands.ML


# 3cae1e5f 20-Jan-2014 blanchet <none@none>

compile


# 38429f1e 16-Jan-2014 blanchet <none@none>

adapted to move of Wfrec


# f55a6e4d 21-Nov-2013 blanchet <none@none>

rationalize imports


# 6d11884a 18-Oct-2013 blanchet <none@none>

killed more "no_atp"s


# 68670fb3 12-Jul-2013 wenzelm <none@none>

hybrid "auto" tool setup, for TTY (within theory) and PIDE (global print function);


# 9eff77bb 31-Oct-2012 blanchet <none@none>

moved "SAT" before "FunDef" and moved back all SAT-related ML files to where they belong


# e3227796 22-Aug-2012 wenzelm <none@none>

prefer ML_file over old uses;


# 109489f9 24-May-2012 wenzelm <none@none>

tuned proofs;


# e60dbeb1 10-May-2012 blanchet <none@none>

fixed "real" after they were redefined as a 'quotient_type'


# 870593bf 15-Mar-2012 wenzelm <none@none>

declare command keywords via theory header, including strict checking outside Pure;


# cadbf5cb 23-Jan-2012 blanchet <none@none>

added problem importer


# 90ee4884 23-Jan-2012 blanchet <none@none>

rebranded Nitrox, for more uniformity

--HG--
rename : src/HOL/TPTP/lib/Tools/nitrox => src/HOL/TPTP/lib/Tools/tptp_nitpick
rename : src/HOL/Tools/Nitpick/nitrox.ML => src/HOL/Tools/Nitpick/nitpick_tptp.ML


# e9912d13 24-Dec-2011 haftmann <none@none>

adjusted to set/pred distinction by means of type constructor `set`


# c5612a1a 13-Oct-2011 haftmann <none@none>

bouned transitive closure

--HG--
extra : rebase_source : 3d0df473619b9c72b32a96ed4951a34dd2ad6c82


# 7994d347 18-Aug-2011 haftmann <none@none>

observe distinction between sets and predicates more properly


# f9d4ee5b 01-Aug-2011 krauss <none@none>

replaced Nitpick's hardwired basic_ersatz_table by context data


# 6e5665ea 02-Aug-2011 krauss <none@none>

moved recdef package to HOL/Library/Old_Recdef.thy

--HG--
rename : src/HOL/Recdef.thy => src/HOL/Library/Old_Recdef.thy


# ffd46dad 22-Mar-2011 blanchet <none@none>

added first-order TPTP version of Nitpick to Isabelle, so that its sources stay in sync with Isabelle and it is easier to install new versions for SystemOnTPTP and CASC -- the tool is called "isabelle nitrox" but is deliberately omitted from the tool list unless the component is explicitly enabled, to avoid clutter


# 621838eb 21-Feb-2011 blanchet <none@none>

rename Nitpick's (internal) auxiliary lemmas


# 47bb2a89 21-Feb-2011 blanchet <none@none>

renamed "nitpick\_def" to "nitpick_unfold" to reflect its new semantics


# 14052b17 07-Dec-2010 blanchet <none@none>

remove the "fin_fun" optimization in Nitpick -- it was always a hack and didn't help much


# 3031f699 07-Dec-2010 blanchet <none@none>

fix special handling of set products


# 02089124 14-Sep-2010 blanchet <none@none>

remove more clutter related to old "fast_descrs" optimization


# 5b59da77 13-Sep-2010 nipkow <none@none>

renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI


# bb8268b1 07-Sep-2010 nipkow <none@none>

expand_fun_eq -> ext_iff
expand_set_eq -> set_ext_iff
Naming in line now with multisets


# ce91ae5c 06-Sep-2010 blanchet <none@none>

remove "minipick" (the toy version of Nitpick) and some tests;
a small step towards making the Nitpick tests take less time


# 4996ea41 12-Aug-2010 haftmann <none@none>

group record-related ML files


# d9e982ba 02-Jul-2010 blanchet <none@none>

adapt Nitpick to "prod_case" and "*" -> "sum" renaming;
the code in "Nitpick_Preproc", which sorted the types using "typ_ord", was wrong and evil; it seems to have worked only because "*" was called "*"


# 557987a9 11-Jun-2010 blanchet <none@none>

adjust Nitpick's handling of "<" on "rat"s and "reals"


# 4dd99738 31-May-2010 blanchet <none@none>

fix handling of "split" w.r.t. new definition + fix exception handling w.r.t. "expect" option


# 264d76c2 14-May-2010 blanchet <none@none>

add "no_atp"s to Nitpick lemmas


# 82fe7ca2 16-Apr-2010 wenzelm <none@none>

replaced generic 'hide' command by more conventional 'hide_class', 'hide_type', 'hide_const', 'hide_fact' -- frees some popular keywords;


# 7d74aa21 17-Mar-2010 blanchet <none@none>

added support for "specification" and "ax_specification" constructs to Nitpick


# 5c492097 10-Mar-2010 blanchet <none@none>

improve precision of "card" in Nitpick


# 31a982c3 09-Mar-2010 blanchet <none@none>

improved Nitpick's precision for "card" and "setsum" + fix incorrect outcome code w.r.t. "bisim_depth = -1"


# 683b5be7 09-Mar-2010 blanchet <none@none>

added "finitize" option to Nitpick + remove dependency on "Coinductive_List"


# ad9ffd9b 23-Feb-2010 blanchet <none@none>

improved Nitpick's support for quotient types


# bfcd1a37 22-Feb-2010 blanchet <none@none>

enabled Nitpick's support for quotient types + shortened the Nitpick tests a bit


# cf775f25 18-Feb-2010 blanchet <none@none>

added support for nonstandard "nat"s to Nitpick and fixed bugs in binary "nat"s and "int"s


# f9f89348 13-Feb-2010 blanchet <none@none>

more work on Nitpick's support for nonstandard models + fix in model reconstruction


# e91c3985 12-Feb-2010 blanchet <none@none>

various cosmetic changes to Nitpick


# 5d17693c 05-Feb-2010 haftmann <none@none>

more consistent naming of type classes involving orderings (and lattices) -- c.f. NEWS


# 1ee6ce9a 04-Feb-2010 blanchet <none@none>

split "nitpick_hol.ML" into two files to make it more manageable;
more refactoring to come


# 234db7fa 02-Feb-2010 blanchet <none@none>

added support for nonstandard models to Nitpick (based on an idea by Koen Claessen) and did other fixes to Nitpick


# 13ba9168 20-Jan-2010 blanchet <none@none>

fix issues with previous Nitpick change


# 5fd8634a 17-Dec-2009 blanchet <none@none>

added support for binary nat/int representation to Nitpick


# a7c13fb7 17-Nov-2009 blanchet <none@none>

bump up Nitpick's axiom/definition unfolding limits, because some real-world problems (e.g. from Boogie) ran into the previous limits;
the limits are there to prevent infinite recursion; they can be set arbitrarily high without much harm


# ef61a487 11-Nov-2009 haftmann <none@none>

tuned imports


# 7ed17ef8 28-Oct-2009 blanchet <none@none>

introduced Auto Nitpick in addition to Auto Quickcheck;
this required generalizing the theorem hook used by Quickcheck,
following a suggestion by Florian


# ce7134e9 27-Oct-2009 blanchet <none@none>

renamed Nitpick option "coalesce_type_vars" to "merge_type_vars" (shorter) and cleaned up old hacks that are no longer necessary


# 3e4102e1 27-Oct-2009 haftmann <none@none>

dropped obsolete comment


# c17e22ae 22-Oct-2009 blanchet <none@none>

added Nitpick's theory and ML files to Isabelle/HOL;
the examples and the documentation are on their way.