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.
merged
2010-06-06, by wenzelm
tuned;
2010-06-06, by wenzelm
removed obsolete dry-run option;
2010-06-06, by wenzelm
Added tag isa2009-2-test1 for changeset d1cdbc7524b6
2010-06-06, by wenzelm
merged
2010-06-05, by haftmann
avoid "$"
2010-06-04, by haftmann
tuned whitespace
2010-06-04, by haftmann
avoid flowerish abbreviation
2010-06-04, by haftmann
merged
2010-06-04, by wenzelm
merge
2010-06-04, by blanchet
don't raise Option.Option if assumptions contain schematic variables
2010-06-04, by blanchet
recongize one more outcome string for "remote_vampire"
2010-06-04, by blanchet
"print_vars_terms" wasn't doing its job properly;
2010-06-04, by blanchet
merged
2010-06-04, by blanchet
made "clausify" attribute a legacy feature;
2010-06-04, by blanchet
made "neg_clausify" a legacy feature
2010-06-04, by blanchet
kill active Sledgehammer threads when running minimize, to avoid confusing the user with too much output
2010-06-04, by blanchet
redid the Isar proofs using the latest Sledgehammer, eliminating the last occurrences of "neg_clausify" in proofs
2010-06-04, by blanchet
fix bugs in Sledgehammer's Isar proof "redirection" code
2010-06-04, by blanchet
handle Vampire's definitions smoothly
2010-06-02, by blanchet
fix bug in direct Isar proofs, which was exhibited by the "BigO" example
2010-06-02, by blanchet
honor "xsymbols"
2010-06-02, by blanchet
kill another neg_clausify proof
2010-06-02, by blanchet
show types in Isar proofs, but not for free variables;
2010-06-02, by blanchet
give more helpful error message
2010-06-02, by blanchet
first proposal for a announcement
2010-06-04, by haftmann
NEWS (more strict internal axioms/defs format)
2010-06-04, by krauss
one all-inclusive bundle for each platform;
2010-06-04, by wenzelm
more robust handling of additional type variables: warning, more canonical order, drop mixfix syntax if implicit type arguments are introduced (to avoid delusion due to shifted arguments);
2010-06-04, by wenzelm
tuned warning;
2010-06-04, by wenzelm
less ambitious settings;
2010-06-04, by wenzelm
spelling;
2010-06-04, by wenzelm
do not open Proofterm, which is very ould style;
2010-06-03, by wenzelm
eliminated ML structure alias;
2010-06-03, by wenzelm
tuned default perspective;
2010-06-03, by wenzelm
tracing in aliceblue;
2010-06-03, by wenzelm
discontinued obsolete Isar.context() -- long superseded by @{context};
2010-06-03, by wenzelm
diagnostic commands 'ML_val' and 'ML_command' may refer to antiquotations @{Isar.state} and @{Isar.goal};
2010-06-03, by wenzelm
allow qualified names;
2010-06-03, by wenzelm
CONTRIBUTORS
2010-06-03, by krauss
clarified
2010-06-03, by krauss
mention unconstrain in NEWS
2010-06-03, by krauss
merged
2010-06-02, by haftmann
hide default, map_entry, map_default
2010-06-02, by haftmann
improved parallelism of proof term normalization;
2010-06-02, by wenzelm
always unconstrain thm proofs;
2010-06-02, by wenzelm
replaced ML pokes by explicit usedir -p;
2010-06-02, by wenzelm
merged
2010-06-02, by haftmann
absolute import -- must work with Main.thy / HOL-Proofs
2010-06-02, by haftmann
avoid duplicate import
2010-06-02, by haftmann
HOL-Proofs is based in Main.thy
2010-06-02, by haftmann
dropped lemma duplicate
2010-06-02, by haftmann
msetprod_empty, msetprod_singleton
2010-06-02, by haftmann
induction over non-empty lists
2010-06-02, by haftmann
removed dependency of Euclid on Old_Number_Theory
2010-06-02, by haftmann
modernized
2010-06-02, by haftmann
removed obsolete usedir -p 1 option;
2010-06-02, by wenzelm
actually test smlnj;
2010-06-02, by wenzelm
updated keywords;
2010-06-02, by wenzelm
Added tag isa2009-2-test0 for changeset 935c75359742
2010-06-02, by wenzelm
more CONTRIBUTORS;
2010-06-02, by wenzelm
merged
2010-06-02, by wenzelm
Hilbert_Classical: disable multithreading altogether, otherwise proof normalization will fork futures independently of Goal.parallel_proofs;
2010-06-02, by wenzelm
merged
2010-06-02, by nipkow
added lemmas
2010-06-02, by nipkow
merged
2010-06-02, by blanchet
merge
2010-06-02, by blanchet
fix parameter settings
2010-06-02, by blanchet
merged
2010-06-01, by blanchet
merged
2010-06-01, by blanchet
update NEWS
2010-06-01, by blanchet
fix Nitpick soundness bug regarding The and Eps
2010-06-01, by blanchet
added examples/tests for THE and SOME
2010-06-01, by blanchet
cosmetics
2010-06-01, by blanchet
adapt example
2010-06-01, by blanchet
fix code that used to raise an exception if bound variables were given a finite function type, because the old vs. new bound variable types were confused
2010-06-01, by blanchet
improved precision of "set" based on an example from Lukas
2010-06-01, by blanchet
remove debug output
2010-06-01, by blanchet
removed "nitpick_intro" attribute -- Nitpick noew uses Spec_Rules instead
2010-06-01, by blanchet
subsumed by NEWS -- for older history, see previous versions of Nitpick
2010-06-01, by blanchet
don't show spurious "..." in Nitpick's output for free variables of set type (e.g., P (op +) example from Manual_Nits.thy); undoes parts of 38ba15040455, which was too aggressive
2010-06-01, by blanchet
honor xsymbols in Nitpick
2010-06-01, by blanchet
added "atoms" option to Nitpick (request from Karlsruhe) + wrap Refute. functions to "nitpick_util.ML"
2010-06-01, by blanchet
document new option
2010-06-01, by blanchet
make Nitpick handle multiple typedef entries for same typedef
2010-06-01, by blanchet
remove comment
2010-06-01, by blanchet
thread along context instead of theory for typedef lookup
2010-06-01, by blanchet
obsolete FIXME
2010-05-31, by blanchet
move SAT solver warning from every invocation of SAT solver to the tool, Refute, that uses it;
2010-05-31, by blanchet
don't include any axioms for "TYPE" in Nitpick
2010-05-31, by blanchet
dropped obsolete script
2010-06-02, by haftmann
normalize and postprocess proof body in a separate future, taking care of platforms without multithreading (greately improves parallelization in general without the overhead of promised proofs, cf. usedir -q 0);
2010-06-02, by wenzelm
merged
2010-06-02, by haftmann
avoid store flag in add_* operations
2010-06-01, by haftmann
arities: no need to maintain original codomain (cf. f795c1164708) -- completion happens in axclass.ML;
2010-06-01, by wenzelm
merged
2010-06-01, by wenzelm
do not expose store flag of AxClass.add_*
2010-06-01, by haftmann
merged
2010-06-01, by haftmann
adapted to changes
2010-06-01, by haftmann
capitalized type variables; added yield as keyword
2010-06-01, by haftmann
brackify_infix etc.: no break before infix operator -- eases survival in Scala
2010-06-01, by haftmann
basic support for sub/superscript token markup -- NB: need to maintain extended token types eagerly, since jEdit occasionally reinstalls a style array that is too short;
2010-06-01, by wenzelm
use local /home/isatest/polyml-5.3.0 on atbroy102 to avoid problems with the SMB filesystem via homebroy;
2010-06-01, by wenzelm
uniform ML environment setup for Isar and PG;
2010-06-01, by wenzelm
merged
2010-06-01, by berghofe
Renamed TypeInfer to Type_Infer.
2010-06-01, by berghofe
merged
2010-06-01, by berghofe
assign now applies meet before update_new to avoid misleading error message.
2010-06-01, by berghofe
Tuned.
2010-06-01, by berghofe
Adapted to new format of proof terms containing explicit proofs of class membership.
2010-06-01, by berghofe
classrel and arity theorems are now stored under proper name in theory. add_arity and
2010-06-01, by berghofe
- outer_constraints with original variable names, to ensure that argsP is consistent with args
2010-06-01, by berghofe
outer_constraints with original variable names, to ensure that argsP is consistent with args
2010-06-01, by berghofe
- Equality check on propositions after lookup of theorem now takes type variable
2010-06-01, by berghofe
Use Proofterm.forall_intr_proof' instead of locally defined forall_intr_prf.
2010-06-01, by berghofe
- Added extra flag to read_term and read_proof functions that allows to parse (proof)terms in which
2010-06-01, by berghofe
merged
2010-06-01, by wenzelm
merged
2010-06-01, by haftmann
corrected printing of characters
2010-06-01, by haftmann
corrected implementation
2010-06-01, by haftmann
added Scala code setup
2010-06-01, by haftmann
tuned code setup
2010-06-01, by haftmann
keep structure ThyLoad for the sake of Proof General;
2010-06-01, by wenzelm
added random instance for word
2010-06-01, by haftmann
notes on Isabelle/jEdit;
2010-05-31, by wenzelm
remove presently unused Isabelle application;
2010-05-31, by wenzelm
modernized some structure names, keeping a few legacy aliases;
2010-05-31, by wenzelm
merged
2010-05-31, by wenzelm
merge
2010-05-31, by blanchet
fix handling of "split" w.r.t. new definition + fix exception handling w.r.t. "expect" option
2010-05-31, by blanchet
updated generated files
2010-05-31, by haftmann
clarified
2010-05-31, by haftmann
adjusted
2010-05-31, by haftmann
terminate ML compiler input produced by ML_Lex.read (cf. 85e864045497);
2010-05-31, by wenzelm
Toplevel.run_command: reraise Interrupt, to terminate the Isar_Document.execution and not store a failed attempt;
2010-05-31, by wenzelm
merged
2010-05-31, by wenzelm
Typo in locales tutorial.
2010-05-30, by ballarin
Theory_Target.pretty: more markup;
2010-05-31, by wenzelm
tuned abbrevs for long arrows, according to usual ASCII syntax;
2010-05-31, by wenzelm
more flexibile font size via CSS <style> instead of old <font> element;
2010-05-31, by wenzelm
tuned;
2010-05-31, by wenzelm
control tooltip font via Swing HTML, with tooltip-font-size property;
2010-05-30, by wenzelm
added HTML.encode (in Scala), similar to HTML.output in ML;
2010-05-30, by wenzelm
one extra space to accomodate symbolic indentifiers etc.;
2010-05-30, by wenzelm
replaced ML_Lex.read_antiq by more concise ML_Lex.read, which includes full read/report with explicit position information;
2010-05-30, by wenzelm
more detailed token markup, including command kind as sub_kind;
2010-05-30, by wenzelm
tuned;
2010-05-30, by wenzelm
separate markup for ML delimiters;
2010-05-30, by wenzelm
less pschedelic token markup;
2010-05-30, by wenzelm
simplified command/keyword markup;
2010-05-30, by wenzelm
markup non-identifier keyword as operator;
2010-05-30, by wenzelm
Isabelle_Process: do not enforce future_terminal_proof by default -- no error propagation yet;
2010-05-30, by wenzelm
more basic default behaviour of ENTER, HOME, END;
2010-05-30, by wenzelm
tuned messages;
2010-05-29, by wenzelm
do not highlight ignored command spans;
2010-05-29, by wenzelm
more explicit handling of document;
2010-05-29, by wenzelm
explicit markup for forked goals, as indicated by Goal.fork;
2010-05-29, by wenzelm
avoid :\ which is not tail-recursive and tends to overflow the tiny JVM stack, which is not resizable at runtime;
2010-05-29, by wenzelm
define_state/new_state: provide state immediately, which is now lazy;
2010-05-29, by wenzelm
force_result within the current execution context -- avoids overhead of potential thread context switch and robustifies Interrupt handling;
2010-05-29, by wenzelm
future result: retain plain Interrupt for vacuous group exceptions;
2010-05-29, by wenzelm
remove two examples, now that the definition of "fst" and "snd" has changed
2010-05-28, by blanchet
merged
2010-05-28, by wenzelm
Got rid of a warning about duplicate rewrite rules.
2010-05-28, by webertj
accumulate only local results -- no proper history support yet;
2010-05-28, by wenzelm
avoid deprecated Iterator.fromArray;
2010-05-28, by wenzelm
more compiler warnings;
2010-05-28, by wenzelm
eliminated hard tabs;
2010-05-28, by wenzelm
assume given SCALA_HOME, e.g. from component settings or external setup;
2010-05-28, by wenzelm
merged
2010-05-28, by wenzelm
merged
2010-05-28, by blanchet
make sure chained facts appear in Isar proofs generated by Sledgehammer -- otherwise the proof won't work
2010-05-28, by blanchet
Nitpick: show "..." in datatype values (e.g., [{0::nat, ...}]), since these are really equivalence classes
2010-05-27, by blanchet
make Nitpick "show_all" option behave less surprisingly
2010-05-27, by blanchet
merged
2010-05-28, by haftmann
avoid reference to thm PairE
2010-05-28, by haftmann
more coherent theory structure; tuned headings
2010-05-28, by haftmann
made SML/NJ quite happy;
2010-05-28, by wenzelm
reuse main view.font from jEdit;
2010-05-28, by wenzelm
deleted some old fonts;
2010-05-28, by wenzelm
also set font for printing, which actually works out of the box;
2010-05-28, by wenzelm
lib/Tools/makeall does not hardiwre logics;
2010-05-28, by wenzelm
discontinued Sun/Solaris tests;
2010-05-28, by wenzelm
some updates for release;
2010-05-28, by wenzelm
merged
2010-05-27, by wenzelm
added function update examples and set examples
2010-05-27, by boehmes
updated SMT certificates
2010-05-27, by boehmes
sort signature in SMT-LIB output (improves sharing of SMT certificates: goals of the same logical structure are translated into equal SMT-LIB benchmarks)
2010-05-27, by boehmes
merged
2010-05-27, by boehmes
renamed constant "apply" to "fun_app" (which is closer to the related "fun_upd")
2010-05-27, by boehmes
made script executable
2010-05-27, by boehmes
use Z3's builtin support for div and mod
2010-05-27, by boehmes
moved SMT into the HOL image
2010-05-27, by boehmes
slightly odd workaround to ignore markup that is typically displaced;
2010-05-27, by wenzelm
substantial performance improvement by avoiding "re-ified" execution structure via future dependencies, instead use singleton execution (dummy future) that forces lazy state updates bottom-up;
2010-05-27, by wenzelm
further formal thread-safety (follow-up to 88300168baf8) -- in practice there is only a single Isar toplevel loop, but this is not enforced;
2010-05-27, by wenzelm
renamed structure PrintMode to Print_Mode, keeping the old name as legacy alias for some time;
2010-05-27, by wenzelm
renamed structure TypeInfer to Type_Infer, keeping the old name as legacy alias for some time;
2010-05-27, by wenzelm
misc updates for release;
2010-05-27, by wenzelm
constant Rat.normalize needs to be qualified;
2010-05-27, by wenzelm
merged
2010-05-27, by wenzelm
merged
2010-05-27, by haftmann
dropped legacy theorem bindings
2010-05-26, by haftmann
dropped legacy theorem bindings
2010-05-26, by haftmann
dropped legacy theorem bindings
2010-05-26, by haftmann
dropped legacy theorem bindings
2010-05-26, by haftmann
dropped legacy theorem bindings
2010-05-26, by haftmann
normalized references to constant "split"
2010-05-26, by haftmann
Revise locale test theory layout.
2010-05-26, by ballarin
Merge mixins of distinct interpretations with same base.
2010-05-26, by ballarin
indicate prospective properties;
2010-05-27, by wenzelm
clarified auto_update vs. update;
2010-05-27, by wenzelm
more reactive message handling, notably for follow_caret mode;
2010-05-27, by wenzelm
Command.toString: include id for debugging;
2010-05-27, by wenzelm
merged
2010-05-26, by wenzelm
refer to polyml-5.3.0-old for ppc-darwin;
2010-05-26, by wenzelm
try logical and theory abstraction before full abstraction (avoids warnings of linarith)
2010-05-26, by boehmes
updated SMT certificates
2010-05-26, by boehmes
hide constants and types introduced by SMT,
2010-05-26, by boehmes
more convenient order of code equations
2010-05-26, by haftmann
misc updates for release;
2010-05-26, by wenzelm
eliminated obsolete priority message from Isabelle_Process protocol;
2010-05-25, by wenzelm
moved ML files where they are actually used;
2010-05-25, by wenzelm
renamed HOLCF/Library/ROOT.ML to HOLCF/Library/HOLCF_Library_ROOT.ML to avoid accidental uses of this ML file via the load path -- see also d7711be8c3a9 (obsolete) and ccae4ecd67f4;
2010-05-25, by wenzelm
eliminated slightly odd Library/Library session setup (cf. d7711be8c3a9) which is obsolete due to usedir -f HOL_Library_ROOT.ML;
2010-05-25, by wenzelm
eliminated various catch-all exception patterns, guessing at the concrete exeptions that are intended here;
2010-05-25, by wenzelm
tuned -- avoid catch-all exception pattern;
2010-05-25, by wenzelm
updated generated files;
2010-05-25, by wenzelm
merged
2010-05-25, by wenzelm
merged
2010-05-24, by webertj
Typo fixed.
2010-05-24, by webertj
move HOLCF/Sum_Cpo.thy to HOLCF/Library
2010-05-24, by huffman
move Strict_Fun and Stream theories to new HOLCF/Library directory; add HOLCF/Library to search path
2010-05-24, by huffman
move unused pattern match syntax stuff into HOLCF/ex
2010-05-24, by huffman
rename type 'a maybe to 'a match; rename Fixrec.return to Fixrec.succeed
2010-05-24, by huffman
more lemmas
2010-05-24, by haftmann
induction and case rules
2010-05-24, by haftmann
Store registrations in efficient data structure.
2010-05-24, by ballarin
Avoid recomputation of registration instance for lookup.
2010-05-24, by ballarin
Consistently use equality for registration lookup.
2010-05-24, by ballarin
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip