Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-480
+480
+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.
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
primitive use_text: let interrupts pass unhindered;
2010-09-10, by wenzelm
Isabelle.load_icon with some sanity checks;
2010-09-09, by wenzelm
ML_Compiler.eval: reported positions need to contain offset, to avoid displaced reports due to synthesized line numbers;
2010-09-09, by wenzelm
NEWS: some notes on interrupts;
2010-09-09, by wenzelm
refined Runtime.toplevel_error/Document.run_command: let interrupts pass unhindered;
2010-09-09, by wenzelm
removed dead code;
2010-09-09, by wenzelm
avoid handling interrupts in user code;
2010-09-09, by wenzelm
Meson.make_clauses_unsorted: removed spurious debug code stemming from 5146d640aa4a -- must not handle arbitrary exceptions in user space;
2010-09-09, by wenzelm
main command loops are supposed to be uninterruptible -- no special treatment here;
2010-09-09, by wenzelm
Exn.is_interrupt: include interrupts that have passed through the IO layer;
2010-09-09, by wenzelm
more abstract treatment of interrupts in structure Exn -- hardly ever need to mention Interrupt literally;
2010-09-09, by wenzelm
avoid mixing of static and runtime errors in compiler output, to accomodate Proof General;
2010-09-09, by wenzelm
ML_Compiler.eval: discontinued extra "Static Errors" of raw Poly/ML;
2010-09-08, by wenzelm
isabelle-jedit.css: suppress "location" markup, which indicates extra positional information intended for plain-old TTY mode;
2010-09-08, by wenzelm
ML_Compiler.eval: more careful printing of messages and regular output, trying to accomodate Poly/ML, Proof General, Isabelle/Scala/jEdit at the same time;
2010-09-08, by wenzelm
clarified -- inlined ML_Env.local_context;
2010-09-08, by wenzelm
merged
2010-09-08, by wenzelm
restricting invocation only if PROLOG_HOME is set
2010-09-08, by bulwahn
tuned proofs (based on fancy gutter icons in Isabelle/jEdit);
2010-09-08, by wenzelm
merge
2010-09-08, by blanchet
remove "safe" (as suggested by Tobias) and added "arith" to "try"
2010-09-08, by blanchet
remove "minipick" (the toy version of Nitpick) and some tests;
2010-09-06, by blanchet
use Future.fork rather than Thread.fork, so that the thread is part of the global thread management
2010-09-06, by blanchet
fix editor
2010-09-06, by blanchet
merged
2010-09-08, by wenzelm
merged
2010-09-08, by paulson
tidied using inductive_simps
2010-09-08, by paulson
NEWS
2010-09-08, by haftmann
removed ancient constdefs command
2010-09-08, by haftmann
put expand_(fun/set)_eq back in as synonyms, for compatibility
2010-09-08, by nipkow
set up Nil and Cons to work as fixrec patterns
2010-09-07, by huffman
merged
2010-09-07, by haftmann
updated generated document
2010-09-07, by haftmann
only write ghc pragma when writing to a file
2010-09-07, by haftmann
added flat_program; tuned signature
2010-09-07, by haftmann
dropped ancient deresolve_base; plain_const_syntax also needs modification of instance statement
2010-09-07, by haftmann
moved flat_program to code_namespace
2010-09-07, by haftmann
dropped outdated substitution
2010-09-07, by haftmann
Haskell uses generic flat_program combinator
2010-09-07, by haftmann
factored out build_module_namespace
2010-09-07, by haftmann
added generic flat_program procedure
2010-09-07, by haftmann
using the proposed modes for starting the fixpoint iteration in the mode analysis
2010-09-07, by bulwahn
merged
2010-09-07, by nipkow
renamed expand_*_eq in HOLCF as well
2010-09-07, by nipkow
expand_fun_eq -> ext_iff
2010-09-07, by nipkow
merged
2010-09-07, by bulwahn
lower expectation in Reg exp example
2010-09-07, by bulwahn
renewing specification in example file; adding invocation in example file
2010-09-07, by bulwahn
handling collection of simprules as sets rather than as lists
2010-09-07, by bulwahn
stating errors in error messages more verbose in predicate compiler
2010-09-07, by bulwahn
raising an exception instead of guessing some reasonable behaviour for this function
2010-09-07, by bulwahn
using linear find_least instead of sorting in the mode analysis of the predicate compiler
2010-09-07, by bulwahn
adding code attribute to definition of equality of finite sets for executability of equality of finite sets
2010-09-07, by bulwahn
adapting example files
2010-09-07, by bulwahn
adding the Reg_Exp example
2010-09-07, by bulwahn
towards time limiting the prolog execution
2010-09-07, by bulwahn
adding IMP quickcheck examples
2010-09-07, by bulwahn
adding the CFG example to the build process
2010-09-07, by bulwahn
adding a List example (challenge from Tobias) for counterexample search
2010-09-07, by bulwahn
adding dependencies to IsaMakefile; increasing negative search limit for predicate_compile_quickcheck; adding tracing of introduction rules in code_prolog
2010-09-07, by bulwahn
disposed some old TODO/FIXME;
2010-09-08, by wenzelm
Document_View: select gutter message icons from markup over line range, not full range results;
2010-09-07, by wenzelm
tuned properties;
2010-09-07, by wenzelm
moved token markup tables to isabelle_markup.scala;
2010-09-07, by wenzelm
concentrate Isabelle specific physical rendering markup selection in isabelle_markup.scala;
2010-09-07, by wenzelm
simplified Markup_Tree.select: Stream instead of Iterator (again), explicit Option instead of default;
2010-09-07, by wenzelm
Document_View: more precise painting of gutter icons, only if line selection area is sufficiently large;
2010-09-07, by wenzelm
basic support for warning/error gutter icons;
2010-09-07, by wenzelm
Document_View: some markup for main inner syntax categories;
2010-09-07, by wenzelm
Command.State.accumulate: check actual source range;
2010-09-07, by wenzelm
Isar_Document.reported_positions: slightly more robust treatment of positions outside the command range, notably parsing beyond EOF;
2010-09-07, by wenzelm
highlight bad range of nested error (here from inner parsing);
2010-09-07, by wenzelm
Isar_Document.reported_positions: exclude proof state output;
2010-09-07, by wenzelm
Document_View: less aggressive background coloring, departing from classic PG highlighting;
2010-09-07, by wenzelm
report token range after inner parse error -- often provides important clues about misunderstanding concerning lexical phase;
2010-09-07, by wenzelm
slightly more robust Plugin.stop -- components might refer to Isabelle.system even after shutdown;
2010-09-07, by wenzelm
turned show_hyps and show_tags into proper configuration option;
2010-09-06, by wenzelm
discontinued obsolete ProofContext.prems_limit;
2010-09-06, by wenzelm
ML_Context.thm and ML_Context.thms no longer pervasive;
2010-09-06, by wenzelm
more explicit indication of Config.raw options, which are only needed for bootstrapping Pure;
2010-09-06, by wenzelm
merged
2010-09-06, by wenzelm
When comparing Floats use integers instead of reals (represented as rationals), generates less code when Floats are used.
2010-09-06, by hoelzl
isatest: back to polyml-5.3.0 due to unresolved stability issues of polyml-5.4.0 and HOL/Decision_Procs/Approximation_Ex.thy;
2010-09-06, by wenzelm
more antiquotations;
2010-09-06, by wenzelm
ML_Context.thm;
2010-09-06, by wenzelm
more explicit HOL-Proofs sessions, including former ex/Hilbert_Classical.thy which works in parallel mode without the antiquotation option "margin" (which is still critical);
2010-09-06, by wenzelm
modernized session ROOT setup;
2010-09-06, by wenzelm
some results of concurrency code inspection;
2010-09-06, by wenzelm
merged;
2010-09-06, by wenzelm
mention ~/.isabelle/etc/settings file
2010-09-06, by blanchet
make remote ATP invocation work for those people who need to go through a proxy;
2010-09-06, by blanchet
enabled do notation for option type
2010-09-05, by krauss
removed duplicate lemma
2010-09-05, by krauss
added Option.bind
2010-09-05, by krauss
merged
2010-09-04, by haftmann
printing combinator for hierarchical programs
2010-09-04, by haftmann
merged
2010-09-04, by haftmann
add lemma cont2cont_Let_simple
2010-09-04, by huffman
add lemma cont2cont_split_simple
2010-09-04, by huffman
add List_Cpo.thy to HOLCF/Library
2010-09-04, by huffman
dropped names from serializer interface
2010-09-04, by haftmann
added more explicit warning
2010-09-04, by haftmann
ML_Context.ml_store_thm(s): operate on thread context instead of Unsynchronized.ref;
2010-09-06, by wenzelm
use setmp_noncritical for PGIP, which is presumably sequential (PG clone);
2010-09-05, by wenzelm
use setmp_noncritical for sequential Pure bootstrap;
2010-09-05, by wenzelm
turned show_brackets into proper configuration option;
2010-09-05, by wenzelm
Syntax.standard_parse_term: eliminated redundant Pretty.pp;
2010-09-05, by wenzelm
structure Syntax: define "interfaces" before actual implementations;
2010-09-05, by wenzelm
turned show_sorts/show_types into proper configuration options;
2010-09-05, by wenzelm
pretty printing: prefer regular Proof.context over Pretty.pp, which is mostly for special bootstrap purposes involving theory merge, for example;
2010-09-05, by wenzelm
refined treatment of multi-line subexpressions;
2010-09-04, by wenzelm
basic support for subexpression highlighting (see also gatchan.jedit.hyperlinks.HyperlinkManager/HyperlinkTextAreaPainter);
2010-09-04, by wenzelm
updated configuration options;
2010-09-04, by wenzelm
recovered options for goal antiquotations from f45d332a90e3: actually pass context to Proof.pretty_goals (see also 45facd8f358e);
2010-09-04, by wenzelm
turned eta_contract into proper configuration option;
2010-09-03, by wenzelm
turned show_structs into proper configuration option;
2010-09-03, by wenzelm
configuration options Syntax.ambiguity_enabled (inverse of former Syntax.ambiguity_is_error), Syntax.ambiguity_level (with Isar attribute "syntax_ambiguity_level"), Syntax.ambiguity_limit;
2010-09-03, by wenzelm
pretty_goals: turned some global references and function arguments into configuration options (goals_limit = 10, goals_total = true, show_main_goal = false) depending on the context;
2010-09-03, by wenzelm
tuned comment;
2010-09-03, by wenzelm
merged
2010-09-03, by wenzelm
merged
2010-09-03, by haftmann
QND_FLAG is a shell variable, not a string
2010-09-03, by haftmann
modernized session ROOT;
2010-09-03, by wenzelm
disposed left-over user preferences;
2010-09-03, by wenzelm
turned show_all_types into proper configuration option;
2010-09-03, by wenzelm
treat show_free_types as plain ML option, without the extras of global default and registration in the attribute name space -- NB: 'print_configs' only shows the latter;
2010-09-03, by wenzelm
more explicit Config.declare vs. Config.declare_global;
2010-09-03, by wenzelm
turned show_no_free_types into proper configuration option show_free_types, with flipped polarity;
2010-09-03, by wenzelm
remove code I submitted accidentally
2010-09-03, by blanchet
merged
2010-09-03, by blanchet
disable "definitional CNF";
2010-09-03, by blanchet
redisable Nitpick from Cygwin, until I've investigated the issue
2010-09-03, by blanchet
show the number of facts for each prover in "verbose" mode
2010-09-02, by blanchet
fix bug in "debug" mode
2010-09-02, by blanchet
make sure "Unknown ATP" errors reach the users -- i.e. don't generate them from a thread
2010-09-02, by blanchet
If Geoff puts some important message in his TPTP problems (e.g., money requests), we should show them to the user
2010-09-02, by blanchet
fix trivial "x = x" fact detection
2010-09-02, by blanchet
merged
2010-09-03, by wenzelm
merged
2010-09-03, by haftmann
merged
2010-09-02, by haftmann
hand out deresolver from serializer invocation
2010-09-02, by haftmann
Revert bij_betw changes to simp set (Problem in afp/Ordinals_and_Cardinals)
2010-09-02, by hoelzl
merged
2010-09-02, by hoelzl
Updated proofs in Dining Cryptographers theory
2010-09-02, by hoelzl
Corrected definition and hence removed sorry.
2010-09-02, by hoelzl
Moved lemmas to appropriate locations
2010-09-02, by hoelzl
merged
2010-09-02, by hoelzl
merged
2010-09-02, by hellerar
measure unique
2010-09-02, by hellerar
merge
2010-09-01, by hellerar
move lemmas to correct theory files
2010-09-02, by hoelzl
factorizable measurable functions
2010-08-27, by hoelzl
Introduced sigma algebra generated by function preimages.
2010-08-27, by hoelzl
vimage of measurable function is a measure space
2010-08-27, by hoelzl
Measurable on product space is equiv. to measurable components
2010-08-27, by hoelzl
Measurable on euclidean space is equiv. to measurable components
2010-08-27, by hoelzl
preimages of open sets over continuous function are open
2010-08-27, by hoelzl
added definition of conditional expectation
2010-08-27, by hoelzl
proved existence of conditional expectation
2010-08-27, by hoelzl
introduced integration on subalgebras
2010-08-26, by hoelzl
changed definition of dynkin; replaces proofs by metis calles
2010-08-26, by hoelzl
dynkin
2010-08-26, by hellerar
dynkin system
2010-08-26, by hellerar
merged
2010-09-02, by hoelzl
Fixes lemma names
2010-09-02, by hoelzl
NEWS
2010-09-02, by hoelzl
Introduce surj_on and replace surj and bij by abbreviations.
2010-09-02, by hoelzl
Permutation implies bij function
2010-09-02, by hoelzl
bij <--> bij_betw
2010-09-02, by hoelzl
Add filter_remove1
2010-09-02, by hoelzl
Add lessThan_Suc_eq_insert_0
2010-09-02, by hoelzl
merged
2010-09-02, by haftmann
updated
2010-09-02, by haftmann
set printmode while marking
2010-09-02, by haftmann
updated
2010-09-02, by haftmann
avoid reference to theory Ferrack altogether
2010-09-02, by haftmann
more canonical theory setup
2010-09-02, by haftmann
set depth to 1
2010-09-02, by haftmann
avoid theory Imperative_HOL altogether
2010-09-02, by haftmann
adapted to change eq -> equal
2010-09-02, by haftmann
corrected printmode handling
2010-09-02, by haftmann
swapped slip
2010-09-02, by haftmann
updated
2010-09-02, by haftmann
restored and added surpression of case combinators
2010-09-02, by haftmann
dropped superfluous presentation names
2010-09-02, by haftmann
manage statement selection for presentation wholly through markup
2010-09-02, by haftmann
formal markup of generated code for statements
2010-09-02, by haftmann
removed namespace stuff from code_printer
2010-09-02, by haftmann
merged
2010-09-02, by blanchet
reenable Nitpick on Cygwin;
2010-09-02, by blanchet
merged;
2010-09-03, by wenzelm
Proof.pretty_state: print everything in the foreground context to give users a chance to configure options, e.g. via "using [[show_consts]]";
2010-09-03, by wenzelm
turned show_consts into proper configuration option;
2010-09-03, by wenzelm
prefer regular Proof.context over background theory;
2010-09-03, by wenzelm
just one refute.ML;
2010-09-02, by wenzelm
use existing Integer.pow, despite its slightly odd argument order;
2010-09-02, by wenzelm
tuned whitespace and indentation, emphasizing the logical structure of this long text;
2010-09-02, by wenzelm
inner parsing: refrain from too many nested position reports to achieve more precise error feedback in the source;
2010-09-02, by wenzelm
Document_View: squiggly underline for messages;
2010-09-02, by wenzelm
added gfx_range convenience;
2010-09-02, by wenzelm
Isar_Document.reported_positions: more precise include/exclude, include root as last resort only;
2010-09-02, by wenzelm
Position.Range: exclude singularity (again);
2010-09-02, by wenzelm
merged
2010-09-02, by wenzelm
merged
2010-09-02, by blanchet
FIXME -> TODO (nothing is broken)
2010-09-02, by blanchet
Let MESON take an additional "preskolemization tactic", which can be used to put the goal in definitional CNF
2010-09-02, by blanchet
use definitional CNFs in Metis rather than plain CNF, following a suggestion by Joe Hurd;
2010-09-02, by blanchet
make definitional CNF translation code more robust in the presence of existential quantifiers in the "literals"
2010-09-02, by blanchet
formal framework for presentation of selected statements
2010-09-02, by haftmann
merged
2010-09-02, by haftmann
Table.map replaces Table.map'
2010-09-02, by haftmann
dropped dead code; tuned
2010-09-02, by haftmann
include names need not be considered as reserved any longer
2010-09-02, by haftmann
skip empty name bunches; fill up trailing positions with NONEs
2010-09-02, by haftmann
use code_namespace module for SML and OCaml code
2010-09-02, by haftmann
Table.map replaces Table.map'
2010-09-02, by haftmann
avoid cyclic modules
2010-09-02, by haftmann
merged
2010-09-02, by haftmann
simultaneous modification of statements: statement names
2010-09-01, by haftmann
simultaneous modification of statements
2010-09-01, by haftmann
explicit modify_stmt parameter
2010-09-01, by haftmann
Graph.map, in analogy to Table.map
2010-09-01, by haftmann
replaced Table.map' by Table.map
2010-09-01, by haftmann
merged
2010-09-01, by haftmann
tuned
2010-09-01, by haftmann
generalized hierarchical data structure over statements
2010-09-01, by haftmann
merged
2010-09-02, by haftmann
normalization is allowed to solve True
2010-09-02, by haftmann
merged
2010-09-02, by blanchet
merged
2010-09-02, by blanchet
cosmetics
2010-09-02, by blanchet
SNARK doesn't like facts
2010-09-02, by blanchet
show real CPU time
2010-09-02, by blanchet
factor out code shared by all ATPs so that it's run only once
2010-09-01, by blanchet
handle all whitespace, not just ASCII 32
2010-09-01, by blanchet
speed up SPASS hack + output time information in "blocking" mode
2010-09-01, by blanchet
remove time information in output, since it's confusing anyway
2010-09-01, by blanchet
minor refactoring
2010-09-01, by blanchet
translate the axioms to FOF once and for all ATPs
2010-09-01, by blanchet
run relevance filter in a thread, to avoid blocking
2010-09-01, by blanchet
add dependency of "spass" script
2010-09-01, by blanchet
more elegant ML
2010-09-01, by blanchet
only kill ATP threads in nonblocking mode
2010-09-01, by blanchet
lower number of facts given to SInE
2010-09-01, by blanchet
share the relevance filter among the provers
2010-09-01, by blanchet
got rid of the "theory_relevant" option;
2010-09-01, by blanchet
generalize theorem argument parsing syntax
2010-09-01, by blanchet
support new option in Mirabelle
2010-09-01, by blanchet
fiddled with fudge factor (based on Mirabelle)
2010-09-01, by blanchet
give priority to assumptions in structured proofs
2010-09-01, by blanchet
introduce fudge factors to deal with "theory const"
2010-09-01, by blanchet
rename sledgehammer config attributes
2010-09-01, by blanchet
finish moving file
2010-09-01, by blanchet
move file
2010-08-31, by blanchet
finished renaming
2010-08-31, by blanchet
fix typo
2010-08-31, by blanchet
shorten a few file names
2010-08-31, by blanchet
added "expect" feature of Nitpick to Sledgehammer, for regression testing
2010-08-31, by blanchet
update docs
2010-08-31, by blanchet
update docs
2010-08-31, by blanchet
added "blocking" option to Sledgehammer to run in synchronous mode;
2010-08-31, by blanchet
normalization fails on unchanged goal
2010-09-02, by haftmann
turned show_question_marks into proper configuration option;
2010-09-02, by wenzelm
prefer regular print functions over slightly low-level Term.string_of_vname;
2010-09-01, by wenzelm
eliminated obsolete old-style goal stack package, which was considered the main Isabelle user interface at some point;
2010-09-01, by wenzelm
eliminated really ancient OldGoals operations in favour of Goal.prove_internal (with its minimal checks and without normalization of result);
2010-09-01, by wenzelm
Document.State.Assignment: eliminated promise in favour of plain values -- signalling is done via event bus in Session;
2010-09-01, by wenzelm
actually declare "_constrainAbs" as @{syntax_const};
2010-09-01, by wenzelm
merged
2010-09-01, by haftmann
repaired attribute code_unfold_post which has ever been broken
2010-09-01, by haftmann
tuned text segment
2010-09-01, by haftmann
merged
2010-09-01, by haftmann
factored out generic part of Scala serializer into code_namespace.ML
2010-09-01, by haftmann
merged
2010-09-01, by wenzelm
do not print object frame around Scala includes -- this is in the responsibility of the user
2010-09-01, by haftmann
repaired codegen tool
2010-09-01, by haftmann
tuned internally and made smlnj happy
2010-09-01, by haftmann
merged
2010-09-01, by bulwahn
renewing specifications in HOL-Auth
2010-08-31, by bulwahn
adapting and tuning example theories
2010-08-31, by bulwahn
adding further example for quickcheck with prolog code generation
2010-08-31, by bulwahn
handling the quickcheck result no counterexample more correctly
2010-08-31, by bulwahn
adding manual reordering of premises to prolog generation
2010-08-31, by bulwahn
towards support of limited predicates for mutually recursive predicates
2010-08-31, by bulwahn
improving clash-free naming of variables and preds in code_prolog
2010-08-31, by bulwahn
exporting mode analysis for use in prolog generation
2010-08-31, by bulwahn
renaming
2010-08-31, by bulwahn
improving naming of predicates in code_prolog; changing order of flattened premises once again
2010-08-31, by bulwahn
changing order of premises generated when flattening functions in premises; adapting example for second attack for hotel key card system
2010-08-31, by bulwahn
added further hotel key card attack in example file
2010-08-31, by bulwahn
avoiding warning for a duplicate rewrite rule in preprocessing of the predicate compiler
2010-08-31, by bulwahn
using Cache_IO interface for a safe parallel prolog execution
2010-08-31, by bulwahn
storing options for prolog code generation in the theory
2010-08-31, by bulwahn
adapting example files to latest changes
2010-08-31, by bulwahn
adding Lambda example theory; tuned
2010-08-31, by bulwahn
added quite adhoc logic program transformations limited_predicates and replacements of predicates
2010-08-31, by bulwahn
distinguish between "by" and "apply"
2010-08-31, by blanchet
merged
2010-08-31, by blanchet
fiddling with "try"
2010-08-31, by blanchet
updated
2010-08-31, by blanchet
"try" -- a new diagnosis tool that tries to apply several methods in parallel
2010-08-31, by blanchet
add one option to Mirabelle
2010-08-31, by blanchet
update docs
2010-08-31, by blanchet
add a penalty for being higher-order
2010-08-31, by blanchet
improve weighting of irrelevant constants, based on Mirabelle experiments
2010-08-31, by blanchet
take into consideration whether a fact is an "intro"/"elim"/"simp" rule as an additional factor influencing the relevance filter
2010-08-31, by blanchet
repaired casual accident; tuned names
2010-08-31, by haftmann
corrected misbehaved additional qualification of generated names
2010-08-31, by haftmann
merged
2010-08-31, by haftmann
avoid strange special treatment of empty module names
2010-08-31, by haftmann
allow explicit parameter for code width
2010-08-31, by haftmann
evaluate takes ml context and ml expression parameter
2010-08-31, by haftmann
modernized; avoid pointless tinkering with structure names
2010-08-31, by haftmann
distinguish code production and code presentation
2010-08-31, by haftmann
dropped single_module parameter
2010-08-31, by haftmann
tuned
2010-08-31, by haftmann
record argument for serializers
2010-08-31, by haftmann
tuned serializer argument interface
2010-08-31, by haftmann
removed serializer interface redundancies
2010-08-31, by haftmann
more coherent naming of syntax data structures
2010-08-31, by haftmann
Code_Printer.tuplify
2010-08-31, by haftmann
dropped legacy interfaces
2010-08-31, by haftmann
more permissive: simplification solves the goal when rhs = undefined
2010-08-31, by krauss
merged
2010-08-30, by haftmann
tuned
2010-08-30, by haftmann
tuned
2010-08-30, by haftmann
tuned
2010-08-30, by haftmann
tuned
2010-08-30, by haftmann
tuned file interface
2010-08-30, by haftmann
tuned
2010-08-30, by haftmann
eliminated some obscure higher-order arguments
2010-08-30, by haftmann
trailing newline by default
2010-08-30, by haftmann
width is a formal parameter of serialization
2010-08-30, by haftmann
whitespace tuning
2010-08-30, by haftmann
tuned comment
2010-08-30, by haftmann
merged
2010-08-30, by blanchet
fiddle with fact filter
2010-08-30, by blanchet
adjust Mirabelle
2010-08-30, by blanchet
rule out low-level class facts
2010-08-30, by blanchet
make Sledgehammer's relevance filter somewhat slacker
2010-08-30, by blanchet
move imperative code to where it belongs
2010-08-30, by blanchet
fiddle with fact filter based on Mirabelle experiments
2010-08-30, by blanchet
allow configuration of fact filter fudge factors
2010-08-30, by blanchet
made all fudge factors in relevance filter references, so that Mirabelle can set them (for experiments)
2010-08-30, by blanchet
execute actions in same order as specified on command line
2010-08-30, by blanchet
show index in fact list of all found facts
2010-08-30, by blanchet
allow multiple invocations of "mirabele_sledgehammer_filter", by multiplexing on ID
2010-08-30, by blanchet
deal with duplicates
2010-08-30, by blanchet
improve new "sledgehammer_filter" action
2010-08-30, by blanchet
remove useless var
2010-08-30, by blanchet
less
more
|
(0)
-30000
-10000
-3000
-1000
-480
+480
+1000
+3000
+10000
+30000
tip