Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+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.
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
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip