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.
make Nitpick tests more robust by specifying SAT solver, singlethreading (in Kodkod, not in Isabelle), and higher time limits
2009-12-14, by blanchet
make Nitpick "Core" test more conservative, to avoid problems on Larry's machine
2009-12-14, by blanchet
made sml/nj happy
2009-12-14, by haftmann
also sort verification conditions before printing
2009-12-14, by boehmes
print assertions in a more natural order
2009-12-13, by boehmes
removed unique ids -- now in session.scala;
2009-12-11, by wenzelm
merged
2009-12-11, by wenzelm
Subgoal.FOCUS (and variants): resulting goal state is normalized as usual for resolution;
2009-12-11, by wenzelm
Subgoal.FOCUS etc.: resulting goal state is normalized as usual for resolution;
2009-12-11, by wenzelm
merged
2009-12-11, by haftmann
repaired accident: do not forget module contents if there are no imports
2009-12-11, by haftmann
option width for Code_Target.code_of
2009-12-11, by haftmann
default_code_width is now proper theory data
2009-12-11, by haftmann
merged
2009-12-11, by boehmes
updated dependencies
2009-12-11, by boehmes
make assertion labels unique already when loading a verification condition,
2009-12-11, by boehmes
depend on HOL-SMT instead of HOL (makes tactic "smt" available for proofs)
2009-12-11, by boehmes
merged
2009-12-11, by haftmann
moved predicate rules to Predicate.thy; weakened default dest rule predicate1D (is not that reliable wrt. sets)
2009-12-11, by haftmann
avoid dependency on implicit dest rule predicate1D in proofs
2009-12-11, by haftmann
merged
2009-12-11, by haftmann
NEWS
2009-12-11, by haftmann
merged
2009-12-11, by haftmann
merged
2009-12-09, by haftmann
take and drop as projections of chop
2009-12-09, by haftmann
explicit lower bound for index
2009-12-09, by haftmann
merged
2009-12-11, by paulson
merged
2009-12-10, by paulson
streamlined proofs
2009-12-10, by paulson
fixed typo
2009-12-10, by paulson
merged
2009-12-10, by wenzelm
only invoke metisFT if metis failed
2009-12-10, by boehmes
added Imperative_HOL examples; added tail-recursive combinator for monadic heap functions; adopted code generation of references; added lemmas
2009-12-10, by bulwahn
merged
2009-12-09, by haftmann
each import resides in its own line
2009-12-09, by haftmann
using existing lattice classes
2009-12-09, by haftmann
added get_data;
2009-12-10, by wenzelm
sealed XML.Tree;
2009-12-10, by wenzelm
simplified Cygwin setup, assuming 1.7 registry layout (version 1.5 suffers from upcaseenv problem anyway);
2009-12-09, by wenzelm
slightly more robust and less ambitious version of install_fonts;
2009-12-09, by wenzelm
more robust Cygwin.config: actually check Wow6432Node, prefer explicit CYGWIN_ROOT in any case;
2009-12-09, by wenzelm
merged
2009-12-09, by blanchet
merged
2009-12-09, by blanchet
merged
2009-12-08, by blanchet
made Nitpick work also for people who import "Plain" instead of "Main"
2009-12-08, by blanchet
make Nitpick output the message "Hint: Maybe you forgot a type constraint?" only for syntactic classes
2009-12-07, by blanchet
keep future Isabelle application entry point;
2009-12-09, by wenzelm
merged
2009-12-09, by wenzelm
also consider the fully-typed version of metis for Mirabelle measurements
2009-12-08, by boehmes
merged
2009-12-08, by boehmes
made SML/NJ happy
2009-12-08, by boehmes
simplified notion of empty module name
2009-12-08, by haftmann
commit
2009-12-08, by haftmann
resorted code equations from "old" number theory version
2009-12-08, by haftmann
merged
2009-12-08, by haftmann
split off evaluation mechanisms in separte module Code_Eval
2009-12-07, by haftmann
register_fonts: more precise error handling;
2009-12-08, by wenzelm
added future;
2009-12-08, by wenzelm
depend on Java 1.6 after all;
2009-12-07, by wenzelm
basic support for IsabelleText fonts;
2009-12-07, by wenzelm
merged
2009-12-07, by haftmann
merged
2009-12-07, by haftmann
tuned inner structure
2009-12-07, by haftmann
merged Crude_Executable_Set into Executable_Set
2009-12-07, by haftmann
merged
2009-12-07, by blanchet
avoid using "prop_logic.ML" and "sat_solver.ML" twice (the other occurrence being in "FunDef.thy");
2009-12-07, by blanchet
better error message in Refute when specifying a non-existing SAT solver
2009-12-07, by blanchet
merged
2009-12-07, by wenzelm
updated certificate
2009-12-07, by boehmes
merged
2009-12-07, by haftmann
repaired read_const_expr, broken in 1e7ca47c6c3d
2009-12-07, by haftmann
merged
2009-12-07, by boehmes
verbose output of loaded data makes a clear distinction between new and already existing data (types, constants, axioms)
2009-12-07, by boehmes
faster preprocessing: before applying a step, test if it is applicable (normalization of binders, unfolding of abs/min/max definitions, lambda lifting, explicit application, monomorphization),
2009-12-03, by boehmes
merged
2009-12-06, by haftmann
tuned proofs
2009-12-06, by haftmann
tuned lattices theory fragements; generlized some lemmas from sets to lattices
2009-12-05, by haftmann
avoid lazy val with side-effects -- spurious null pointers!?
2009-12-07, by wenzelm
toString: more robust handling of null;
2009-12-07, by wenzelm
proper markup text for loc;
2009-12-06, by wenzelm
output_syms: permissive treatment of control symbols, cf. Scala version;
2009-12-06, by wenzelm
basic treatment of special control symbols;
2009-12-06, by wenzelm
elements: more convenient result;
2009-12-06, by wenzelm
more robust treatment of line breaks -- Java "split" has off semantics;
2009-12-06, by wenzelm
added auxiliary constructors;
2009-12-06, by wenzelm
added elements: Interator;
2009-12-06, by wenzelm
merged
2009-12-05, by wenzelm
merged
2009-12-05, by haftmann
tuned whitespace
2009-12-04, by haftmann
merged, resolving minor conflicts
2009-12-04, by haftmann
NEWS
2009-12-04, by haftmann
signatures for generated code; tuned
2009-12-04, by haftmann
tuned
2009-12-04, by haftmann
avoid misleading name "superarities"
2009-12-04, by haftmann
more speaking function names for Code_Printer; added doublesemicolon
2009-12-04, by haftmann
tuned code setup
2009-12-04, by haftmann
version of IsabelleMono that retains plain ASCII and ISO-LATIN-1 from Bitstream Vera;
2009-12-05, by wenzelm
output linefeed as </br> -- workaround problem with <pre> in Lobo Browser 0.98.4;
2009-12-05, by wenzelm
added markup for hidden text;
2009-12-05, by wenzelm
Basic HTML output.
2009-12-04, by wenzelm
output "'" as "'" which is a bit more portable ("'" is defined in XML/XHTML, but not in old-style HTML4);
2009-12-04, by wenzelm
fixed paths in Nitpick's ML file headers
2009-12-04, by blanchet
added soundness fix to Nitpick's history
2009-12-04, by blanchet
export symbols from Minipick (so I can use them in other programs)
2009-12-04, by blanchet
make proof work again
2009-12-04, by blanchet
fix soundness bug in Nitpick's "destroy_constrs" optimization
2009-12-04, by blanchet
merged, resolving minor conflict, and recovering sane state;
2009-12-04, by wenzelm
merged
2009-12-04, by wenzelm
merged
2009-12-04, by wenzelm
merged, resolving minor conflicts;
2009-12-04, by wenzelm
merged
2009-12-04, by haftmann
merged
2009-12-04, by haftmann
modernized structure Datatype_Aux
2009-12-04, by haftmann
tuned
2009-12-02, by haftmann
dropped some unused bindings
2009-11-30, by haftmann
modernized structures and tuned headers of datatype package modules; joined former datatype.ML and datatype_rep_proofs.ML
2009-11-30, by haftmann
more accurate linerarity
2009-11-30, by haftmann
merged
2009-11-30, by haftmann
Inl and Inr now with authentic syntax
2009-11-27, by haftmann
renamed former datatype.ML to datatype_data.ML
2009-11-27, by haftmann
renamed former datatype.ML to datatype_data.ML; datatype.ML provides uniform view on datatype.ML and datatype_rep_proofs.ML
2009-11-27, by haftmann
modernized; dropped ancient constant Part
2009-11-27, by haftmann
centralized sum type matter in Sum_Type.thy
2009-11-25, by haftmann
tuned
2009-11-25, by haftmann
bootstrap datatype_rep_proofs in Datatype.thy (avoids unchecked dynamic name references)
2009-11-25, by haftmann
merged
2009-11-25, by haftmann
normalized uncurry take/drop
2009-11-25, by haftmann
merged
2009-11-24, by haftmann
curried take/drop
2009-11-24, by haftmann
backported parts of abstract byte code verifier from AFP/Jinja
2009-11-24, by haftmann
added document_node;
2009-12-04, by wenzelm
document init_component shell function;
2009-12-04, by wenzelm
back to after-release mode;
2009-12-04, by wenzelm
back to main repository;
2009-12-04, by wenzelm
merged
2009-12-04, by wenzelm
merged
2009-12-04, by haftmann
added Crude_Executable_Set
2009-12-04, by haftmann
removed redundant lemma
2009-12-04, by nipkow
added remdups_filter lemma
2009-12-04, by nipkow
merged
2009-12-02, by haftmann
subst_signatures
2009-12-02, by haftmann
tuned
2009-12-02, by haftmann
exported build_tsig
2009-12-02, by haftmann
crude support for type aliasses and corresponding constant signatures
2009-12-02, by haftmann
generalized some lemmas
2009-12-02, by haftmann
added Crude_Executable_Set.thy
2009-12-02, by haftmann
read_dimacs_cnf_file can now read DIMACS files that contain successive
2009-12-01, by webertj
Expand nested abbreviations before applying dummy patterns.
2009-11-29, by kleing
Removed eq_to_mono2, added not_mono.
2009-11-27, by berghofe
Streamlined setup for monotonicity rules (no longer requires classical rules).
2009-11-27, by berghofe
Simplified treatment of monotonicity rules.
2009-11-27, by berghofe
removed obsolete test tags;
2009-12-03, by wenzelm
Added tag Isabelle2009-1 for changeset 6a973bd43949
2009-12-03, by wenzelm
slightly less ambitious settings, to avoid potential out-of-memory problem;
Isabelle2009-1
2009-12-02, by wenzelm
even higher proof-shell-quit-timeout -- saving main HOL takes 20s on a *fast* machine;
2009-11-30, by wenzelm
updated date;
2009-11-30, by wenzelm
more robust treatment of spaces in directory names;
2009-11-30, by wenzelm
adding subsection about the predicate compiler to the code generator tutorial
2009-11-30, by bulwahn
Added tag isa2009-1-test for changeset e1c262952b02
2009-11-29, by wenzelm
updated date;
2009-11-29, by wenzelm
Expand nested abbreviations before applying dummy patterns.
2009-11-29, by kleing
raised proof-shell-quit-timeout to accomodate bulky write-back images;
2009-11-29, by wenzelm
deactivated default for E_HOME, SPASS_HOME -- now configured as components;
2009-11-29, by wenzelm
double check file permissions of write-back image -- more robust for root or administrator on Cygwin;
2009-11-29, by wenzelm
tuned message;
2009-11-29, by wenzelm
added HOLCF image;
2009-11-29, by wenzelm
workaround for strange compiler crash of Poly/ML 5.0 and 5.1 at this point http://isabelle.in.tum.de/repos/isabelle/file/a2fc533175ff/src/HOL/Tools/Nitpick/nitpick_nut.ML#l997
2009-11-28, by wenzelm
updated generated files;
2009-11-28, by wenzelm
proper quoting of array expansion -- allow spaces in components;
2009-11-28, by wenzelm
added "sos";
2009-11-28, by wenzelm
PG version 3.7.1.1;
2009-11-28, by wenzelm
allow spaces within PROOFGENERAL_EMACS;
2009-11-28, by wenzelm
allow spaces within command-line arguments;
2009-11-28, by wenzelm
proper quotes;
2009-11-27, by wenzelm
more abstract handling of repository name;
2009-11-27, by wenzelm
more menu entries -- backport from PG 4.0 branch;
2009-11-27, by wenzelm
re-package Isabelle distribution with add-on components;
2009-11-27, by wenzelm
fixed csdp output parser
2009-11-26, by Philipp Meyer
additional menu entries;
2009-11-26, by wenzelm
Added tag isa2009-1-test for changeset 14ff44e21bec
2009-11-26, by wenzelm
adhoc delay after font installation -- increases chance that Emacs will actually see them;
2009-11-26, by wenzelm
implicit font installation for Mac OS;
2009-11-26, by wenzelm
modernized interface script for PG 3.7.1 -- backport from PG 4.0 branch;
2009-11-26, by wenzelm
patch for the infamous antiquotation font-lock problem of Proof General 3.7.1 with GNU Emacs, cf. http://proofgeneral.inf.ed.ac.uk/trac/ticket/236
2009-11-26, by wenzelm
refer to isabelle-release branch;
2009-11-25, by wenzelm
include HOL-SMT keywords;
2009-11-25, by wenzelm
tuned affiliation;
2009-11-25, by wenzelm
extended list of HOL-Boogie contributors
2009-11-25, by boehmes
only add nat/int conversion rules if necessary
2009-11-25, by boehmes
more generic explosion of options (also accept newlines, etc.)
2009-11-25, by boehmes
respect "unique" attribute: generate distinctness axioms
2009-11-25, by boehmes
fixed arity of some empty relations in Nitpick's Kodkod generator;
2009-11-24, by blanchet
fix soundness bug in "uncurry" option of Nitpick
2009-11-24, by blanchet
Added tag isa2009-1-test for changeset 4328de748fb2
2009-11-24, by wenzelm
some rearangement of load order to keep preferences adjacent -- slightly fragile;
2009-11-24, by wenzelm
use correct Isabelle version name in README file
2009-11-24, by blanchet
remove version number from Nitpick manual
2009-11-24, by blanchet
fix soundness bug in Nitpick's Kodkod generator for the relational composition case
2009-11-24, by blanchet
merged
2009-11-24, by blanchet
generate clearer atom names in Nitpick for types that end with a digit;
2009-11-24, by blanchet
Added tag isa2009-1-test for changeset 9db7854eafc7
2009-11-24, by wenzelm
fix soundness bug in Nitpick's handling of negative literals (e.g., -1::rat)
2009-11-24, by blanchet
consisten upper/lower case
2009-11-24, by haftmann
merge
2009-11-24, by blanchet
fixed soundness bug / type error in handling of unpolarized (co)inductive predicates in Nitpick
2009-11-24, by blanchet
removed "nitpick_def" attributes from (r)trancl(p), since "Nitpick.thy" overrides these
2009-11-24, by blanchet
fix Nitpick soundness bug related to "finite (UNIV::'a set)" where "'a" is constrained by a sort to be infinite
2009-11-23, by blanchet
fixed soundness bug in Nitpick's handling of typedefs
2009-11-23, by blanchet
multiplatform polyml.tar.gz;
2009-11-23, by wenzelm
updated keywords;
2009-11-23, by wenzelm
more tuning for release;
2009-11-23, by wenzelm
added command 'ProofGeneral.pr' for PG 4.0;
2009-11-23, by wenzelm
merged
2009-11-23, by bulwahn
improving the setup for the tabled transitive closure thanks to usage of Andreas Lochbihler
2009-11-23, by bulwahn
updated for release;
2009-11-23, by wenzelm
Generated files.
2009-11-23, by ballarin
Typos in documenation.
2009-11-23, by ballarin
ANNOUNCE
2009-11-23, by haftmann
merge
2009-11-23, by blanchet
fix Nitpick soundness bugs related to integration (in particular, "code_numeral")
2009-11-23, by blanchet
generate arguments of relational composition in the right order in Nitpick
2009-11-23, by blanchet
CONTRIBUTORS
2009-11-23, by haftmann
merged
2009-11-23, by haftmann
tuned NEWS
2009-11-23, by haftmann
do not add host suffix -- it is appended by test framework
2009-11-23, by krauss
documented size_change in isar-ref manual
2009-11-23, by krauss
clarified; checked
2009-11-23, by krauss
mentioned method size_change in function tutorial
2009-11-23, by krauss
eliminated dead code and some unused bindings, reported by polyml
2009-11-23, by krauss
fixed a Kodkod generation exception in Nitpick, reported by a Karlsruhe user
2009-11-23, by blanchet
fixed soundness bug in Nitpick that occurred because unrolled predicate iterators were considered to be a "precise" type
2009-11-23, by blanchet
improved annotated type of equality in Nitpick's monotonicity check, based on a discovery by Alex
2009-11-23, by blanchet
fixed error in Nitpick's "star_linear_preds" optimization, which resulted in an ill-typed term;
2009-11-23, by blanchet
merged
2009-11-22, by wenzelm
more uniform view on various number theory refinement steps
2009-11-22, by haftmann
Merged.
2009-11-22, by ballarin
Generated latex code.
2009-11-22, by ballarin
Updated locale documentation.
2009-11-22, by ballarin
made SML/NJ happy;
2009-11-22, by wenzelm
remove presently unused Isabelle application;
2009-11-22, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip