Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-224
+224
+1000
+3000
+10000
+30000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
adding values to show and ensure that values works with complex terms and restores numerals on natural numbers
2010-09-16, by bulwahn
adding restoring of numerals for natural numbers for values command
2010-09-16, by bulwahn
values command for prolog supports complex terms and not just variables
2010-09-16, by bulwahn
adapting examples
2010-09-16, by bulwahn
registering code_prolog as component; using environment variable; adding settings file for prolog code generation
2010-09-16, by bulwahn
adding mode inference to prolog compilation; separate between (ad-hoc) code modifications and system_configuration; adapting quickcheck
2010-09-16, by bulwahn
merged
2010-09-16, by paulson
tidied a few proofs
2010-09-16, by paulson
merged
2010-09-16, by blanchet
avoid code duplication
2010-09-16, by blanchet
tuning
2010-09-16, by blanchet
merge constructors
2010-09-16, by blanchet
factor out the inverse of "nice_atp_problem"
2010-09-16, by blanchet
use the same TSTP/Vampire/SPASS parser for one-liners as for Isar proofs
2010-09-16, by blanchet
factored out TSTP/SPASS/Vampire proof parsing;
2010-09-16, by blanchet
prevent exception when calling "Mirabelle.can_apply" on empty proof sequence;
2010-09-16, by blanchet
supply the Metis parameter defaults as argument, instead of patching the Metis sources;
2010-09-16, by blanchet
regenerated "metis.ML"
2010-09-16, by blanchet
streamlined "make_metis"
2010-09-16, by blanchet
put Isabelle-specifics in a "PortableIsabelle" file maintained by us;
2010-09-16, by blanchet
handy little script
2010-09-16, by blanchet
reintroduce missing "critical"s by hand
2010-09-16, by blanchet
MIT license -> BSD License
2010-09-16, by blanchet
copied the unmodified official Metis 2.3 (15 Sept. 2010) sources into Isabelle
2010-09-16, by blanchet
tuned;
2010-09-17, by wenzelm
allow embedded reports in regular prover messages, to avoid side-effects for errors for example;
2010-09-17, by wenzelm
simplified/clarified (Context_)Position.markup/reported_text;
2010-09-17, by wenzelm
eliminated markup "location" in favour of more explicit "no_report", which is actually deleted from messages;
2010-09-17, by wenzelm
Isar "default" step needs to fail for solved problems, for clear distinction of '.' and '..' for example -- amending lapse introduced in 9de4d64eee3b (April 2004);
2010-09-16, by wenzelm
updated generated file;
2010-09-16, by wenzelm
tuned whitespace
2010-09-16, by haftmann
reverse order of datatype declarations so that declarations only depend on already declared datatypes
2010-09-16, by boehmes
merged
2010-09-15, by blanchet
make "metis.ML" building process slightly more robust by eliminating the need for "FILES";
2010-09-15, by blanchet
dropped obsolete src/Tools/random_word.ML -- superseded by src/Tools/Metis/src/Random.sml stemming from the Metis distribution;
2010-09-15, by wenzelm
merged
2010-09-15, by blanchet
document Metis updating procedure
2010-09-15, by blanchet
move "CRITICAL" to "PortableXxx", where it belongs and used to be;
2010-09-15, by blanchet
regenerated "metis.ML"
2010-09-15, by blanchet
update comment
2010-09-15, by blanchet
make "Unprotected concurrency introduces some true randomness." be true;
2010-09-15, by blanchet
fix parsing of higher-order formulas;
2010-09-15, by blanchet
merged
2010-09-15, by haftmann
load code_runtime immediately again
2010-09-15, by haftmann
proper interface for code_reflect
2010-09-15, by haftmann
introduced "holds" as synthetic datatype constructor for "prop"; moved Pure code generator setup to Code_Generator.thy
2010-09-15, by haftmann
merged
2010-09-15, by blanchet
"Metis." -> "Metis_" to reflect change in "metis.ML"
2010-09-15, by blanchet
no need for "metis_env.ML" anymore;
2010-09-15, by blanchet
regenerate "metis.ML", this time without manual hacks
2010-09-15, by blanchet
remove needless file for us
2010-09-15, by blanchet
got rid of three crude regexps from "make_metis"
2010-09-15, by blanchet
more Isabelle-specific changes
2010-09-15, by blanchet
tuning
2010-09-15, by blanchet
rename
2010-09-15, by blanchet
use "Metis_" prefix rather than "Metis" structure;
2010-09-15, by blanchet
no need for TPTP
2010-09-15, by blanchet
put "foldl" and "foldr" in "Useful";
2010-09-15, by blanchet
reintroduce the CRITICAL sections from change 3880d21d6013
2010-09-15, by blanchet
apply Larry's hacks directly to the "src" files;
2010-09-15, by blanchet
"FILES" is not (anymore?) part of the official Metis sources, so move it up
2010-09-15, by blanchet
merged
2010-09-15, by wenzelm
Code_Runtime.value, corresponding to ML_Context.value; tuned
2010-09-15, by haftmann
Code_Runtime.value, corresponding to ML_Context.value
2010-09-15, by haftmann
more accurate dependencies
2010-09-15, by haftmann
code_eval renamed to code_runtime
2010-09-15, by haftmann
merged
2010-09-15, by wenzelm
static nbe conversion
2010-09-15, by haftmann
ignore code cache optionally; corrected scope of term value in static_eval_conv
2010-09-15, by haftmann
ignore code cache optionally
2010-09-15, by haftmann
dropped redundant normal_form command
2010-09-15, by haftmann
more explicit theory name
2010-09-15, by haftmann
more accurate dependencies
2010-09-15, by haftmann
merged
2010-09-15, by haftmann
more clear separation of static compilation and dynamic evaluation
2010-09-15, by haftmann
Document.async_state: some attempts to make this more robust wrt. cancelation of the main transaction -- avoid confusing feedback about pending forks;
2010-09-15, by wenzelm
isatest: reactivated kodkodi and thus HOL-Nitpick_Examples -- being now on a local file system greatly increases the chance that it works;
2010-09-15, by wenzelm
merged
2010-09-15, by haftmann
replaced ML_Context.evaluate by ML_Context.value -- using context data instead of bare metal references
2010-09-15, by haftmann
replaced ML_Context.evaluate by ML_Context.value -- using context data instead of bare metal references; tuned structures
2010-09-15, by haftmann
merge
2010-09-15, by blanchet
compile on SML/NJ
2010-09-15, by blanchet
in debug mode, don't touch "$true" and "$false"
2010-09-15, by blanchet
adding option show_invalid_clauses for a more detailed message when modes are not inferred
2010-09-15, by bulwahn
proposed modes for code_pred now supports modes for mutual predicates
2010-09-15, by bulwahn
merged
2010-09-15, by haftmann
established emerging canonical names *_eqI and *_eq_iff
2010-09-13, by haftmann
moved lemmas map_of_eqI and map_of_eq_dom to Map.thy
2010-09-13, by haftmann
more precise name for activation of improveable syntax
2010-09-13, by haftmann
tuning
2010-09-14, by blanchet
tuning
2010-09-14, by blanchet
prefer version 0.6 of Vampire, now that we can parse its output
2010-09-14, by blanchet
fix splitting of proof lines for one-line metis calls;
2010-09-14, by blanchet
finish support for E 1.2 proof reconstruction;
2010-09-14, by blanchet
first step in generalizing to nonnumeric proof step names (e.g. remote Vampire 0.6)
2010-09-14, by blanchet
clarify message
2010-09-14, by blanchet
use same hack as in "Async_Manager" to work around Proof General bug
2010-09-14, by blanchet
export function
2010-09-14, by blanchet
generalize proof reconstruction code;
2010-09-14, by blanchet
tuning
2010-09-14, by blanchet
handle relevance filter corner cases more gracefully;
2010-09-14, by blanchet
remove more clutter related to old "fast_descrs" optimization
2010-09-14, by blanchet
Sledgehammer should be called in "prove" mode;
2010-09-14, by blanchet
added a timeout around "try" call in Mirabelle
2010-09-14, by blanchet
adapt examples to latest Nitpick changes + speed them up a little bit
2010-09-14, by blanchet
tuning
2010-09-14, by blanchet
eliminate more clutter related to "fast_descrs" optimization
2010-09-14, by blanchet
remove "fast_descs" option from Nitpick;
2010-09-14, by blanchet
fixed bug in the "fast_descrs" optimization;
2010-09-14, by blanchet
speed up helper function
2010-09-14, by blanchet
tuning
2010-09-14, by blanchet
rename internal Sledgehammer constant
2010-09-14, by blanchet
merged
2010-09-14, by blanchet
merged
2010-09-13, by blanchet
adapt to latest Metis version
2010-09-13, by blanchet
regenerated "metis.ML" and reintroduced Larry's old hacks manually;
2010-09-13, by blanchet
update scripts
2010-09-13, by blanchet
change license, with Joe Hurd's permission
2010-09-13, by blanchet
new version of the Metis files
2010-09-13, by blanchet
remove old sources
2010-09-13, by blanchet
remove "atoms" from the list of options with default values
2010-09-13, by blanchet
remove unreferenced identifiers
2010-09-13, by blanchet
make Auto Nitpick go through fewer scopes
2010-09-13, by blanchet
move equation up where it's not ignored
2010-09-13, by blanchet
correctly thread parameter through
2010-09-13, by blanchet
indicate triviality in the list of proved things
2010-09-13, by blanchet
indicate which goals are trivial
2010-09-13, by blanchet
tuning
2010-09-13, by blanchet
tuning
2010-09-13, by blanchet
keep track of trivial vs. nontrivial calls using "try" for 30 seconds
2010-09-13, by blanchet
change signature of "Try.invoke_try" to make it more flexible
2010-09-13, by blanchet
use 30 s instead of 60 s as the default Sledgehammer timeout;
2010-09-13, by blanchet
no timeout for Auto Try, since the Auto Tools framework takes care of timeouts
2010-09-13, by blanchet
add Proof General option
2010-09-11, by blanchet
make Try's output more concise
2010-09-11, by blanchet
added Auto Try to the mix of automatic tools
2010-09-11, by blanchet
crank up Auto Tools timeout;
2010-09-11, by blanchet
make Auto Solve part of the "Auto Tools"
2010-09-11, by blanchet
tuning
2010-09-11, by blanchet
tuning
2010-09-11, by blanchet
tuning
2010-09-11, by blanchet
tuning
2010-09-11, by blanchet
finished renaming "Auto_Counterexample" to "Auto_Tools"
2010-09-11, by blanchet
start renaming "Auto_Counterexample" to "Auto_Tools";
2010-09-11, by blanchet
setup Auto Sledgehammer
2010-09-11, by blanchet
make Mirabelle happy
2010-09-11, by blanchet
added Auto Sledgehammer docs
2010-09-11, by blanchet
change order of default ATPs;
2010-09-11, by blanchet
implemented Auto Sledgehammer
2010-09-11, by blanchet
document changes to Auto Nitpick
2010-09-11, by blanchet
change defaults of Auto Nitpick so that it consumes less resources (time and Kodkod threads)
2010-09-11, by blanchet
always handle type variables in typedefs as global
2010-09-11, by blanchet
removed duplicate lemma
2010-09-14, by nipkow
adding two more examples to example theory
2010-09-13, by bulwahn
handling function types more carefully than in e98a06145530
2010-09-13, by bulwahn
adding order on modes
2010-09-13, by bulwahn
removing obsolete argument in prepare_intrs; passing context instead of theory in prepare_intrs
2010-09-13, by bulwahn
type antiquotation: allow arbitrary type abbreviations, but fail with user-space exception on bad input
2010-09-13, by haftmann
merged
2010-09-13, by haftmann
added Imperative HOL overview
2010-09-13, by haftmann
print mode for Imperative HOL overview; tuned and more accurate dependencies
2010-09-13, by haftmann
'class' and 'type' are now antiquoations by default
2010-09-13, by haftmann
merged
2010-09-13, by wenzelm
merged
2010-09-13, by nipkow
renamed lemmas: ext_iff -> fun_eq_iff, set_ext_iff -> set_eq_iff, set_ext -> set_eqI
2010-09-13, by nipkow
added and renamed lemmas
2010-09-13, by nipkow
merged
2010-09-13, by bulwahn
directly computing the values of interest instead of composing functions in an unintelligent way that causes exponential much garbage; using the latest theory
2010-09-10, by bulwahn
added preliminary support for SMT datatypes (for now restricted to tuples and lists); only the Z3 interface (in oracle mode) makes use of it, there is especially no Z3 proof reconstruction support for datatypes yet
2010-09-13, by boehmes
use eta-contracted version for occurrence check (avoids possible non-termination)
2010-09-10, by krauss
tuned signature;
2010-09-13, by wenzelm
Type_Infer.finish: index 0 -- freshness supposedly via Name.invents;
2010-09-13, by wenzelm
simplified Type_Infer: eliminated separate datatypes pretyp/preterm -- only assign is_paramT TVars;
2010-09-13, by wenzelm
tuned;
2010-09-13, by wenzelm
Type_Infer.preterm: eliminated separate Constraint;
2010-09-12, by wenzelm
Type_Infer.infer_types: plain error instead of kernel exception TYPE;
2010-09-12, by wenzelm
load type_infer.ML later -- proper context for Type_Infer.infer_types;
2010-09-12, by wenzelm
common Type.appl_error, which also covers explicit constraints;
2010-09-12, by wenzelm
eliminated aliases of Type.constraint;
2010-09-12, by wenzelm
tuned;
2010-09-12, by wenzelm
tuned messages;
2010-09-12, by wenzelm
avoid extra wrapping for interrupts;
2010-09-10, by wenzelm
tuned markup;
2010-09-09, by wenzelm
updated keywords;
2010-09-10, by wenzelm
proper antiquotations;
2010-09-10, by wenzelm
fixed antiquotation;
2010-09-10, by wenzelm
updated generated file;
2010-09-10, by wenzelm
updated config options;
2010-09-10, by wenzelm
removed spurious addition from 9e58f0499f57;
2010-09-10, by wenzelm
merged
2010-09-10, by wenzelm
improved error message for common mistake (fun f where "g x = ...")
2010-09-10, by krauss
adding another String.literal example
2010-09-10, by bulwahn
fiddling with the correct setup for String.literal
2010-09-10, by bulwahn
refactoring mode inference so that the theory is not changed in the mode inference procedure
2010-09-10, by bulwahn
Haskell == is infix, not infixl
2010-09-10, by haftmann
more correct dependencies
2010-09-10, by haftmann
merged
2010-09-09, by blanchet
use definitional CNF for the goal if at least one of the premisses would lead to too many clauses in Meson
2010-09-09, by blanchet
use the Meson cutoff as the cutoff for using definitional CNF -- it's simpler that way
2010-09-09, by blanchet
clarify comment
2010-09-09, by blanchet
improve on 65903ec4e8e8: fix more "add_ffpair" exceptions in failed ATP proofs
2010-09-09, by blanchet
allow Sledgehammer proofs containing nameless local facts with schematic variables in them
2010-09-09, by blanchet
tuning
2010-09-09, by blanchet
more precise error messages when Vampire is interrupted or SPASS runs into an internal bug
2010-09-09, by blanchet
better error reporting when the Sledgehammer minimizer is interrupted
2010-09-09, by blanchet
add cutoff beyond which facts are handled using definitional CNF
2010-09-09, by blanchet
"resurrected" a Metis proof
2010-09-09, by blanchet
replace two slow "metis" proofs with faster proofs
2010-09-09, by blanchet
workaround to avoid subtle "add_ffpairs" unification exception in Sledgehammer;
2010-09-08, by blanchet
improve SInE-E failure message
2010-09-08, by blanchet
merged
2010-09-09, by bulwahn
adding an example with integers and String.literals
2010-09-09, by bulwahn
adding an example to show how code_pred must be invoked with locales
2010-09-09, by bulwahn
removing report from the arguments of the quickcheck functions and refering to it by picking it from the context
2010-09-09, by bulwahn
changing the container for the quickcheck options to a generic data
2010-09-09, by bulwahn
Tidied up proofs using sledgehammer, also deleting unnecessary semicolons
2010-09-09, by paulson
changing String.literal to a type instead of a datatype
2010-09-09, by bulwahn
increasing the number of iterations to ensure to find a counterexample by random generation
2010-09-09, by bulwahn
only conceal primitive definition theorems, not predicate names
2010-09-09, by haftmann
merged
2010-09-08, by haftmann
modernized primrec
2010-09-08, by haftmann
Markup_Tree is already scalable;
2010-09-10, by wenzelm
Isabelle_Markup.tooltip: explicit indication of ML;
2010-09-10, by wenzelm
Future.promise: more robust treatment of concurrent abort vs. fulfill (amending 047c96f41455);
2010-09-10, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-224
+224
+1000
+3000
+10000
+30000
tip