Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-224
+224
+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.
tuned signature;
2011-04-07, by wenzelm
merged
2011-04-07, by wenzelm
removing decrement of cardinality in quickcheck -- counting cardinalities starts at 1
2011-04-07, by bulwahn
removing instantiation exhaustive for unit in Quickcheck_Exhaustive
2011-04-07, by bulwahn
correcting bounded_forall construction; tuned
2011-04-07, by bulwahn
dropped unused lemmas; proper Isar proof
2011-04-07, by haftmann
further development of new Skolemizer -- make sure constructed terms have correct types and fixed a few bugs where the goal was out of sync with what we had in mind
2011-04-07, by blanchet
make new Skolemizer more robust
2011-04-07, by blanchet
tuned comment
2011-04-07, by blanchet
discontinued user-defined token translations;
2011-04-07, by wenzelm
simplified printer context: uniform externing and static token translations;
2011-04-07, by wenzelm
clarified Pretty.mark;
2011-04-07, by wenzelm
parallel parsing of big specifications;
2011-04-06, by wenzelm
separate structure Term_Position;
2011-04-06, by wenzelm
type syntax as regular mixfix specification (type_ext for bootstrapping has been obsolete for many years);
2011-04-06, by wenzelm
moved type syntax translations to syn_trans.ML;
2011-04-06, by wenzelm
made SML/NJ happy (cf. 578a51fae383);
2011-04-06, by wenzelm
merged
2011-04-06, by wenzelm
merged
2011-04-06, by bulwahn
changing ensure_sort_datatype call in narrowing quickcheck (missed in 1491b7209e76)
2011-04-06, by bulwahn
prove measurable_into_infprod_algebra and measure_infprod
2011-04-05, by hoelzl
Rename extensional to extensionalD (extensional is also defined in FuncSet)
2011-04-05, by hoelzl
eliminated slightly odd Syntax.rep_syntax;
2011-04-06, by wenzelm
more abstract print translation;
2011-04-06, by wenzelm
more abstract syntax translation;
2011-04-06, by wenzelm
tuned;
2011-04-06, by wenzelm
explicit Syntax.tokenize, Syntax.parse;
2011-04-06, by wenzelm
eliminated odd object-oriented type_context/term_context;
2011-04-06, by wenzelm
simplified standard parse/unparse;
2011-04-06, by wenzelm
discontinued old-style Syntax.constrainC;
2011-04-06, by wenzelm
typed_print_translation: discontinued show_sorts argument;
2011-04-06, by wenzelm
misc tuning and simplification;
2011-04-06, by wenzelm
moved unparse material to syntax_phases.ML;
2011-04-06, by wenzelm
more symbol abbrevs;
2011-04-06, by wenzelm
renamed Standard_Syntax to Syntax_Phases;
2011-04-06, by wenzelm
moved decode/parse operations to standard_syntax.ML;
2011-04-05, by wenzelm
separate module for standard implementation of inner syntax operations;
2011-04-05, by wenzelm
moved Isar/local_syntax.ML to Syntax/local_syntax.ML;
2011-04-05, by wenzelm
merged
2011-04-05, by wenzelm
added "no_atp" to Cantor's paradox
2011-04-05, by blanchet
renamed "const_args" option value to "args"
2011-04-05, by blanchet
temporarily allow useless encoding of helper facts (e.g. fequal_def) instead of throwing exception
2011-04-05, by blanchet
updated instructions
2011-04-05, by blanchet
minor doc edits
2011-04-05, by blanchet
killed unimplemented type encoding "preds"
2011-04-05, by blanchet
remove debugging code
2011-04-05, by blanchet
removing bounded_forall code equation for characters when loading Code_Char
2011-04-05, by bulwahn
deriving bounded_forall instances in quickcheck_exhaustive
2011-04-05, by bulwahn
generalizing ensure_sort_datatype for bounded_forall instances
2011-04-05, by bulwahn
document "type_sys" option
2011-04-04, by blanchet
if "monomorphize" is enabled, mangle the type information in the names by default
2011-04-04, by blanchet
use standard tables with standard argument order;
2011-04-05, by wenzelm
discontinued special treatment of structure Parser -- directly accessible;
2011-04-05, by wenzelm
discontinued special treatment of structure Ast: no pervasive content, no inclusion in structure Syntax;
2011-04-05, by wenzelm
more precise propagation of reports/results through some inner syntax layers;
2011-04-05, by wenzelm
accumulate parsetrees in canonical reverse order;
2011-04-04, by wenzelm
tuned;
2011-04-04, by wenzelm
tuned -- removed redundancy;
2011-04-04, by wenzelm
tuned signatures;
2011-04-04, by wenzelm
streamlined token list operations, assuming that the order of union does not matter;
2011-04-04, by wenzelm
misc tuning and clarification;
2011-04-04, by wenzelm
merged
2011-04-04, by wenzelm
document "nitpick(_params)", "refute(_params)", "try", "sledgehammer(_params)", and "solve_direct"
2011-04-04, by blanchet
refactoring generator definition in quickcheck and removing clone
2011-04-04, by bulwahn
use the proper contexts/simpsets/etc. in the TPTP proof method
2011-04-04, by blanchet
merged
2011-04-04, by blanchet
make sure that Nitpick problem generation for cardinality 50 doesn't cause problems for lower cardinality by specifying the "batch_size" option
2011-04-04, by blanchet
merged
2011-04-04, by paulson
Deletion of all semicolons, because they interfere with Proof General
2011-04-04, by paulson
raised timeouts further, for SML/NJ -- because of variations in machines/compilers, fixed timeouts can merely prevent non-termination, not enforce particular performance characteristics.
2011-04-04, by krauss
tuned proofs
2011-04-03, by haftmann
tuned proof
2011-04-02, by haftmann
direct pretty printing of parsetrees -- prevent diagnostic output from crashing due to undeclared entities;
2011-04-04, by wenzelm
added Position.reports convenience;
2011-04-03, by wenzelm
show more tooltip/sub-expression markup;
2011-04-03, by wenzelm
show tooltip/sub-expression for entity markup;
2011-04-03, by wenzelm
merged
2011-04-01, by wenzelm
remove unnecessary prob_preserving
2011-04-01, by hoelzl
add prob_space_vimage
2011-04-01, by hoelzl
use Unsynchronized.change convenience, which also emphasizes the raw access to these references (which happen to be local here);
2011-04-01, by wenzelm
fixed accidental redefinition
2011-04-01, by krauss
save reflexivity steps in discharging Z3 Skolemization hypotheses
2011-04-01, by boehmes
adding an exhaustive validator for quickcheck's batch validating; moving strip_imp; minimal setup for bounded_forall
2011-04-01, by bulwahn
adding general interface for batch validators in quickcheck
2011-04-01, by bulwahn
remove workaround 8f25605e646c, which is no longer necessary thanks to 173b0f488428
2011-04-01, by blanchet
scheduler for judgement day
2011-04-01, by krauss
re-implemented proof reconstruction for Z3 skolemization: do not explicitly construct definitions for Skolem constants, and let higher-order resolution do most of the work in the end
2011-04-01, by boehmes
make configuration of (SMT) full monomorphization more flexible: turn boolean argument into a configuration option
2011-04-01, by boehmes
merged
2011-04-01, by bulwahn
adding time profiling in quickcheck's batch testing for further diagnosis in IsaCoSy
2011-04-01, by bulwahn
raised timeouts further, for SML/NJ
2011-04-01, by krauss
adapted parsing of session timing (cf. e86b10c68f0b)
2011-04-01, by krauss
merged
2011-03-31, by bulwahn
adapting Quickcheck_Narrowing (overseen in 234ec7011e5d); commenting out some examples temporarily
2011-03-31, by bulwahn
provide a flag controlling whether all provided facts should be instantiated, possibly inventing new types (which does not work well with Sledgehammer)
2011-03-31, by boehmes
start monomorphization process with subgoal, not entire goal, to avoid needless instances (and only print monomorphization messages in debug mode)
2011-03-31, by blanchet
temporary workaround: filter out spurious monomorphic instances
2011-03-31, by blanchet
added monomorphization option to Sledgehammer ATPs -- this looks promising but is still off by default
2011-03-31, by blanchet
added support for "dest:" to "try"
2011-03-31, by blanchet
corrected infix precedence for boolean operators in Haskell
2011-03-31, by haftmann
merged
2011-03-31, by bulwahn
removing dead code in exhaustive_generators
2011-03-30, by bulwahn
removing junk that should not have been committed
2011-03-30, by bulwahn
modernized specifications;
2011-03-30, by wenzelm
accomodate autofix discipline of non-body context;
2011-03-30, by wenzelm
session timing: show pseudo-speedup factor;
2011-03-30, by wenzelm
visualize skolem and hilite (undeclared frees);
2011-03-30, by wenzelm
more informative markup_free;
2011-03-30, by wenzelm
inline lemmas instead of accidental physical addressing -- explicit is better than implicit;
2011-03-30, by wenzelm
tuned white space and indentation;
2011-03-30, by wenzelm
actually check list comprehension examples;
2011-03-30, by wenzelm
products of probability measures are probability measures
2011-03-30, by hoelzl
real multiplication is continuous
2011-03-30, by hoelzl
add lebesgue_real_affine
2011-03-30, by hoelzl
renewing specifications in HOL: replacing types by type_synonym
2011-03-30, by bulwahn
moved TimeLimit.timeLimit closure to limit time of compilation and execution to avoid the strange, occasional occuring message Exception trace for exception - Interrupt -- probably due to race conditions of a fast execution within the TimeLimit.timelimit closure
2011-03-30, by bulwahn
adding a regression test for SML_Quickcheck; putting SML_Quickcheck back in shape
2011-03-30, by bulwahn
NEWS
2011-03-30, by bulwahn
generalizing compilation scheme of quickcheck generators to multiple arguments; changing random and exhaustive tester to use one code invocation for polymorphic instances with multiple cardinalities
2011-03-30, by bulwahn
merged
2011-03-29, by wenzelm
added missing smlnj target
2011-03-29, by krauss
modernized specifications -- less axioms;
2011-03-29, by wenzelm
modernized specifications -- some attempts to avoid wild axiomatizations;
2011-03-29, by wenzelm
tuned proofs;
2011-03-29, by wenzelm
use shared copy of hoare_syntax.ML;
2011-03-29, by wenzelm
Hoare syntax: standard abstraction syntax admits source positions;
2011-03-29, by wenzelm
tuned headers;
2011-03-29, by wenzelm
tuned headers;
2011-03-29, by wenzelm
NEWS
2011-03-29, by hoelzl
rename Probability_Space to Probability_Measure
2011-03-29, by hoelzl
add infinite product measure
2011-03-29, by hoelzl
split Product_Measure into Binary_Product_Measure and Finite_Product_Measure
2011-03-29, by hoelzl
proved caratheodory_empty_continuous
2011-03-29, by hoelzl
list comprehension: strip positions where the translation cannot handle them right now;
2011-03-28, by wenzelm
address serious problem of type inference (introduced in 6f085332c7d3): _type_constraint_ needs type scheme A --> A with proper scope of parameters, otherwise term "(f :: _ => _) :: 'c => 'c" will get type "'a => 'b", for example;
2011-03-28, by wenzelm
raised various timeouts to accommodate sluggish SML/NJ
2011-03-28, by krauss
changing values_timeout from a static option to a dynamic option as required for testing with SML/NJ
2011-03-28, by bulwahn
keep smlnj HOL images around
2011-03-28, by krauss
merged
2011-03-27, by wenzelm
added make target 'smlnj' to refer to what can/should be tested using smlnj -- allows the use of "isabelle makeall smlnj";
2011-03-27, by krauss
avoid *** in normal output, which usually marks errors in logs
2011-03-27, by krauss
added Markup.Name and Markup.Kind convenience;
2011-03-27, by wenzelm
decode_term: some context-sensitive markup;
2011-03-27, by wenzelm
tuned signatures;
2011-03-27, by wenzelm
decode_term: more precise reports;
2011-03-27, by wenzelm
adhoc token style for free/bound;
2011-03-27, by wenzelm
decode_term/disambig: report resolved term variables for the unique (!) result;
2011-03-27, by wenzelm
removed unclear comments stemming from ed24ba6f69aa;
2011-03-27, by wenzelm
present theory content as future, depending on intermediate proof state futures -- potential to reduce memory requirements and improve parallelization;
2011-03-26, by wenzelm
added Future.cond_forks convenience;
2011-03-26, by wenzelm
Isabelle_System.create_tmp_path/with_tmp_file: optional extension;
2011-03-26, by wenzelm
tuned;
2011-03-26, by wenzelm
more direct loose_bvar1;
2011-03-26, by wenzelm
suppress Mercurial backup files;
2011-03-26, by wenzelm
updated generated file;
2011-03-26, by wenzelm
merged
2011-03-26, by wenzelm
SML_makeall: run with -j 3
2011-03-26, by krauss
fixed incomplete rename (1cdf54e845fa)
2011-03-25, by krauss
eliminated hardwired MUTABELLE_OUTPUT_PATH (cf. 6a147393c62a)
2011-03-25, by krauss
merged
2011-03-25, by bulwahn
changing iteration scheme of functions to use minimal number of function updates for exhaustive testing
2011-03-25, by bulwahn
added configurations SML_HOL and SML_makeall (even though the latter is practically infeasible)
2011-03-24, by krauss
mira interface to 'isabelle make' in addition to usedir and makeall;
2011-03-24, by krauss
clarified
2011-03-24, by krauss
parameterize configurations by custom settings
2011-03-24, by krauss
Change coercion for RealDef to use function application (not composition)
2011-03-25, by noschinl
revisiting Code_Prolog (cf. 6fe4abb9437b)
2011-03-25, by bulwahn
fixed postprocessing for term presentation in quickcheck; tuned spacing
2011-03-25, by bulwahn
enable Z3 in the test configuration
2011-03-24, by krauss
add "-?" to "nitrox" tool
2011-03-24, by blanchet
clean up new Skolemizer code -- some old hacks are no longer necessary
2011-03-24, by blanchet
specify proper defaults for Nitpick and Refute on TPTP + tuning
2011-03-24, by blanchet
added "nitrox" tool (Nitpick for first-order TPTP problems) to components
2011-03-24, by blanchet
made one more Metis example use the new Skolemizer
2011-03-24, by blanchet
Metis examples use the new Skolemizer to test it
2011-03-24, by blanchet
new version of Metis 2.3 (29 Dec. 2010)
2011-03-24, by blanchet
remove newly added wrong logic
2011-03-24, by blanchet
more precise failure reporting in Sledgehammer/SMT
2011-03-24, by blanchet
avoid evil "export_without_context", which breaks if there are local "fixes"
2011-03-24, by blanchet
more robust handling of variables in new Skolemizer
2011-03-24, by blanchet
merged
2011-03-24, by haftmann
added subsection on Scala specialities
2011-03-24, by haftmann
added more judgement day provers
2011-03-24, by krauss
allowing special set comprehensions in values command; adding an example for special set comprehension in values
2011-03-24, by bulwahn
merged
2011-03-24, by bulwahn
adding documentation about the eval option in quickcheck
2011-03-23, by bulwahn
adapting Quickcheck_Prolog to latest changes
2011-03-23, by bulwahn
changing Quickcheck_Narrowing's main function to enumerate the depth instead upto the depth
2011-03-23, by bulwahn
adapting mutabelle; exporting more Quickcheck functions
2011-03-23, by bulwahn
making quickcheck's result value more formal; allowing more result information to be returned after timeout; adding output of timing information in quickcheck
2011-03-23, by bulwahn
changing timeout behaviour of quickcheck to proceed after command rather than failing; adding a test case for timeout
2011-03-23, by bulwahn
added Syntax.const_abs_tr' with proper eta_abs and Term.is_dependent;
2011-03-26, by wenzelm
tuned;
2011-03-26, by wenzelm
dependent_tr': formal treatment of bounds after stripping Abs, although it should only happen for malformed terms, since print_translations work top-down;
2011-03-26, by wenzelm
added Term.is_open and Term.is_dependent convenience, to cover common situations of loose bounds;
2011-03-24, by wenzelm
more direct loose_bvar1;
2011-03-24, by wenzelm
indentation;
2011-03-24, by wenzelm
update_name: more uniform treatment of type constraints (NB: type equality is hard to establish in parse trees);
2011-03-24, by wenzelm
added editor mode line;
2011-03-23, by wenzelm
isolate change of Proofterm.proofs in TPTP.thy from rest of session;
2011-03-23, by wenzelm
list Isabelle tools via perl script, which is much faster that bash plumbing, especially on Cygwin;
2011-03-23, by wenzelm
updated contributed components
2011-03-23, by boehmes
Z3 non-commercial usage may explicitly be declined
2011-03-23, by boehmes
export status function to query whether Z3 has been activated for usage within Isabelle
2011-03-23, by boehmes
merge
2011-03-23, by blanchet
avoid illegal variable names, which then yield "Not an identifier" errors in "rename_tac"
2011-03-23, by blanchet
move "TPTP" wrapper and "Sledgehammer as a tactic" to "HOL/ex"
2011-03-23, by blanchet
really be quiet
2011-03-23, by boehmes
replace hardwired MIRABELLE_OUTPUT_PATH by temporary directory derived from ISABELLE_TMP_PREFIX and $$ -- old behaviour can be achieved by manually setting MIRABELLE_OUTPUT_PATH
2011-03-23, by krauss
merged
2011-03-22, by wenzelm
standardized headers
2011-03-22, by hoelzl
generalized Caratheodory from algebra to ring_of_sets
2011-03-22, by hoelzl
add ring_of_sets and subset_class as basis for algebra
2011-03-22, by hoelzl
added first-order TPTP version of Nitpick to Isabelle, so that its sources stay in sync with Isabelle and it is easier to install new versions for SystemOnTPTP and CASC -- the tool is called "isabelle nitrox" but is deliberately omitted from the tool list unless the component is explicitly enabled, to avoid clutter
2011-03-22, by blanchet
added "TPTP" theory with IsabelleP tactic, so that it is maintained alongside with Isabelle and that the CASC version of Isabelle is provided by Isabelle itself instead of being stored on the TPTP servers
2011-03-22, by blanchet
remove lie from documentation
2011-03-22, by blanchet
let SMT errors through -- the main reason for keeping them quiet was that the SMT bridge used to suffer from internal bugs, but these have been fixed for some time now
2011-03-22, by blanchet
make Minimizer honor "verbose" and "debug" options better
2011-03-22, by blanchet
fixed a printing problem for bounded quantifiers and bounded set operators in the case of tuples
2011-03-22, by nipkow
moved some configurations to AFP, and fixed others
2011-03-21, by krauss
more selective strip_positions in case patterns -- reactivate translations based on "case _ of _" in HOL and special patterns in HOLCF;
2011-03-22, by wenzelm
enable inner syntax source positions by default (controlled via configuration option);
2011-03-22, by wenzelm
binder_tr: more informative exception;
2011-03-22, by wenzelm
Hoare syntax: strip positions where they crash translation functions;
2011-03-22, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-224
+224
+1000
+3000
+10000
+30000
tip