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.
avoid confusing selector output
2011-11-13, by blanchet
remove unsound line in Nitpick's "rat" setup
2011-11-13, by blanchet
tuned proofs;
2011-11-12, by wenzelm
merged
2011-11-12, by wenzelm
removed some old-style semicolons
2011-11-12, by huffman
index markup elements for more efficient cumulate/select operations;
2011-11-12, by wenzelm
tuned;
2011-11-12, by wenzelm
tuned markup -- prefer user-perspective;
2011-11-12, by wenzelm
tuned specifications and proofs;
2011-11-12, by wenzelm
more precise type;
2011-11-12, by wenzelm
refined Markup_Tree implementation: stacked markup within each entry;
2011-11-12, by wenzelm
tuned signature;
2011-11-12, by wenzelm
tuned signature;
2011-11-12, by wenzelm
merged
2011-11-11, by wenzelm
merged
2011-11-11, by huffman
abel_cancel.ML: avoid canceling zeros, which would cause the simproc to return a trivial rewrite;
2011-11-11, by huffman
use simproc_setup for the remaining nat_numeral simprocs
2011-11-11, by huffman
use simproc_setup for more nat_numeral simprocs; add simproc tests
2011-11-11, by huffman
using more conventional names for monad plus operations
2011-11-11, by bulwahn
more tooltip content;
2011-11-11, by wenzelm
added markup_cumulate operator;
2011-11-11, by wenzelm
depth-first proof forking for improved locality (wrt. cancellation and overall memory usage);
2011-11-11, by wenzelm
tuned;
2011-11-11, by wenzelm
more abstract Markup_Tree;
2011-11-11, by wenzelm
prefer statically typed Text.Markup;
2011-11-11, by wenzelm
discontinued entity text color, notably historic red for classes;
2011-11-11, by wenzelm
more scalable Proof_Context.prepare_sorts;
2011-11-11, by wenzelm
increasing values_timeout to avoid failures of isatest with HOL-IMP
2011-11-11, by bulwahn
renaming example invocations: tester predicate_compile is renamed to smart_exhaustive
2011-11-11, by bulwahn
adding CPS compilation to predicate compiler;
2011-11-11, by bulwahn
adding option allow_function_inversion to quickcheck options
2011-11-11, by bulwahn
more efficient prepare_sorts -- bypass encoded positions;
2011-11-10, by wenzelm
suppress irrelevant positions;
2011-11-10, by wenzelm
more generous margin;
2011-11-10, by wenzelm
pass term positions into check phase, where resulting types are reported accordingly, and eventually shown as tooltips;
2011-11-10, by wenzelm
tuned signature;
2011-11-10, by wenzelm
discontinued unused Thm.compress (again);
2011-11-10, by wenzelm
renewed prolog-quickcheck
2011-11-10, by bulwahn
adding some test cases for preprocessing and narrowing
2011-11-10, by bulwahn
adding a minimalistic preprocessing rewriting common boolean operators; tuned
2011-11-10, by bulwahn
merged
2011-11-10, by huffman
merged
2011-11-09, by huffman
tune post-processing of simproc-generated rules so they won't produce Numeral0 or Numeral1
2011-11-09, by huffman
use simproc_setup for some nat_numeral simprocs; add simproc tests
2011-11-09, by huffman
add ring_char_0 class constraints to several simprocs (internal proofs of #n ~= 0 fail for type
2011-11-09, by huffman
simultaneous check;
2011-11-10, by wenzelm
avoid separate typ_check phases, integrate into main term_check 0 instead (cf. its Syntax.check_typs in Type_Infer_Context.prepare);
2011-11-09, by wenzelm
clarified singleton_fixate: intersection with supersort is identity, only replace actual type inference parameters;
2011-11-09, by wenzelm
misc tuning and simplification;
2011-11-09, by wenzelm
misc tuning;
2011-11-09, by wenzelm
tuned signature;
2011-11-09, by wenzelm
quickcheck invocations in mutabelle must not catch codegenerator errors internally
2011-11-09, by bulwahn
sort assignment before simultaneous term_check, not isolated parse_term;
2011-11-09, by wenzelm
tuned;
2011-11-09, by wenzelm
avoid inconsistent sort constraints;
2011-11-09, by wenzelm
localized Record.decode_type: use standard Proof_Context.get_sort;
2011-11-09, by wenzelm
tuned signature -- emphasize internal role of these operations;
2011-11-09, by wenzelm
proper configuration option;
2011-11-09, by wenzelm
tuned layout;
2011-11-09, by wenzelm
more precise messages with the tester's name in quickcheck; tuned
2011-11-09, by bulwahn
quickcheck fails with code generator errors only if one tester is invoked
2011-11-09, by bulwahn
removing extra arguments
2011-11-09, by bulwahn
removing deactivated timeout handling; catching compilation errors and only outputing an urgent message to enable parallel sucessful quickcheck compilations and runs to present their result
2011-11-09, by bulwahn
tuned
2011-11-09, by bulwahn
more fragments to export, removed the one from Com
2011-11-09, by kleing
updated functor Named_Thms;
2011-11-08, by wenzelm
disabled Thm.compress (again) -- costs for building tables tend to be higher than potential benefit;
2011-11-08, by wenzelm
entity markup for bound variables;
2011-11-08, by wenzelm
merged
2011-11-08, by wenzelm
made SML/NJ happy
2011-11-08, by boehmes
adding some documentation about the values command to the isar reference
2011-11-08, by bulwahn
adding a minimal documentation about the code_pred command to the isar reference
2011-11-08, by bulwahn
more specific treatment of defines/assumes -- avoid normalizing defs by themselves (NB: locale specifications and Local_Theory.define may lead to arbitrary mixture);
2011-11-08, by wenzelm
clarified Local_Defs.export: avoid costly still_fixed test, return all defs;
2011-11-08, by wenzelm
eliminated obsolete tuning (NB: Thm.eta_conversion/Envir.eta_contract based on Same.operation);
2011-11-08, by wenzelm
tuned;
2011-11-08, by wenzelm
tuned;
2011-11-08, by wenzelm
tweaked comment
2011-11-08, by blanchet
made SML/NJ happy
2011-11-08, by blanchet
merged;
2011-11-08, by wenzelm
added FIXME comment
2011-11-07, by blanchet
avoid infinite recursion in peephole optimizer function -- this had a debilitating effect on rationals and reals
2011-11-07, by blanchet
revived Refute in Mutabelle
2011-11-07, by blanchet
tuned;
2011-11-07, by wenzelm
more scalable zero_var_indexes, depending on canonical order within table;
2011-11-07, by wenzelm
more benchmarks;
2011-11-07, by wenzelm
try different alternatives in discharging extra assumptions when schematic theorems obtained from lambda-lifting can be instantiated in different ways
2011-11-07, by boehmes
replace higher-order matching against schematic theorem with dedicated reconstruction method
2011-11-07, by boehmes
merged
2011-11-07, by wenzelm
tuned signature -- avoid spurious Thm.mixed_attribute;
2011-11-07, by wenzelm
discontinued numbered structure indexes (legacy feature);
2011-11-07, by wenzelm
tuned proofs;
2011-11-07, by wenzelm
return outcome code, so that it can be picked up by Mutabelle
2011-11-07, by blanchet
align columns in output and keep error log around
2011-11-07, by blanchet
offline build of java_ext_dirs.jar, to avoid runtime dependency on javac/jar executables;
2011-11-07, by wenzelm
clarified attribute "mono_set": pure declaration, proper export in ML;
2011-11-07, by wenzelm
misc tuning;
2011-11-07, by wenzelm
made SML/NJ happy;
2011-11-07, by wenzelm
more millisecond cleanup
2011-11-06, by blanchet
updated documentation
2011-11-06, by blanchet
try "smt" as a fallback for ATPs if "metis" fails/times out
2011-11-06, by blanchet
more detailed preplay output
2011-11-06, by blanchet
tuning
2011-11-06, by blanchet
tuning
2011-11-06, by blanchet
more explicit representation of rule_attribute vs. declaration_attribute vs. mixed_attribute;
2011-11-06, by wenzelm
tuned;
2011-11-06, by wenzelm
merged
2011-11-06, by wenzelm
cascading timeouts in minimizer, part 2
2011-11-06, by blanchet
tuning
2011-11-06, by blanchet
use "Time.time" rather than milliseconds internally
2011-11-06, by blanchet
tune: no need for option
2011-11-06, by blanchet
cascading timeouts in minimizer
2011-11-06, by blanchet
shortcut binary minimization algorithm
2011-11-06, by blanchet
speed up binary minimizer in practice by preferring the first half of the used facts (which are likelier to be relevant) to the second half
2011-11-06, by blanchet
renamed experimental systems
2011-11-06, by blanchet
repaired quantification over type variables for non-TFF1/THF encodings
2011-11-06, by blanchet
misc tuning and modernization;
2011-11-06, by wenzelm
misc tuning and modernization;
2011-11-06, by wenzelm
tuned;
2011-11-06, by wenzelm
some statespace benchmarks;
2011-11-06, by wenzelm
write changed .prv files only, to avoid writing into src file-space by default;
2011-11-06, by wenzelm
tuned document;
2011-11-06, by wenzelm
more precise dependencies;
2011-11-06, by wenzelm
inlined antiquotations;
2011-11-06, by wenzelm
misc tuning and modernization;
2011-11-06, by wenzelm
optional timing, to avoid redundant allocation of mutable cells;
2011-11-06, by wenzelm
tuned;
2011-11-05, by wenzelm
misc tuning;
2011-11-05, by wenzelm
merged
2011-11-05, by wenzelm
more use of global operations (see 98ec8b51af9c)
2011-11-05, by Christian Urban
more uniform instT_subst vs. inst_subst: compare variable names only;
2011-11-05, by wenzelm
tuned cterm_instantiate: avoid somewhat expensive Term.map_types and cterm_of;
2011-11-05, by wenzelm
misc tuning and modernization;
2011-11-05, by wenzelm
some performance tuning via Term_Subst/Same.operation;
2011-11-05, by wenzelm
pruned signature;
2011-11-05, by wenzelm
added Logic.varify_types_global/unvarify_types_global, which avoids somewhat expensive Term.map_types;
2011-11-05, by wenzelm
more conventional syntax const;
2011-11-05, by wenzelm
proper syntactic category for abstraction syntax, to avoid low-level exception for malformed "\<integral> x y. f \<partial>M", for example;
2011-11-04, by wenzelm
merged
2011-11-04, by wenzelm
prefer global Quotient_Info lookup to accomodate Quotient_Term, which is not quite localized yet (cf. 9fd6fce8a230);
2011-11-04, by wenzelm
document new experimental provers
2011-11-04, by blanchet
added remote iProver(-Eq) for experimentation
2011-11-04, by blanchet
merged
2011-11-04, by wenzelm
ex/Tree23.thy: automate proof of gfull_add
2011-11-04, by huffman
ex/Tree23.thy: simplify proof of bal_del0
2011-11-04, by huffman
ex/Tree23.thy: simplify proof of bal_add0
2011-11-04, by huffman
ex/Tree23.thy: simpler definition of ordered-ness predicate
2011-11-04, by huffman
ex/Tree23.thy: prove that deletion preserves balance
2011-11-03, by huffman
more liberal Parse.fixes, to avoid overlap of mixfix with is-pattern (notably in 'obtain' syntax);
2011-11-04, by wenzelm
more general Proof_Context.bind_propp, which allows outer parameters;
2011-11-03, by wenzelm
tuned whitespace;
2011-11-03, by wenzelm
tuned signature;
2011-11-03, by wenzelm
tuned signature -- canonical argument order;
2011-11-03, by wenzelm
tuned -- Variable.declare_term is already part of Variable.auto_fixes;
2011-11-03, by wenzelm
ex/Tree23.thy: prove that insertion preserves tree balance and order
2011-11-03, by huffman
more IMP fragments
2011-11-03, by kleing
string -> vname
2011-11-03, by kleing
JMPF(LESS|GE) -> JMP(LESS|GE) because jumps are int now.
2011-11-03, by kleing
more IMP text fragments
2011-11-03, by kleing
moved latex generation for HOL-IMP out of distribution
2011-11-03, by kleing
renaming Quotient_Set and List_Quotient_Set to Quotient_Cset and List_Quotient_Cset to avoid name clash with existing Quotient_Set (again, cf. 66823a0066db)
2011-11-01, by bulwahn
merged
2011-10-31, by bulwahn
more robust, declarative and unsurprising computation of types in the quotient type definition
2011-10-31, by bulwahn
improve handling of bound type variables (esp. for TFF1)
2011-10-31, by blanchet
improved TFF1 output
2011-10-31, by blanchet
clarified signature
2011-10-31, by bulwahn
tuned
2011-10-31, by bulwahn
tuned
2011-10-31, by bulwahn
even more uniform Local_Theory.declaration for locales (cf. 57def0b39696, aa35859c8741);
2011-10-30, by wenzelm
removed obsolete argument (cf. aa35859c8741);
2011-10-30, by wenzelm
removed ad-hoc simp rules sin_cos_eq[symmetric], minus_sin_cos_eq[symmetric], cos_sin_eq[symmetric]
2011-10-30, by huffman
extend cancellation simproc patterns to cover terms like '- (2 * pi) < pi'
2011-10-30, by huffman
merged
2011-10-30, by huffman
remove unused function
2011-10-29, by huffman
also export DFG formats
2011-10-29, by blanchet
always use DFG format to talk to SPASS -- since that's what we'll need to use anyway to benefit from sorts and other extensions
2011-10-29, by blanchet
added DFG unsorted support (like in the old days)
2011-10-29, by blanchet
gracefully do nothing if the SPASS input file is already in DFG format
2011-10-29, by blanchet
added sorted DFG output for coming version of SPASS
2011-10-29, by blanchet
specify proof output level 1 (i.e. no detailed, potentially huge E proofs) to LEO-II; requires version 1.2.9
2011-10-29, by blanchet
check "sound" flag before doing something unsound...
2011-10-29, by blanchet
uniform treatment of syntax declaration wrt. aux. context (NB: notation avoids duplicate mixfix internally);
2011-10-29, by wenzelm
tuned;
2011-10-29, by wenzelm
more accurate class constraints on cancellation simproc patterns
2011-10-28, by huffman
tuned;
2011-10-29, by wenzelm
tuned Named_Thms: proper binding;
2011-10-28, by wenzelm
refined Local_Theory.declaration {syntax = false, pervasive} semantics: update is applied to auxiliary context as well;
2011-10-28, by wenzelm
more robust data storage (NB: the morphism can change the shape of qconst, and in the auxiliary context it is not even a constant yet);
2011-10-28, by wenzelm
uniform Local_Theory.declaration with explicit params;
2011-10-28, by wenzelm
tuned signature -- refined terminology;
2011-10-28, by wenzelm
slightly more explicit/syntactic modelling of morphisms;
2011-10-28, by wenzelm
correct import path
2011-10-28, by hoelzl
allow to build Probability and MV-Analysis with one ROOT.ML
2011-10-28, by hoelzl
removing dead code
2011-10-28, by bulwahn
ex/Simproc_Tests.thy: remove duplicate simprocs
2011-10-28, by huffman
use simproc_setup for cancellation simprocs, to get proper name bindings
2011-10-28, by huffman
tuned;
2011-10-27, by wenzelm
eliminated aliases of standard functions;
2011-10-27, by wenzelm
more standard attribute setup;
2011-10-27, by wenzelm
localized quotient data;
2011-10-27, by wenzelm
simplified/standardized signatures;
2011-10-27, by wenzelm
tuned signature;
2011-10-27, by wenzelm
uses IMP and hence requires its tex setup
2011-10-27, by nipkow
merged
2011-10-27, by nipkow
tuned text
2011-10-27, by nipkow
respecting isabelle's programming style in the quotient package by simplifying qconsts_lookup function for data access; removing odd NotFound exception
2011-10-27, by bulwahn
respecting isabelle's programming style in the quotient package by simplifying map_lookup function for data access
2011-10-27, by bulwahn
respecting isabelle's programming style in the quotient package by simplifying quotdata_lookup function for data access
2011-10-27, by bulwahn
merged
2011-10-27, by huffman
fix bug in cancel_factor simprocs so they will work on goals like 'x * y < x * z' where the common term is already on the left
2011-10-27, by huffman
more robust ML pretty printing (cf. b6c527c64789);
2011-10-26, by wenzelm
tuned;
2011-10-26, by wenzelm
renaming Cset and List_Cset in Quotient_Examples to Quotient_Set and List_Quotient_Set to avoid a name clash of theory names with the ones in HOL-Library
2011-10-25, by bulwahn
tuned text
2011-10-25, by nipkow
tuned names to avoid shadowing
2011-10-25, by nipkow
merge Gcd/GCD and Lcm/LCM
2011-10-25, by huffman
clarify types of terms: use proper set type
2011-10-25, by boehmes
instance bool :: linorder
2011-10-24, by huffman
removing poor man's dictionary construction which were only for the ancient code generator with no support of type classes
2011-10-24, by bulwahn
fixed typo
2011-10-24, by bulwahn
latex output not needed because errors manifest themselves earlier
2011-10-24, by nipkow
some text on inner-syntax;
2011-10-23, by wenzelm
renamed in ASM
2011-10-23, by nipkow
tuned order of eqns
2011-10-23, by nipkow
tuned
2011-10-23, by nipkow
script for exporting filtered IMP files as tar.gz
2011-10-23, by kleing
removed Norbert's email from isatest (bounces)
2011-10-23, by kleing
class Lexicon as abstract datatype;
2011-10-22, by wenzelm
more private stuff;
2011-10-22, by wenzelm
class Text.Edit as abstract datatype;
2011-10-22, by wenzelm
class Time as abstract datatype;
2011-10-22, by wenzelm
class Volatile as abstract datatype;
2011-10-22, by wenzelm
merged
2011-10-22, by nipkow
added isaverbatimwrite that allows to cut out snippets of thy files in their latex form and dump them in a file
2011-10-22, by nipkow
experimental support for Scala 2.9.1.final;
2011-10-22, by wenzelm
class Path as abstract datatype;
2011-10-22, by wenzelm
class Counter as abstract datatype;
2011-10-22, by wenzelm
discontinued redundant ASCII syntax;
2011-10-22, by wenzelm
modernized specifications;
2011-10-22, by wenzelm
proper normal form for Perspective.ranges (overlapping ranges could be joined in wrong order, crashing multiple editor views);
2011-10-21, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-240
+240
+1000
+3000
+10000
+30000
tip