History log of /seL4-l4v-master/isabelle/src/HOL/Mutabelle/MutabelleExtra.thy
Revision Date Author Comments
# e60cf64d 06-Jan-2019 wenzelm <none@none>

isabelle update -u path_cartouches;


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

isabelle update -u control_cartouches;


# 17bc899d 18-Aug-2017 wenzelm <none@none>

session-qualified theory imports: isabelle imports -U -i -d '~~/src/Benchmarks' -a;


# 66281660 26-May-2016 wenzelm <none@none>

isabelle update_cartouches -c -t;


# 61fb80ee 04-May-2014 blanchet <none@none>

added 'satx' proof method to Try0


# 538e72a6 14-Mar-2014 wenzelm <none@none>

prefer more robust Synchronized.var;


# e46f39e8 12-Jul-2013 wenzelm <none@none>

system options for Isabelle/HOL proof tools;


# 3c4fbca6 31-Oct-2012 blanchet <none@none>

repaired "Mutabelle" after Refute move


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

prefer ML_file over old uses;


# e71aab02 10-Feb-2012 bulwahn <none@none>

making num_mutations a configuration that can be changed with the mutabelle bash command


# 680d93a7 11-Feb-2012 bulwahn <none@none>

making max_mutants an option that can be changed in the Mutabelle-script


# 3e4271be 27-May-2011 blanchet <none@none>

renamed "Auto_Tools" "Try"

--HG--
rename : src/Tools/auto_tools.ML => src/Tools/try.ML


# 644aabca 03-Dec-2010 blanchet <none@none>

run synchronous Auto Tools in parallel


# 14392075 22-Nov-2010 bulwahn <none@none>

adding AFP tests to Mutabelle_Extra; adopting mutabelle to recent quickcheck changes; filtering strange mutants; adding solvers to mutabelle; restructuring mutabelle


# 020b02b6 03-Nov-2010 blanchet <none@none>

standardize on seconds for Nitpick and Sledgehammer timeouts


# c2042d3e 25-Oct-2010 wenzelm <none@none>

more explicit indication of Output.Private_Hooks (still public to accomodate clones of Proof General for now);


# 93623054 25-Oct-2010 wenzelm <none@none>

renamed Output.priority to Output.urgent_message to emphasize its special role more clearly;


# 8a52405a 11-Sep-2010 blanchet <none@none>

finished renaming "Auto_Counterexample" to "Auto_Tools"


# 9e216094 25-Jan-2010 bulwahn <none@none>

adding Mutabelle to repository