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.
moving options; tuned
2010-08-26, by bulwahn
added generation of predicates for size-limited enumeration of values
2010-08-26, by bulwahn
NEWS
2010-08-26, by haftmann
merged
2010-08-26, by haftmann
formerly unnamed infix impliciation now named HOL.implies
2010-08-26, by haftmann
merged
2010-08-26, by haftmann
proper passing of optional module name
2010-08-26, by haftmann
For sublocale it is sufficient to reconsider ancestors of the target.
2010-08-26, by ballarin
only print qualified implicits
2010-08-26, by haftmann
merged
2010-08-26, by haftmann
stub for (later) correct deresolving of class method names
2010-08-26, by haftmann
tuned serializer interface
2010-08-26, by haftmann
private version of commas, cf. printmode
2010-08-26, by haftmann
merged
2010-08-26, by haftmann
merged
2010-08-26, by haftmann
re-added accidental omission
2010-08-26, by haftmann
tuned includes
2010-08-26, by haftmann
prevent line breaks after Scala symbolic operators
2010-08-26, by haftmann
corrected semantics of presentation_stmt_names; do not print includes on presentation selection
2010-08-26, by haftmann
code_include Scala: qualify module nmae
2010-08-26, by haftmann
merged
2010-08-25, by haftmann
preliminary implementation of hierarchical module name space
2010-08-25, by haftmann
tuned
2010-08-25, by haftmann
proper context for various Thy_Output options, via official configuration options in ML and Isar;
2010-08-27, by wenzelm
Thy_Output: options based on proper context, although Thy_Output.add_wrapper still allows to maintain old-style wrapper combinators (setmp_CRITICAL etc.);
2010-08-27, by wenzelm
eliminated old 'local' command;
2010-08-27, by wenzelm
more uniform descriptions, which end up in the collective output of 'print_attributes' for example;
2010-08-26, by wenzelm
Fast_Lin_Arith.number_of: more conventional merge that prefers the left side -- note that former ordering wrt. serial numbers makes it depend on accidental load order;
2010-08-26, by wenzelm
slightly more abstract data handling in Fast_Lin_Arith;
2010-08-26, by wenzelm
theory data merge: prefer left side uniformly;
2010-08-26, by wenzelm
tuned;
2010-08-26, by wenzelm
simplification/standardization of some theory data;
2010-08-26, by wenzelm
misc tuning and simplification, notably theory data;
2010-08-26, by wenzelm
renamed Local_Theory.theory(_result) to Local_Theory.background_theory(_result) to emphasize that this belongs to the infrastructure and is rarely appropriate in user-space tools;
2010-08-26, by wenzelm
renamed ProofContext.theory(_result) to ProofContext.background_theory(_result) to emphasize that this belongs to the infrastructure and is rarely appropriate in user-space tools;
2010-08-26, by wenzelm
standardized Context.copy_thy to Theory.copy alias, with slightly more direct way of using it;
2010-08-26, by wenzelm
merged
2010-08-26, by wenzelm
merged
2010-08-26, by blanchet
consider "locality" when assigning weights to facts
2010-08-26, by blanchet
add a bonus for chained facts, since they are likely to be relevant;
2010-08-26, by blanchet
merged
2010-08-26, by blanchet
add a penalty for lambda-abstractions;
2010-08-26, by blanchet
renaming
2010-08-26, by blanchet
fiddle with relevance filter
2010-08-26, by blanchet
update docs
2010-08-25, by blanchet
reorganize options regarding to the relevance threshold and decay
2010-08-25, by blanchet
make relevance filter work in term of a "max_relevant" option + use Vampire SOS;
2010-08-25, by blanchet
simplify more code
2010-08-25, by blanchet
cosmetics
2010-08-25, by blanchet
get rid of "defs_relevant" feature;
2010-08-25, by blanchet
make SML/NJ happy
2010-08-25, by blanchet
renamed "relevance_convergence" to "relevance_decay"
2010-08-25, by blanchet
make sure that "undo_ascii_of" is the inverse of "ascii_of", also for non-printable characters -- and avoid those in ``-style facts
2010-08-24, by blanchet
better workaround for E's off-by-one-second issue
2010-08-24, by blanchet
merged
2010-08-26, by bulwahn
renaming variables to conform to prolog names
2010-08-25, by bulwahn
changing hotel trace definition; adding simple handling of numerals on natural numbers
2010-08-25, by bulwahn
added quickcheck generator for prolog generation; first example of counterexample search with prolog for hotel key card system
2010-08-25, by bulwahn
moving preprocessing to values in prolog generation
2010-08-25, by bulwahn
invocation of values for prolog execution does not require invocation of code_pred anymore
2010-08-25, by bulwahn
adding hotel keycard example for prolog generation
2010-08-25, by bulwahn
improving output of set comprehensions; adding style_check flags
2010-08-25, by bulwahn
improving ensure_groundness in prolog generation; added further example
2010-08-25, by bulwahn
adding very basic transformation to ensure groundness before negations
2010-08-25, by bulwahn
Markup_Tree.select: uniform treatment of root_range wrt. singularities, yielding empty result stream;
2010-08-26, by wenzelm
tuned signature;
2010-08-26, by wenzelm
Pretty: tuned markup objects;
2010-08-25, by wenzelm
tuned;
2010-08-25, by wenzelm
organized markup properties via apply/unapply patterns;
2010-08-25, by wenzelm
added some proof state markup, notably number of subgoals (e.g. for indentation);
2010-08-25, by wenzelm
ML_Context.eval: produce antiquotation environment preferably in invisible context, to avoid displaced report messages from ML_Compiler;
2010-08-25, by wenzelm
merged
2010-08-25, by wenzelm
tuned code
2010-08-25, by Christian Urban
quotient package: deal correctly with frees in lifted theorems
2010-08-25, by Christian Urban
approximation_oracle: actually match true/false in ML, not arbitrary values;
2010-08-25, by wenzelm
renamed Simplifier.simproc(_i) to Simplifier.simproc_global(_i) to emphasize that this is not the real thing;
2010-08-25, by wenzelm
more precise Command.State accumulation;
2010-08-25, by wenzelm
eliminated some old camel case stuff;
2010-08-25, by wenzelm
some attempts to recover Isabelle/ML style from the depths of time;
2010-08-25, by wenzelm
keep persistent production tables as immutable vectors -- potential performance improvement on modern hardware;
2010-08-25, by wenzelm
select tangible text ranges here -- more robust against ongoing changes of the markup query model
2010-08-25, by wenzelm
structure Thm: less pervasive names;
2010-08-25, by wenzelm
discontinued obsolete 'global' and 'local' commands;
2010-08-25, by wenzelm
merged
2010-08-25, by wenzelm
merged
2010-08-25, by hoelzl
moved generic lemmas in Probability to HOL
2010-08-24, by hoelzl
merged
2010-08-25, by wenzelm
traling newline on standard output
2010-08-25, by haftmann
Quotient Package / lemma for regularization of bex1_rel for equivalence relations
2010-08-25, by Cezary Kaliszyk
merged
2010-08-24, by blanchet
make Mirabelle happy
2010-08-24, by blanchet
compute names lazily;
2010-08-24, by blanchet
clean handling of whether a fact is chained or not;
2010-08-24, by blanchet
don't backtick facts that contain schematic variables, since this doesn't work (for some reason)
2010-08-24, by blanchet
quote facts whose names collide with a keyword or command name (cf. "subclass" in "Jinja/J/TypeSafe.thy")
2010-08-24, by blanchet
revert this idea of automatically invoking "metisFT" when "metis" fails;
2010-08-24, by blanchet
use matching of types than just equality - this is needed in nominal to cope with type variables
2010-08-24, by Christian Urban
merge
2010-08-24, by blanchet
cosmetics
2010-08-24, by blanchet
use a soft time limit for E
2010-08-24, by blanchet
make remote ATP versions more robust, by starting with "preferred" version numbers and falling back on any version
2010-08-24, by blanchet
cosmetics
2010-08-23, by blanchet
optimize fact filter some more
2010-08-23, by blanchet
cache previous iteration's weights, and keep track of what's dirty and what's clean;
2010-08-23, by blanchet
modified relevance filter
2010-08-23, by blanchet
adjust fudge factors in the light of experiments
2010-08-23, by blanchet
invert semantics of "relevance_convergence", to make it more intuitive
2010-08-23, by blanchet
if no facts were selected on first iteration, try again with a lower threshold
2010-08-23, by blanchet
weed out junk in relevance filter
2010-08-23, by blanchet
no need for "eq" facts -- good old "=" is good enough for us
2010-08-23, by blanchet
revert unintended change
2010-08-23, by blanchet
destroy elim rules before checking for finite exhaustive facts
2010-08-23, by blanchet
prevent double inclusion of the fact "True_or_False" in TPTP problems
2010-08-23, by blanchet
merged
2010-08-24, by haftmann
tuned
2010-08-24, by haftmann
merged
2010-08-23, by haftmann
dropped pre_post_conv
2010-08-23, by haftmann
use conv alias
2010-08-23, by haftmann
preliminary versions of static_eval_conv(_simple)
2010-08-23, by haftmann
use Code_Thingol.static_eval_conv_simple
2010-08-23, by haftmann
added static_eval_conv
2010-08-23, by haftmann
refined and unified naming convention for dynamic code evaluation techniques
2010-08-23, by haftmann
tap_thy conversional
2010-08-23, by haftmann
dropped now obsolete purge_data -- happens implicitly on change of theory identity
2010-08-23, by haftmann
merged
2010-08-24, by bulwahn
introducing simplification equations for inductive sets; added data structure for storing equations; rewriting retrieval of simplification equation for inductive predicates and sets
2010-08-23, by bulwahn
added support for xsymbol syntax for mode annotations in code_pred command
2010-08-23, by bulwahn
tuned raw Sidekick output;
2010-08-25, by wenzelm
Text.Range.is_singleton;
2010-08-24, by wenzelm
Markup_Tree.+: new info tends to sink to bottom, where it is prefered by select;
2010-08-24, by wenzelm
tuned;
2010-08-24, by wenzelm
Markup_Tree.select: more straight-forward recursion producing one main stream, avoid fragmentation of parent info due to ignored subtree;
2010-08-24, by wenzelm
tuned root markup;
2010-08-24, by wenzelm
misc tuning of important special cases;
2010-08-23, by wenzelm
Rewrite the Probability theory.
2010-08-23, by hoelzl
merged
2010-08-23, by wenzelm
merged
2010-08-23, by blanchet
use different name for debugging purposes
2010-08-23, by blanchet
perform eta-expansion of quantifier bodies in Sledgehammer translation when needed + transform elim rules later;
2010-08-23, by blanchet
"no_atp" fact that leads to unsound Sledgehammer proofs
2010-08-23, by blanchet
"no_atp" fact that leads to unsound proofs in Sledgehammer
2010-08-23, by blanchet
"no_atp" fact that leads to unsound proofs
2010-08-23, by blanchet
"no_atp" a few facts that often lead to unsound proofs
2010-08-23, by blanchet
play with fudge factor + parse one more Vampire error
2010-08-23, by blanchet
fiddle a bit with the SPASS fudge number
2010-08-23, by blanchet
be more generous towards SPASS's -SOS mode
2010-08-22, by blanchet
don't penalize abstractions in relevance filter + support nameless `foo`-style facts
2010-08-22, by blanchet
merged
2010-08-23, by haftmann
dropped type classes mult_mono and mult_mono1; tuned names of technical rule duplicates
2010-08-23, by haftmann
Document_Model.token_marker: lock jEdit buffer here, which is presumably a critical spot (the model is not necessarily accessed from the Swing thread);
2010-08-23, by wenzelm
sporadic locking of jEdit buffer;
2010-08-23, by wenzelm
main session actor as independent thread, to avoid starvation via regular worker pool;
2010-08-23, by wenzelm
optional daemon flag;
2010-08-23, by wenzelm
tuned;
2010-08-23, by wenzelm
module for simplified thread operations (Scala version);
2010-08-23, by wenzelm
added ML toplevel pretty-printing for tables, using dummy for anything other than Poly/ML 5.3.0 (or later);
2010-08-23, by wenzelm
recognize more "smlnj" variants;
2010-08-23, by wenzelm
merged
2010-08-23, by wenzelm
treat "using X by metis" (more or less) the same as "by (metis X)"
2010-08-22, by blanchet
prefer TPTP "conjecture" tag to "hypothesis" on ATPs where this is possible;
2010-08-22, by blanchet
merged
2010-08-22, by blanchet
more work on finite axiom detection
2010-08-22, by blanchet
revert junk submitted by mistake
2010-08-22, by blanchet
make sure minimizer facts go through "transform_elim_theorems"
2010-08-20, by blanchet
use a smaller simpset in order to not solve refl-instances
2010-08-22, by Christian Urban
allow for pre-simplification of lifted theorems
2010-08-22, by Christian Urban
changed to a more convenient argument order
2010-08-22, by Christian Urban
merged
2010-08-20, by haftmann
split and enriched theory SetsAndFunctions
2010-08-20, by haftmann
more concise characterization of of_nat operation and class semiring_char_0
2010-08-20, by haftmann
inj_comp and inj_fun
2010-08-20, by haftmann
tuned: less formal noise in Named_Target, more coherence in Class
2010-08-20, by haftmann
remove trivial facts
2010-08-20, by blanchet
unbreak "only" option of Sledgehammer
2010-08-20, by blanchet
merged
2010-08-20, by blanchet
improve "x = A | x = B | x = C"-style axiom detection
2010-08-20, by blanchet
temporarily disable "fequal" handling in Metis;
2010-08-20, by blanchet
use "hypothesis" rather than "conjecture" for hypotheses in TPTP format;
2010-08-20, by blanchet
merged
2010-08-20, by blanchet
improve "x = A | x = B | x = C"-style fact discovery
2010-08-20, by blanchet
transform elim theorems before filtering "bool" and "prop" variables out;
2010-08-20, by blanchet
more fiddling with Sledgehammer's "add:" option
2010-08-20, by blanchet
beta eta contract the Sledgehammer conjecture (and also the axioms, although this might not be needed), just like Metis does (implicitly);
2010-08-20, by blanchet
generalize the "too general equality" code to handle facts like "x ~= A ==> x = B"
2010-08-19, by blanchet
encode "fequal" reasoning rules in Metis problem, just as is done for Sledgehammer -- otherwise any proof that relies on "fequal" found by Sledgehammer can't be reconstructed
2010-08-19, by blanchet
fix atomize
2010-08-19, by blanchet
improve atomization
2010-08-19, by blanchet
fix SInE's error handling + run "vampire" locally if either SPASS or E is missing
2010-08-19, by blanchet
added entries
2010-08-19, by blanchet
update docs
2010-08-19, by blanchet
tuning
2010-08-19, by blanchet
parse SNARK proofs
2010-08-19, by blanchet
added remote SInE and remote SNARK
2010-08-19, by blanchet
no spurious trailing "\n" at the end of Sledgehammer's output
2010-08-19, by blanchet
don't get confused by wrong slice
2010-08-18, by blanchet
make sure that "add:" doesn't influence the relevance filter too much
2010-08-18, by blanchet
tuning of relevance filter
2010-08-18, by blanchet
minor cleanup
2010-08-18, by blanchet
bound variables can be just as evil as schematic variables and lead to unsound proofs (e.g. "all_bool_eq")
2010-08-18, by blanchet
update docs
2010-08-18, by blanchet
get rid of "minimize_timeout", now that there's an automatic adaptive timeout mechanism in "minimize"
2010-08-18, by blanchet
added "max_relevant_per_iter" option to Sledgehammer
2010-08-18, by blanchet
thank Andrei instead of Tanya
2010-08-18, by blanchet
fix the relevance filter so that it ignores If, Ex1, Ball, Bex
2010-08-18, by blanchet
tuning
2010-08-18, by blanchet
reactivated -segprot options, just to make double-sure;
2010-08-20, by wenzelm
tuned Markup_Tree.+ : slightly more expensive version to rebuild rest avoids crash of RedBlack.scala:120 (version Scala 2.8.0), e.g. on the following input:
2010-08-22, by wenzelm
tuned;
2010-08-22, by wenzelm
tuned signature;
2010-08-22, by wenzelm
simplified Command.status again, reverting most of e5eed57913d0 (note that more complex information can be represented with full markup reports);
2010-08-22, by wenzelm
proper range for hyperlinks and tooltips, using original markup information;
2010-08-22, by wenzelm
tuned signature;
2010-08-22, by wenzelm
misc tuning and simplification;
2010-08-22, by wenzelm
renamed Markup_Tree.Node to Text.Info;
2010-08-22, by wenzelm
removed obsolete Markup_Tree.flatten/filter;
2010-08-22, by wenzelm
Isabelle_Hyperlinks: select relevant information directly from Markup_Tree, without intermediate RefInfo;
2010-08-22, by wenzelm
Document_View.text_area_extension: select relevant information directly from Markup_Tree, without intermediate TypeInfo;
2010-08-22, by wenzelm
tuned signatures;
2010-08-22, by wenzelm
Command.State: accumulate markup reports uniformly;
2010-08-22, by wenzelm
Markup_Tree.select: misc simplification, proper restriction of parent in subtree;
2010-08-20, by wenzelm
added Text.Range.- convenience;
2010-08-20, by wenzelm
tuned signatures;
2010-08-20, by wenzelm
alternative constructor for Range singularities;
2010-08-20, by wenzelm
concentrate protocol message formats in Isar_Document;
2010-08-20, by wenzelm
Branches.overlapping: proper treatment of stop_range that overlaps with end;
2010-08-20, by wenzelm
further clarification/unification of Position.Range and Text.Range concerning singularities: start offset is always included;
2010-08-20, by wenzelm
parameterized type Markup_Tree.Node;
2010-08-19, by wenzelm
added toString methods;
2010-08-19, by wenzelm
misc tuning and simplification;
2010-08-19, by wenzelm
updated some isatest settings;
2010-08-19, by wenzelm
added generated file;
2010-08-19, by wenzelm
merged
2010-08-19, by wenzelm
tuned quotes
2010-08-19, by haftmann
more antiquotations
2010-08-19, by haftmann
deglobalized named HOL constants
2010-08-19, by haftmann
deglobalized named HOL constants
2010-08-19, by haftmann
corrected some long-overseen misperceptions in recdef
2010-08-19, by haftmann
use HOLogic.boolT and @{typ bool} more pervasively
2010-08-19, by haftmann
tuned
2010-08-19, by haftmann
some more antiquotations
2010-08-19, by haftmann
tuned
2010-08-19, by haftmann
use antiquotations for remaining unqualified constants in HOL
2010-08-19, by haftmann
tuned
2010-08-19, by haftmann
tuned declaration order
2010-08-19, by haftmann
merged
2010-08-18, by haftmann
NEWS
2010-08-18, by haftmann
re-added instantiation of type class random for records
2010-08-18, by haftmann
tuned signature and code
2010-08-18, by haftmann
adjusted to restored naming convention of logical record types
2010-08-18, by haftmann
robustified proof
2010-08-18, by haftmann
adjusted to changed naming convention of logical record types
2010-08-18, by haftmann
removed separate quickcheck_record module
2010-08-18, by haftmann
liberal instantiation of class eq; tuned naming scheme
2010-08-18, by haftmann
more helpful NEWS entry
2010-08-18, by haftmann
dropped SML typedef_codegen: does not fit to code equations for record operations any longer
2010-08-17, by haftmann
preemptive NEWS
2010-08-17, by haftmann
tuned code
2010-08-17, by haftmann
use extension constant as formal constructor of logical record type
2010-08-17, by haftmann
deleted typecopy package
2010-08-17, by haftmann
authentic syntax allows simplification of type names
2010-08-17, by haftmann
dropped make_/dest_ naming convention
2010-08-17, by haftmann
formally integrated typecopy layer into record package
2010-08-17, by haftmann
eliminated typecopy interpretation
2010-08-17, by haftmann
moved spurious auxiliary lemma here
2010-08-18, by haftmann
tuned proof
2010-08-18, by haftmann
qualified constants Let and If
2010-08-18, by haftmann
NEWS
2010-08-18, by haftmann
merged
2010-08-18, by haftmann
deglobalization
2010-08-18, by haftmann
merged
2010-08-18, by blanchet
merged
2010-08-18, by blanchet
rename enum values
2010-08-18, by blanchet
handle bound name conflicts gracefully in FOF translation
2010-08-18, by blanchet
with Kodkodi 1.2.15, Java 1.5 is fine
2010-08-18, by blanchet
gracefully handle the case where the JVM is too old in Nitpick
2010-08-18, by blanchet
improve SPASS clause numbering hack
2010-08-18, by blanchet
deglobalization
2010-08-18, by haftmann
more antiquotations
2010-08-18, by haftmann
added equality instantiation
2010-08-18, by haftmann
use command_def more consciously
2010-08-18, by haftmann
stub for evaluation chapter
2010-08-18, by haftmann
updated generated document
2010-08-18, by haftmann
dropped errorneous underscore
2010-08-18, by haftmann
output whitespace tuning
2010-08-18, by haftmann
use command_def
2010-08-18, by haftmann
use command_def vs. command more consciously
2010-08-18, by haftmann
removed Code_Prolog: modifies global environment setup non-conservatively
2010-08-18, by haftmann
pretty constraint syntax; tuned theory imports
2010-08-18, by haftmann
added quick and dirty section on invariants
2010-08-18, by haftmann
base on HOL-Library
2010-08-18, by haftmann
more antiquotations
2010-08-17, by haftmann
deglobalization
2010-08-17, by haftmann
Tuned.
2010-08-17, by webertj
merged
2010-08-17, by blanchet
repair translation of "c_fequal"
2010-08-17, by blanchet
tweaking
2010-08-17, by blanchet
merged
2010-08-17, by haftmann
enforcing a singleton type inference parameter after type inference and before fixation prevents multiple type variables in import during class declaration
2010-08-17, by haftmann
merged
2010-08-17, by blanchet
invoke Variable.export/import_term on the entire formula, to make sure that schematic variables don't get different indices in different subterms;
2010-08-17, by blanchet
tuning
2010-08-17, by blanchet
more parentheses in TPTP formulas, just in case
2010-08-17, by blanchet
handle E's Skolem constants more gracefully
2010-08-17, by blanchet
improve detection of old Vampire versions
2010-08-17, by blanchet
Markup_Tree.select: crude version of stream-based filtering;
2010-08-19, by wenzelm
Text.Range: improved handling of singularities;
2010-08-19, by wenzelm
tuned XML.content: Stream based iteration is supposed to be declarative *and* efficient;
2010-08-19, by wenzelm
moved Isar_Document to Pure/PIDE;
2010-08-19, by wenzelm
tuned Markup_Tree, using SortedMap more carefully;
2010-08-19, by wenzelm
Output_Position.report_text -- markup with potential "arguments";
2010-08-19, by wenzelm
Command.status: full XML.Tree, i.e. Markup with potential "arguments";
2010-08-19, by wenzelm
more efficient Markup_Tree, based on branches sorted by quasi-order;
2010-08-18, by wenzelm
tuned;
2010-08-18, by wenzelm
refined notion of Text.Range;
2010-08-18, by wenzelm
decode Isabelle symbol positions in one spot;
2010-08-18, by wenzelm
tuned;
2010-08-18, by wenzelm
uniform Markup.empty/Markup.Empty in ML and Scala;
2010-08-18, by wenzelm
digesting strings according to SHA-1 -- Scala version;
2010-08-17, by wenzelm
pro-forma support for further platforms;
2010-08-17, by wenzelm
report command token name instead of kind, which can be retrieved later via Outer_Syntax.keyword_kind;
2010-08-17, by wenzelm
discontinued support for Poly/ML 5.0 and 5.1 versions;
2010-08-17, by wenzelm
updated for prospective Poly/ML 5.4;
2010-08-17, by wenzelm
multi-platform build script for Poly/ML;
2010-08-17, by wenzelm
updated keywords;
2010-08-17, by wenzelm
updated Named_Target.init;
2010-08-17, by wenzelm
made 9043eefe8d71 actually compile;
2010-08-17, by wenzelm
merged
2010-08-17, by wenzelm
merged
2010-08-17, by haftmann
formally document `code abstype` and `code abstract` attributes
2010-08-17, by haftmann
NEWS and CONTRIBUTORS
2010-08-17, by haftmann
nicer code for rev
2010-08-17, by haftmann
reworked section on simple datatype refinement
2010-08-17, by haftmann
tuned whitespace
2010-08-17, by haftmann
merged
2010-08-17, by blanchet
typos in comment
2010-08-16, by blanchet
more debug output
2010-08-16, by blanchet
detect old Vampire and give a nicer error message
2010-08-16, by blanchet
merged
2010-08-17, by nipkow
now works for schematic terms as well, thanks to Alex for the `how-to'
2010-08-17, by nipkow
added section on program refinement
2010-08-17, by haftmann
tuned whitespace
2010-08-17, by haftmann
tune;
2010-08-17, by wenzelm
added functor Linear_Set, based on former adhoc structures in document.ML;
2010-08-17, by wenzelm
HOL-Proofs-Extraction: some workaround to make it work in low-memory situations (e.g. atbroy102 with as little as 1GB heap space);
2010-08-16, by wenzelm
XML.Cache: pipe-lined (thread-safe) version using actor;
2010-08-16, by wenzelm
simplified internal message format: dropped special Symbol.STX header;
2010-08-16, by wenzelm
HTML.spans: explicit flag for preservation of original data (which would be turned into org.w3c.dom user data in XML.document_node);
2010-08-16, by wenzelm
merged
2010-08-16, by wenzelm
merged
2010-08-16, by haftmann
tuned section on predicate compiler
2010-08-16, by haftmann
section "if something goes utterly wrong"
2010-08-16, by haftmann
merged
2010-08-16, by haftmann
merged
2010-08-16, by haftmann
adaptation to new outline
2010-08-16, by haftmann
merged
2010-08-13, by haftmann
corrected handling of `constrains` elements
2010-08-13, by haftmann
removed non-BSD compatible option from cp
2010-08-16, by kleing
Geoff's formatter now needs closed formulas
2010-08-16, by blanchet
Using type real does not require a separate logic now.
2010-08-15, by nipkow
merged
2010-08-15, by nipkow
tuned text about "value" and added note on comments.
2010-08-15, by nipkow
simplified command status: interpret stacked markup on demand;
2010-08-16, by wenzelm
event_bus.scala rather belongs to system plumbing;
2010-08-15, by wenzelm
some derived operations on Text.Range;
2010-08-15, by wenzelm
specific types Text.Offset and Text.Range;
2010-08-15, by wenzelm
moved Text_Edit to Text.Edit;
2010-08-15, by wenzelm
moved History/Snapshot to document.scala;
2010-08-15, by wenzelm
renamed raw_results to raw_protocol;
2010-08-15, by wenzelm
rename "unit" to "atom", to avoid confusion with the unit type;
2010-08-15, by wenzelm
document commands: maintain transition as future (wrt. potentially slow Outer_Syntax.prepare_command), refrain from second Toplevel.put_id;
2010-08-15, by wenzelm
use Synchronized.var and prevent global CRITICAL sections in this hot spot;
2010-08-15, by wenzelm
renamed create_id to new_id;
2010-08-15, by wenzelm
more explicit / functional ML version of document model;
2010-08-15, by wenzelm
renamed class Document to Document.Version etc.;
2010-08-15, by wenzelm
fixed Isabelle/Scala build (cf. f3220ef79d51);
2010-08-15, by wenzelm
Snapshot.state: fall back on Command.empty_state -- looked-up command might be unavailable due to editing divergence;
2010-08-14, by wenzelm
more basic Markup.parse_int/print_int (using signed_string_of_int) (ML);
2010-08-14, by wenzelm
Keyword.status: always suppress position;
2010-08-14, by wenzelm
moved isar_document.ML/scala to Pure/System/ -- side-by-side with isar.ML;
2010-08-14, by wenzelm
merged
2010-08-14, by wenzelm
robustified proof
2010-08-13, by haftmann
lemma execute_bind_case
2010-08-13, by haftmann
unit and bool are instances of heap
2010-08-13, by haftmann
merged
2010-08-13, by haftmann
sketch of new outline
2010-08-13, by haftmann
sketch of new outline
2010-08-13, by haftmann
ditem
2010-08-13, by haftmann
refined abstract
2010-08-13, by haftmann
added stub "If something utterly fails"
2010-08-13, by haftmann
avoid variable name acc (cf. cs. 3142c1e21a0e)
2010-08-13, by haftmann
import swap prevents strange failure of SML code generator for datatypes
2010-08-13, by haftmann
added setup
2010-08-13, by haftmann
merged
2010-08-12, by haftmann
group record-related ML files
2010-08-12, by haftmann
merged
2010-08-12, by haftmann
dropped dead code
2010-08-12, by haftmann
moved Record.thy from session Plain to Main; avoid variable name acc
2010-08-12, by haftmann
group record-related ML files
2010-08-12, by haftmann
Class.declare -> Class.const
2010-08-12, by haftmann
named target is optional; explicit Name_Target.reinit
2010-08-12, by haftmann
named target is optional
2010-08-12, by haftmann
Named_Target.init: empty string represents theory target
2010-08-12, by haftmann
Named_Target.theory_init
2010-08-12, by haftmann
simplified code
2010-08-12, by Christian Urban
tuned
2010-08-12, by haftmann
tuned
2010-08-12, by haftmann
merged
2010-08-11, by haftmann
tuned whitespace
2010-08-11, by haftmann
tuned internal structure
2010-08-11, by haftmann
remove reinit operation alltogether
2010-08-11, by haftmann
avoid arcane Local_Theory.reinit entirely
2010-08-11, by haftmann
more convenient split of class modules: class and class_declaration
2010-08-11, by haftmann
tuned
2010-08-11, by haftmann
stripped signature
2010-08-11, by haftmann
explicit accessed to structure Class_Target
2010-08-11, by haftmann
tuned lowercase
2010-08-11, by haftmann
moved Document.text_edits to Thy_Syntax;
2010-08-14, by wenzelm
tuned;
2010-08-14, by wenzelm
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
less
more
|
(0)
-30000
-10000
-3000
-1000
-480
+480
+1000
+3000
+10000
+30000
tip