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.
added Isabelle_Process.input_bytes, which avoids the somewhat slow Standard_System.string_bytes (just in case someone wants to stream raw data at 250MB/s);
2010-08-13, by wenzelm
do not buffer fifo streams here -- done in Isabelle_Process;
2010-08-13, by wenzelm
explicit Document.State value, instead of individual state variables in Session, Command, Document;
2010-08-13, by wenzelm
edit_document: more precise status position;
2010-08-13, by wenzelm
added get_after convenience;
2010-08-13, by wenzelm
more basic notion of unparsed input;
2010-08-12, by wenzelm
simplified/clarified Change: transition prev --edits--> result, based on futures;
2010-08-12, by wenzelm
moved snapshot to Session (cf. 96b22dfeb56a);
2010-08-12, by wenzelm
Change: eliminated id, which is merely the resulting document id and is only required in joined state anyway;
2010-08-12, by wenzelm
clarified "state" (accumulated data) vs. "exec" (execution that produces data);
2010-08-12, by wenzelm
misc tuning and simplification;
2010-08-12, by wenzelm
specific command state;
2010-08-12, by wenzelm
specific Session.Commands_Changed;
2010-08-12, by wenzelm
consider snapshot as service of Session, not Document.Change;
2010-08-12, by wenzelm
tuned scope;
2010-08-12, by wenzelm
Document.print_id;
2010-08-11, by wenzelm
consider command state as part of Snapshot, not Document;
2010-08-11, by wenzelm
represent document ids by (long) int, to benefit from the somewhat faster Inttab in ML (LinearSet in Scala is invariably indexed by native object ids);
2010-08-11, by wenzelm
Named_Target;
2010-08-11, by wenzelm
modernized specifications;
2010-08-11, by wenzelm
spelling;
2010-08-11, by wenzelm
merged
2010-08-11, by wenzelm
renamed Theory_Target to the more appropriate Named_Target
2010-08-11, by haftmann
discontinue old implementation of `foundation`
2010-08-11, by haftmann
moved instantiation target formally to class_target.ML
2010-08-11, by haftmann
NEWS
2010-08-11, by haftmann
merged
2010-08-11, by haftmann
print fcomp combinator only monadic in connection with other monadic expressions
2010-08-11, by haftmann
merged
2010-08-11, by haftmann
merged
2010-08-11, by haftmann
moved overloading target formally to overloading.ML
2010-08-11, by haftmann
moved theory-level target operation fragements to Generic_Target; adjusted bootstrap order
2010-08-11, by haftmann
merged
2010-08-11, by haftmann
whitespace tuning
2010-08-11, by haftmann
remove overloading and instantiation from data slot
2010-08-11, by haftmann
removed obsolete Toplevel.enter_proof_body;
2010-08-11, by wenzelm
standardized pretty printing of consts (e.g. see find_theorems, print_theory);
2010-08-11, by wenzelm
misc tuning and simplification;
2010-08-11, by wenzelm
simplified/unified command setup;
2010-08-11, by wenzelm
removed obsolete Proof.get_thmss_cmd (cf. Attrib.eval_thms);
2010-08-11, by wenzelm
prefer plain Attrib.eval_thmss -- also means the assert_forward of Proof.get_thmss_cmd is skipped, leading to uniform (albeit odd) behaviour concerning forward chaining;
2010-08-11, by wenzelm
prefer plain Attrib.eval_thms with plain Proof.context instead of Proof.state;
2010-08-11, by wenzelm
tuned eval_thms (cf. note etc. in proof.ML);
2010-08-11, by wenzelm
use Pretty.enum convenience;
2010-08-11, by wenzelm
tuned whitespace;
2010-08-11, by wenzelm
more precise and more maintainable dependencies;
2010-08-11, by wenzelm
merged, resolving conflict in src/Pure/IsaMakefile concerning General/xml_data.ML;
2010-08-11, by wenzelm
* -> prod
2010-08-11, by haftmann
added .ML extension
2010-08-11, by haftmann
avoid old unnamed infix
2010-08-11, by haftmann
avoid inclusion of Natural module in generated code
2010-08-11, by haftmann
explicit ML extension
2010-08-11, by haftmann
merged
2010-08-11, by haftmann
separate initialisation for overloading and instantiation target
2010-08-10, by haftmann
different foundations for different targets; simplified syntax handling of abbreviations
2010-08-10, by haftmann
deleted duplicate lemma
2010-08-11, by Christian Urban
Revert performance improvement of 8ed3a5fb4d25 since it breaks notes element declarations.
2010-08-10, by ballarin
basic renumbering
2010-08-10, by haftmann
avoiding redundant primes
2010-08-10, by haftmann
separated type from term parameters
2010-08-10, by haftmann
moved extra_tfrees check for mixfix syntax to Generic_Target
2010-08-10, by haftmann
name and argument grouping tuning
2010-08-10, by haftmann
whitespace tuning
2010-08-10, by haftmann
added generic_target.ML
2010-08-10, by haftmann
try to uniformly follow define/note/abbrev/declaration order as close as possible
2010-08-10, by haftmann
split off structure Generic_Target into separate file
2010-08-10, by haftmann
split off generic parts of target implementations into separate structure
2010-08-10, by haftmann
restructured code for `declaration`
2010-08-10, by haftmann
executable relation operations contributed by Tjark Weber
2010-08-10, by haftmann
factored out foundation of `define` into separate function
2010-08-09, by haftmann
combine declaration and definition of foundation constant
2010-08-09, by haftmann
more appropriate outline of `define`
2010-08-09, by haftmann
backlink definition to target `notes`
2010-08-09, by haftmann
merged
2010-08-09, by haftmann
dropped idle local_facts argument; factored out theory_abbrev and locale_abbrev
2010-08-09, by haftmann
more convenient order
2010-08-09, by haftmann
dropped misleading comments
2010-08-09, by haftmann
merged
2010-08-09, by haftmann
separated foundation of `notes`
2010-08-09, by haftmann
more clear separation into local and global facts
2010-08-09, by haftmann
sharpened and tuned educated guess for canonical class morphism
2010-08-09, by haftmann
minimize sorts in certificate instantiation
2010-08-09, by haftmann
prevent ATP thread for staying around for 1 minute if an exception occurred earlier;
2010-08-09, by blanchet
adapt "too_general_equality" blacklisting to the new FOF context, where quantifiers are sometimes present
2010-08-09, by blanchet
"declare" -> "declaration" (typo)
2010-08-09, by blanchet
replace "setup" with "declaration"
2010-08-09, by blanchet
disable Nitpick on Cygwin while I'm on vacation;
2010-08-09, by blanchet
merged
2010-08-09, by blanchet
use "declaration" instead of "setup" to register Nitpick extensions
2010-08-09, by blanchet
remove needless "open"
2010-08-09, by blanchet
move Sledgehammer's HOL -> FOL translation to separate file (sledgehammer_translate.ML)
2010-08-09, by blanchet
fiddle some more with "max_new_relevant_facts_per_iter"
2010-08-09, by blanchet
replace recursion with "fold"
2010-08-09, by blanchet
remove debugging output
2010-08-09, by blanchet
remove now needless "Thm.transfer"
2010-08-09, by blanchet
reintroduced old code that removed axioms from the conjecture assumptions, ported to FOF
2010-08-09, by blanchet
merge
2010-08-09, by blanchet
fix embarrassing bug in elim rule handling, introduced during the port to FOF
2010-08-09, by blanchet
minor doc changes
2010-08-06, by blanchet
modernized some specifications;
2010-08-11, by wenzelm
tuned;
2010-08-11, by wenzelm
Isar_Document command input via native Isabelle_Process commands, using YXML and XML_Data representation;
2010-08-11, by wenzelm
native Isabelle_Process commands, based on efficient byte channel protocol for string lists;
2010-08-11, by wenzelm
proper handling of empty text;
2010-08-11, by wenzelm
more uniform XML/YXML string_of_body/string_of_tree;
2010-08-11, by wenzelm
type XML.Body as basic data representation language (Scala version);
2010-08-10, by wenzelm
type XML.body as basic data representation language;
2010-08-10, by wenzelm
renamed YXML.binary_text to YXML.escape_controls to emphasize what it actually does;
2010-08-10, by wenzelm
added string_bytes convenience;
2010-08-10, by wenzelm
tuned;
2010-08-10, by wenzelm
removed obsolete methods for (ML) commands;
2010-08-10, by wenzelm
prefer Nimbus look and feel on all platforms, instead of the somewhat ugly javax.swing.plaf.metal.MetalLookAndFeel, which presumably is implicit fall-back nonetheless;
2010-08-10, by wenzelm
edit_document: synchronous reply to ensure consistent state wrt. calling (AWT) thread;
2010-08-10, by wenzelm
distinguish proper Isabelle_Process INPUT vs. raw STDIN, tuned corresponding method names;
2010-08-10, by wenzelm
added Library.thread_actor -- thread as actor;
2010-08-10, by wenzelm
clarified JEDIT_JAVA_OPTIONS vs. JEDIT_SYSTEM_OPTIONS -- discontinued JEDIT_APPLE_PROPERTIES;
2010-08-10, by wenzelm
auto_flush: higher frequency;
2010-08-09, by wenzelm
uniform raw_dump for input/output fifos on Cygwin;
2010-08-09, by wenzelm
more robust fifo rendezvous: Cygwin 1.7 does not really block as expected;
2010-08-09, by wenzelm
Isabelle_Process: separate input fifo for commands (still using the old tty protocol);
2010-08-09, by wenzelm
tuned comments;
2010-08-09, by wenzelm
merged
2010-08-09, by wenzelm
added Lars Noschinski to isatest report
2010-08-09, by haftmann
merged
2010-08-09, by wenzelm
discontinued separation of `define` and `declare_const`
2010-08-08, by haftmann
unravelled target initialization code
2010-08-08, by haftmann
added filter for Boogie verification conditions (to prune assertions already proved by Boogie/Z3)
2010-08-08, by boehmes
added scanning of if-then-else expressions
2010-08-08, by boehmes
merged
2010-08-06, by blanchet
added support for partial quotient types;
2010-08-06, by blanchet
adapt occurrences of renamed Nitpick functions
2010-08-06, by blanchet
document the non-legacy interfaces
2010-08-06, by blanchet
local versions of Nitpick.register_xxx functions
2010-08-06, by blanchet
parse_spans: somewhat faster low-level implementation;
2010-08-08, by wenzelm
proper context for Syntax.parse_token;
2010-08-08, by wenzelm
prefer Context_Position.report where a proper context is available -- notably for "inner" entities;
2010-08-08, by wenzelm
explicitly distinguish Output.status (essential feedback) vs. Output.report (useful markup);
2010-08-08, by wenzelm
fixed odd runtime type error, which appears to have escaped the scala-2.8.0.final compiler;
2010-08-08, by wenzelm
YXML.parse: refrain from interning, let XML.Cache do it (partially);
2010-08-08, by wenzelm
cache_string: store trimmed string value;
2010-08-08, by wenzelm
simple_dialog: allow scala.swing.Component as well;
2010-08-07, by wenzelm
simplified some Markup;
2010-08-07, by wenzelm
simplified type XML.Tree: embed Markup directly, avoid slightly odd triple;
2010-08-07, by wenzelm
more robust treatment of Markup.token;
2010-08-07, by wenzelm
simplified type XML.tree: embed Markup.T directly, avoid slightly odd triple;
2010-08-07, by wenzelm
concentrate structural document notions in document.scala;
2010-08-07, by wenzelm
maintain editor history independently of Swing thread, which is potentially a bottle-neck or might be unavailable (e.g. in batch mode);
2010-08-07, by wenzelm
tuned;
2010-08-07, by wenzelm
more explicit model of pending text edits;
2010-08-07, by wenzelm
more explicit treatment of Swing thread context;
2010-08-07, by wenzelm
replaced individual Document_Model history by all-inclusive one in Session;
2010-08-07, by wenzelm
misc tuning and clarification;
2010-08-07, by wenzelm
avoid null in Scala;
2010-08-06, by wenzelm
updated keywords;
2010-08-06, by wenzelm
removed obsolete Goal.local_future_enforced: Toplevel.run_command is no longer interactive, so Goal.local_future_enabled is sufficient (cf. 349e9223c685 and e07dacec79e7);
2010-08-06, by wenzelm
merged
2010-08-06, by wenzelm
merged
2010-08-06, by blanchet
quotient types registered as codatatypes are no longer quotient types
2010-08-06, by blanchet
added a friendly warning
2010-08-06, by blanchet
extend the scope of limitation about nonconservative extensions
2010-08-06, by blanchet
improved "merge_type_vars" option: map supersorts to subsorts, to avoid distinguishing, say, "{}", and "HOL.type"
2010-08-06, by blanchet
Remove duplicate locale activation code; performance improvement.
2010-08-05, by ballarin
added record field
2010-08-05, by blanchet
added "whack"
2010-08-05, by blanchet
handle "Rep_unit" & Co. gracefully
2010-08-05, by blanchet
added support for "Abs_" and "Rep_" functions on quotient types
2010-08-05, by blanchet
fiddle with specialization etc.
2010-08-05, by blanchet
handle inductive predicates correctly after change in "def" semantics
2010-08-05, by blanchet
don't specialize built-ins or constructors
2010-08-05, by blanchet
more docs
2010-08-05, by blanchet
prevent the expansion of too large definitions -- use equations for these instead
2010-08-05, by blanchet
make nitpick accept "==" for "nitpick_(p)simp"s
2010-08-05, by blanchet
fix bug in Nitpick's "equationalize" function (the prems were ignored) + make it do some basic extensionalization
2010-08-05, by blanchet
deal correctly with Pure.conjunction in mono check
2010-08-05, by blanchet
rename internal functions
2010-08-05, by blanchet
remove buggy and needless condition
2010-08-05, by blanchet
renamed internal function
2010-08-05, by blanchet
Cycle breaking in the bounds takes care of singly recursive datatypes, so we don't need to do it again;
2010-08-04, by blanchet
avoid "<=>" in sym break constraint generation (since these are SAT-unfreundlich) + fix "epsilon2" to "epsilon1" (subtle bug)
2010-08-04, by blanchet
improve datatype symmetry breaking;
2010-08-04, by blanchet
merged
2010-08-04, by blanchet
make SML/NJ happy
2010-08-04, by blanchet
get rid of all "optimizations" regarding "unit" and other cardinality-1 types
2010-08-04, by blanchet
tuning
2010-08-03, by blanchet
better "Pretty" handling
2010-08-03, by blanchet
change formula for enumerating scopes
2010-08-03, by blanchet
example tweaking -- also prevents Nitpick_Tests from using more than 1 thread
2010-08-03, by blanchet
speed up Nitpick examples a little bit
2010-08-03, by blanchet
minor changes
2010-08-03, by blanchet
updated example timings
2010-08-03, by blanchet
more helpful message
2010-08-03, by blanchet
also mention gfp
2010-08-03, by blanchet
bump up the max cardinalities, to use up more of the time given to us by the user
2010-08-03, by blanchet
make tracing monotonicity easier
2010-08-03, by blanchet
more documentation, based on email discussions with a user
2010-08-03, by blanchet
make example easier to parse
2010-08-03, by blanchet
clarify attribute documentation
2010-08-03, by blanchet
choose better example
2010-08-03, by blanchet
fix newly introduced bug w.r.t. conditional equations
2010-08-03, by blanchet
document something I explained in an email to a poweruser
2010-08-03, by blanchet
make Nitpick more flexible when parsing (p)simp rules
2010-08-03, by blanchet
fix soundness bug w.r.t. "Suc" with "binary_ints"
2010-08-03, by blanchet
handle free variables even more gracefully;
2010-08-03, by blanchet
optimize local "def"s by treating them as definitions
2010-08-03, by blanchet
careful about which linear inductive predicates should be starred
2010-08-02, by blanchet
help Nitpick
2010-08-02, by blanchet
fix Skolemizer -- last week's optimizations resulted in UnequalLengths errors
2010-08-02, by blanchet
prevent generation of needless specialized constants etc.
2010-08-02, by blanchet
optimize generated Kodkod formula
2010-08-02, by blanchet
prefer implication to equality, to be more SAT solver friendly
2010-08-02, by blanchet
minor symmetry breaking for codatatypes like llist
2010-08-02, by blanchet
fix bug with mutually recursive and nested codatatypes
2010-08-02, by blanchet
fix minor bug in sym breaking
2010-08-01, by blanchet
modernized specifications;
2010-08-06, by wenzelm
Document_Model: include token marker here;
2010-08-05, by wenzelm
tuned;
2010-08-05, by wenzelm
misc tuning -- produce reverse_edits at most once (note that foldRight produces a reversed list internally, while recursion is infisible due to small stack vs. large stack frames on JVM);
2010-08-05, by wenzelm
editor mode;
2010-08-05, by wenzelm
Text_Edit.convert/revert;
2010-08-05, by wenzelm
renamed to_current to convert, and from_current to revert;
2010-08-05, by wenzelm
Change.Snapshot: include from_current/to_current here, with precomputed changes;
2010-08-05, by wenzelm
explicit Change.Snapshot and Document.Node;
2010-08-05, by wenzelm
simplified/refined document model: collection of named nodes, without proper dependencies yet;
2010-08-05, by wenzelm
somewhat uniform Thy_Header.split_thy_path in ML and Scala;
2010-08-05, by wenzelm
uniform naming of imports (source specification) vs. parents (thy node names) vs. parent_thys (theory values);
2010-08-04, by wenzelm
load_thy/after_load: explicit check of parent theories, which might have failed to join proofs -- avoid uninformative crash via Graph.UNDEF;
2010-08-04, by wenzelm
export use_thys_wrt;
2010-08-04, by wenzelm
more precise CRITICAL sections, using NAMED_CRITICAL uniformly;
2010-08-04, by wenzelm
updated to Netbeans 6.9;
2010-08-04, by wenzelm
schedule_futures: discontinued special treatment of non-parallel proofs, which might have affected memory usage at some point, but does not seem to make a difference with as little as 2GB RAM;
2010-08-04, by wenzelm
more precise CRITICAL sections;
2010-08-03, by wenzelm
removed unused Update_Time data (cf. ac94ff28e9e1);
2010-08-03, by wenzelm
modernized specifications;
2010-08-03, by wenzelm
eliminated Thy_Info.thy_ord, which is not really stable in interactive mode, since it depends on the somewhat accidental load order;
2010-08-03, by wenzelm
find_and_undo: no need to kill_thy again -- Thy_Info.toplevel_begin_theory does that initially (cf. 3ceccd415145);
2010-08-03, by wenzelm
renamed funny Library ROOT files back to default ROOT.ML -- ML files are no longer located via implicit load path (cf. 2b9bfa0b44f1);
2010-08-03, by wenzelm
tuned headers -- more precise load path;
2010-08-03, by wenzelm
theory loading: only the master source file is looked-up in the implicit load path;
2010-08-03, by wenzelm
load_thy: refer to physical master directory (not accumulated source import directory) and enable loading files relatively to that;
2010-08-03, by wenzelm
simplified/clarified Thy_Load path: search for master only, lookup other files relative to that;
2010-08-03, by wenzelm
only test prolog code examples if environment variable is set
2010-08-03, by bulwahn
Revised proof of long division contributed by Jesus Aransay.
2010-08-02, by ballarin
fix bug with Kodkodi < 1.2.14
2010-08-01, by blanchet
merged
2010-08-01, by blanchet
document new Nitpick options
2010-08-01, by blanchet
tweak datatype sym break code
2010-08-01, by blanchet
added manual symmetry breaking for datatypes
2010-08-01, by blanchet
change the order of the SAT solvers, from fastest to slowest
2010-07-31, by blanchet
started implementation of custom sym break
2010-07-31, by blanchet
clarify Nitpick's output in case of a potential counterexample
2010-07-31, by blanchet
added support for CryptoMiniSat
2010-07-31, by blanchet
gracefully handle the case where no integers occur in the formula and the "max" option is used
2010-07-30, by blanchet
merged
2010-08-01, by bulwahn
adding Code_Prolog theory to IsaMakefile and HOL-Library root file
2010-08-01, by bulwahn
inductive_simps learns to have more tool compliance
2010-08-01, by bulwahn
setting up Code_Prolog_Examples
2010-08-01, by bulwahn
adding queens and symbolic derivation example for prolog code generation
2010-08-01, by bulwahn
adding parsing of numbers; improving output of solution without free variables in prolog code generation
2010-08-01, by bulwahn
adding preprocessing of introduction rules to replace the constant Predicate.eq in the prolog code generation
2010-08-01, by bulwahn
adding basic arithmetic support for prolog code generation
2010-08-01, by bulwahn
adding numbers as basic term in prolog code generation
2010-08-01, by bulwahn
More consistent naming of locale api functions.
2010-07-31, by ballarin
Documentation of 'interpret' updated.
2010-07-31, by ballarin
print_interps shows interpretations in proofs.
2010-07-31, by ballarin
Interpretation in proofs supports mixins.
2010-07-31, by ballarin
Make registrations generic data.
2010-07-31, by ballarin
merged
2010-07-30, by blanchet
don't choke on synonyms when parsing SPASS's Flotter output + renamings;
2010-07-30, by blanchet
fix Mirabelle timeout
2010-07-29, by blanchet
make Mirabelle happy
2010-07-29, by blanchet
fix bug in the newly introduced "bound concealing" code
2010-07-29, by blanchet
handle division by zero gracefully (used to raise Unordered later on)
2010-07-29, by blanchet
use "explicit_apply" in the minimizer whenever it might make a difference to prevent freak failures;
2010-07-29, by blanchet
fix Meson's definition of first-orderness to prevent errors later on elsewhere (e.g. in Metis)
2010-07-29, by blanchet
handle schematic vars the same way in Sledgehammer as in Metis, to avoid unreplayable proofs
2010-07-29, by blanchet
revert exception throwing in FOL_SOLVE, since they're not caught anyway
2010-07-29, by blanchet
avoid "ATP Error: Error: blah" style messages
2010-07-29, by blanchet
avoid "_def_raw" theorems
2010-07-29, by blanchet
better error and minimizer output
2010-07-29, by blanchet
deal with chained facts more gracefully
2010-07-29, by blanchet
speed up the minimizer by using the time taken for the first iteration as a timeout for the following iterations, and fix a subtle bug in "string_for_failure"
2010-07-29, by blanchet
work around atomization failures
2010-07-29, by blanchet
fiddle with the fudge factors, to get similar results as before
2010-07-29, by blanchet
perform the presimplification done by Metis.make_nnf in Sledgehammer again, to deal with "If" and similar constructs
2010-07-29, by blanchet
fix bug with "=" vs. "fequal" introduced by last change (dddb8ba3a1ce)
2010-07-29, by blanchet
generate correct names for "$true" and "$false";
2010-07-29, by blanchet
don't assume canonical rule format
2010-07-29, by blanchet
avoid "clause" and "cnf" terminology where it no longer makes sense
2010-07-29, by blanchet
"axiom_clauses" -> "axioms" (these are no longer clauses)
2010-07-29, by blanchet
remove the "extra_clauses" business introduced in 19a5f1c8a844;
2010-07-29, by blanchet
adapting output for first solution
2010-07-29, by bulwahn
removing pointless type information in internal prolog terms
2010-07-29, by bulwahn
cleaning example file; more natural ordering of variable names
2010-07-29, by bulwahn
improving translation to prolog; restoring terms from prolog output; adding tracing support
2010-07-29, by bulwahn
working on parser for prolog reponse
2010-07-29, by bulwahn
querying for multiple solutions in values command for prolog execution
2010-07-29, by bulwahn
correcting scanning
2010-07-29, by bulwahn
adding values command and parsing prolog output
2010-07-29, by bulwahn
adding example file for prolog code generation; adding prolog code generation example to IsaMakefile
2010-07-29, by bulwahn
adding a mockup version for prolog code generation
2010-07-29, by bulwahn
exporting retrieval function for graph of introduction rules in the predicate compiler core
2010-07-29, by bulwahn
merged
2010-07-29, by haftmann
rebinding ref is illegal
2010-07-29, by haftmann
tuned example
2010-07-29, by haftmann
intermediate operation avoids invariance problem in Scala
2010-07-29, by haftmann
merged
2010-07-29, by blanchet
kill polymorphic "val"s
2010-07-29, by blanchet
improved ATP error handling some more
2010-07-29, by blanchet
shorter URL
2010-07-29, by blanchet
mention version numbers
2010-07-28, by blanchet
fiddled with usage text
2010-07-28, by blanchet
handle Perl and "libwww-perl" failures more gracefully, giving the user some clues about what goes on
2010-07-28, by blanchet
merged
2010-07-29, by haftmann
tuned printing of applications and let cascades
2010-07-29, by haftmann
checking Scala_imp
2010-07-29, by haftmann
proper unit type in transformed program
2010-07-29, by haftmann
merged
2010-07-29, by haftmann
merged
2010-07-28, by haftmann
tuned; added pretty numerals for code generation
2010-07-28, by haftmann
may use `int` in Isabelle runtime environment
2010-07-28, by haftmann
dropped dead code
2010-07-28, by haftmann
merged
2010-07-28, by blanchet
make Mirabelle happy
2010-07-28, by blanchet
renamed environment variable
2010-07-28, by blanchet
updated component name
2010-07-28, by blanchet
consequence of directory renaming
2010-07-28, by blanchet
rename directory
2010-07-28, by blanchet
minor refactoring
2010-07-28, by blanchet
minor refactoring
2010-07-28, by blanchet
updated Sledgehammer docs
2010-07-28, by blanchet
remove needless "-x" option, now that (1) we can't handle remote SPASS anymore; and (2) we can a priori parse the SPASS syntax in "Sledgehammer_Proof_Reconstruct" anyway
2010-07-28, by blanchet
remove "remote_spass" because there's no way to find out which clauses come from which facts + rename scripts
2010-07-28, by blanchet
fix bug in the SPASS Flotter hack, when a conjecture FOF is translated to several CNF clauses
2010-07-28, by blanchet
revive "e" and "remote_e"'s fact extraction so that it works with E 1.2 as well;
2010-07-28, by blanchet
more robust proof reconstruction
2010-07-28, by blanchet
adapt to new (?) TPTP output
2010-07-28, by blanchet
fix remote_vampire's proof reconstruction
2010-07-28, by blanchet
fix proof reconstruction for latest Vampire
2010-07-28, by blanchet
renaming
2010-07-28, by blanchet
support latest version of Vampire (1.0) locally
2010-07-28, by blanchet
improve detection of installed SPASS
2010-07-28, by blanchet
merged
2010-07-28, by wenzelm
merge
2010-07-27, by blanchet
compile
2010-07-27, by blanchet
minor refactoring
2010-07-27, by blanchet
standardize "Author" tags
2010-07-27, by blanchet
remove unused fun
2010-07-27, by blanchet
reorder ML files in theory
2010-07-27, by blanchet
get rid of "FOLClause" (obsoleted by FOF-enabled "FOLFormula")
2010-07-27, by blanchet
more refactoring
2010-07-27, by blanchet
kill needless tracing
2010-07-27, by blanchet
rename "ATP_Manager" ML module to "Sledgehammer";
2010-07-27, by blanchet
rename
2010-07-27, by blanchet
complete renaming of "Sledgehammer_TPTP_Format" to "ATP_Problem"
2010-07-27, by blanchet
renamed file
2010-07-27, by blanchet
move Sledgehammer-specific code out of "Sledgehammer_TPTP_Format"
2010-07-27, by blanchet
get rid of more dead wood
2010-07-27, by blanchet
implemented "sublinear" minimization algorithm
2010-07-27, by blanchet
extract sort constraints from FOFs properly;
2010-07-27, by blanchet
merged
2010-07-27, by haftmann
delete structure Basic_Record; avoid `record` in names in structure Record
2010-07-27, by haftmann
no polymorphic "var"
2010-07-27, by blanchet
merged
2010-07-27, by blanchet
shrink the "max_new_relevant_facts_per_iter" fudge factors, now that we count formulas and not clauses
2010-07-27, by blanchet
negate tfree conjecture
2010-07-27, by blanchet
handle Vampire's equality proxy axiom correctly
2010-07-27, by blanchet
simplify code
2010-07-27, by blanchet
prevent schematic variable clash in combinator-introduction code, when invoked from Sledgehammer (another consequence of the CNF -> FOF transition)
2010-07-26, by blanchet
remove obsolete field in record
2010-07-26, by blanchet
simplify code
2010-07-26, by blanchet
get rid of obsolete "axiom ID" component, since it's now always 0
2010-07-26, by blanchet
reintroduced more preprocessing steps to Sledgehammer, adapted to the new FOF setting
2010-07-26, by blanchet
added extensionalization to Sledgehammer, mimicking what the Clausifier used to do
2010-07-26, by blanchet
simplify code
2010-07-26, by blanchet
remove more Skolemization-aware code
2010-07-26, by blanchet
kill Skolem handling in Sledgehammer
2010-07-26, by blanchet
simplify "conjecture_shape" business, as a result of using FOF instead of CNF
2010-07-26, by blanchet
generate full first-order formulas (FOF) in Sledgehammer
2010-07-26, by blanchet
make TPTP generator accept full first-order formulas
2010-07-26, by blanchet
generate close formulas for SPASS, but not for the others (to avoid clutter)
2010-07-26, by blanchet
renamed internal function
2010-07-26, by blanchet
proof reconstruction for full FOF terms
2010-07-26, by blanchet
remove confusing line in SPASS output (because the axiom names are off -- bug in SPASS)
2010-07-26, by blanchet
reorder SPASS conjectures correctly, based on Flotter output
2010-07-26, by blanchet
Deleted an obsolete file
2010-07-27, by paulson
explicit Keyword.control markup for various control commands -- to prevent them from occurring in proof documents;
2010-07-28, by wenzelm
use file names relative to master directory of theory source -- Proof General can now handle that due to the ThyLoad.add_path deception (cf. 3ceccd415145);
2010-07-28, by wenzelm
simplified handling of update_time -- do not store within deps;
2010-07-27, by wenzelm
clarified register_thy: clean slate via kill_thy, more precise CRITICAL section;
2010-07-27, by wenzelm
updated keywords;
2010-07-27, by wenzelm
updated manual concerning theory loader;
2010-07-27, by wenzelm
theory loader: removed obsolete touch/outdate operations (require_thy no longer changes the database implicitly);
2010-07-27, by wenzelm
avoid repeated File.read for theory text (as before);
2010-07-27, by wenzelm
tuned messages and comments;
2010-07-27, by wenzelm
simplified Thy_Header.read -- include Source.of_string_limited here;
2010-07-27, by wenzelm
simplified/clarified theory loader: more explicit task management, kill old versions at start, commit results only in the very end, non-optional master dependency, do not store text in deps;
2010-07-27, by wenzelm
more precise stats;
2010-07-27, by wenzelm
merged
2010-07-26, by wenzelm
quickcheck images of goals under registration morphisms
2010-07-26, by haftmann
get_registrations interface
2010-07-26, by haftmann
restored unusual snd-biased merge/join policy -- required due to non-conservative code setups
2010-07-26, by haftmann
merged
2010-07-26, by haftmann
reactivated Scala check
2010-07-26, by haftmann
corrected range check once more
2010-07-26, by haftmann
added Code_Natural.thy
2010-07-26, by haftmann
reactivated Scala check; tuned import order
2010-07-26, by haftmann
reactivated Scala check
2010-07-26, by haftmann
modified namespace policy
2010-07-26, by haftmann
use Natural as index type for Haskell and Scala
2010-07-26, by haftmann
merged
2010-07-25, by blanchet
keep track of clause numbers for SPASS now that we generate FOF rather than CNF problems;
2010-07-23, by blanchet
first step in using "fof" rather than "cnf" in TPTP problems
2010-07-23, by blanchet
fix polymorphic "val"
2010-07-23, by blanchet
temporarily deactivating check for Scala
2010-07-24, by haftmann
another refinement chapter in the neverending numeral story
2010-07-24, by haftmann
inductive_cases: crude parallelization via Par_List.map;
2010-07-26, by wenzelm
modernized/unified some specifications;
2010-07-26, by wenzelm
Thy_Info.loaded_files: Thy_Load.loaded_files depends on master -- i.e. no files for finished theory;
2010-07-26, by wenzelm
simplified/clarified register_thy: more precise treatment of new dependencies, remove descendants;
2010-07-25, by wenzelm
simplified handling of theory begin/end wrt. toplevel and theory loader;
2010-07-25, by wenzelm
Thy_Load.check_loaded via Theory.at_end;
2010-07-25, by wenzelm
tuned;
2010-07-24, by wenzelm
moved basic thy file name operations from Thy_Load to Thy_Header;
2010-07-24, by wenzelm
moved management of auxiliary theory source files to Thy_Load -- as theory data instead of accidental loader state;
2010-07-24, by wenzelm
merged
2010-07-23, by wenzelm
avoid unreliable Haskell Int type
2010-07-23, by haftmann
proper subclass instead of sublocale
2010-07-23, by haftmann
repaired tool invocation
2010-07-23, by haftmann
observe standard conventions for doc-strings;
2010-07-23, by wenzelm
tuned message;
2010-07-22, by wenzelm
eliminated some unused Thy_Info operations;
2010-07-22, by wenzelm
refrain from generating <hr/> and from "hiding" it in isabelle.css -- the latter might be used in other situations as well;
2010-07-22, by wenzelm
generic external source files -- nothing special about ML here;
2010-07-22, by wenzelm
discontinued special treatment of ML files -- no longer complete extensions on demand;
2010-07-22, by wenzelm
eliminated obsolete/unused with_path(s) -- hardly usable because of CRITICAL;
2010-07-22, by wenzelm
tuned signature;
2010-07-22, by wenzelm
updated some headers;
2010-07-22, by wenzelm
merged
2010-07-22, by haftmann
dedicated exec ... syntax for open state monad (partly already introduces in d00a3f47b607)
2010-07-22, by haftmann
merged
2010-07-22, by wenzelm
more generous memory settings for scala check
2010-07-22, by haftmann
no polymorphic "var"s
2010-07-22, by blanchet
merged
2010-07-22, by bulwahn
adding checking of expected result for the tool quickcheck; annotated a few quickcheck examples
2010-07-21, by bulwahn
do a better job at Skolemizing in Nitpick, for TPTP FOF
2010-07-21, by blanchet
revert code that was submitted by mistake
2010-07-21, by blanchet
renamings + only need second component of name pool to reconstruct proofs
2010-07-21, by blanchet
rename "classrel" to "class_rel"
2010-07-21, by blanchet
rename "combtyp" constructors
2010-07-21, by blanchet
renamed "Literal" to "FOLLiteral"
2010-07-21, by blanchet
renamed "HOLClause" to "FOLClause" -- it's really a FOL clause with combinators
2010-07-21, by blanchet
merged
2010-07-21, by bulwahn
fixing quickcheck invocation in HOL-Mirabelle
2010-07-21, by bulwahn
hiding constants in Quickcheck_Types
2010-07-21, by bulwahn
adding a type for flat complete lattice to Quickcheck_Types
2010-07-21, by bulwahn
added new theories to IsaMakefile and ROOT.ML
2010-07-21, by bulwahn
adding Quickcheck examples for other quickcheck default types
2010-07-21, by bulwahn
adding Library theory for other quickcheck default types
2010-07-21, by bulwahn
removing obsolete ID in Quickcheck_Examples
2010-07-21, by bulwahn
correcting wellsortedness check and improving error message
2010-07-21, by bulwahn
using multiple default types in quickcheck
2010-07-21, by bulwahn
correcting merging of default_types
2010-07-21, by bulwahn
reordering quickcheck signature; exporting test_params and inspection function
2010-07-21, by bulwahn
changed default types to a list of types; extended quickcheck parameters to be a list of values to parse a list of default types
2010-07-21, by bulwahn
putting proof in the right context; adding if rewriting; tuned
2010-07-21, by bulwahn
load_thy: parallel parsing of units, which consist of statement/proof each;
2010-07-22, by wenzelm
eliminated some unreferenced identifiers;
2010-07-22, by wenzelm
tuned;
2010-07-22, by wenzelm
tuned comments;
2010-07-22, by wenzelm
replaced Source.of_list_limited by slightly more economic Source.of_string_limited;
2010-07-21, by wenzelm
deps_thy/load_thy: store compact text to reduce space by factor 12;
2010-07-21, by wenzelm
make SML/NJ happy, by adhoc type-constraints;
2010-07-21, by wenzelm
recovered benchmarks, which are not tested automatically;
2010-07-21, by wenzelm
made SML/NJ happy;
2010-07-21, by wenzelm
merged
2010-07-21, by wenzelm
abstract visualization of locale ingredients; all_locales yields proper locale identifiers
2010-07-21, by haftmann
tuned
2010-07-20, by haftmann
accomodate for scope of "as" binding in ML
2010-07-20, by haftmann
tuned code
2010-07-20, by haftmann
datatype classes are abstract
2010-07-20, by haftmann
less
more
|
(0)
-30000
-10000
-3000
-1000
-480
+480
+1000
+3000
+10000
+30000
tip