Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-960
+960
+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.
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
merged
2011-10-21, by nipkow
tuned
2011-10-21, by nipkow
merged
2011-10-21, by wenzelm
replacing metis proofs with facts xt1 by new proof with more readable names
2011-10-21, by bulwahn
more robust parsing of TSTP sources -- Vampire has nonstandard "introduced()" tags and Waldmeister(OnTPTP) has weird "theory(...)" dependencies
2011-10-21, by blanchet
disable Vampire's BDD optimization, which sometimes yields so huge proofs that this causes problems for reconstruction
2011-10-21, by blanchet
NEWS
2011-10-21, by bulwahn
updating documentation: code_inline -> code_unfold; added documentation about attribute code_unfold_post
2011-10-21, by bulwahn
replacing code_inline by code_unfold, removing obsolete code_unfold, code_inline del now that the ancient code generator is removed
2011-10-21, by bulwahn
removing redundant attribute code_inline in the code generator
2011-10-21, by bulwahn
tuned;
2011-10-21, by wenzelm
tuned;
2011-10-21, by wenzelm
improving mutabelle script again after missing some changes in f4896c792316
2011-10-21, by bulwahn
correcting code_prolog
2011-10-21, by bulwahn
merged
2011-10-21, by huffman
add HOL/ex/Simproc_Tests.thy: testing for Tools/numeral_simprocs.ML
2011-10-21, by huffman
merged
2011-10-21, by nipkow
tuned
2011-10-21, by nipkow
mark "xt..." rules as "no_atp", since they are easy consequences of other better named properties
2011-10-20, by blanchet
merged
2011-10-20, by huffman
removed mult_Bit1 from int_arith_rules (cf. 882403378a41 and 3078fd2eec7b, where mult_num1 erroneously replaced mult_1)
2011-10-20, by huffman
removed [trans] concept from basic material
2011-10-20, by kleing
merged
2011-10-20, by nipkow
tuned
2011-10-20, by nipkow
merged
2011-10-20, by bulwahn
modernizing predicate_compile_quickcheck
2011-10-20, by bulwahn
adding depth as an quickcheck configuration
2011-10-20, by bulwahn
renamed name -> vname
2011-10-20, by nipkow
removed some remaining artefacts of ancient SML code generator
2011-10-19, by haftmann
NEWS
2011-10-19, by haftmann
cleaner LEO-II extensionality step detection
2011-10-19, by blanchet
marginally cleaner proof parsing, that doesn't stumble upon LEO-II's E-step proofs
2011-10-19, by blanchet
one more LEO-II failure
2011-10-19, by blanchet
merged
2011-10-19, by wenzelm
merged
2011-10-19, by huffman
hide typedef-generated constants Product_Type.prod and Sum_Type.sum
2011-10-18, by huffman
more uniform SZS status handling
2011-10-19, by blanchet
avoid generating too meta theorems -- this sometimes leads to type errors, e.g. when "pp" is applied to a "prop" instead of a "bool"
2011-10-19, by blanchet
merged
2011-10-19, by nipkow
renamed B to Bc
2011-10-19, by nipkow
tuned comment;
2011-10-19, by wenzelm
proper source positions for @{lemma};
2011-10-19, by wenzelm
more robust toplevel_error reporting (NB: Context.proof_of on a stale theory crashes ungracefully);
2011-10-19, by wenzelm
inlined @{thms} (ML compile-time) allows to get rid of legacy zadd_ac as well (cf. 49e305100097);
2011-10-19, by wenzelm
tuned legacy signature;
2011-10-19, by wenzelm
further cleanup of stats (cf. 97e81a8aa277);
2011-10-19, by wenzelm
updated keywords;
2011-10-19, by wenzelm
really document just one code generator;
2011-10-19, by wenzelm
NEWS
2011-10-19, by bulwahn
removing old code generator
2011-10-19, by bulwahn
removing declaration of code_unfold to address the old code generator
2011-10-19, by bulwahn
removing dependency of the generic code generator to old code generator functions thyname_of_type and thyname_of_const
2011-10-19, by bulwahn
removing documentation about the old code generator
2011-10-19, by bulwahn
removing old code generator setup for executable sets
2011-10-19, by bulwahn
removing old code generator setup for efficient natural numbers; cleaned typo
2011-10-19, by bulwahn
removing old code generator setup for real numbers; tuned
2011-10-19, by bulwahn
removing old code generator setup for rational numbers; tuned
2011-10-19, by bulwahn
removing old code generator setup for strings
2011-10-19, by bulwahn
removing old code generator setup for lists
2011-10-19, by bulwahn
removing old code generator setup for integers
2011-10-19, by bulwahn
removing old code generator for inductive predicates
2011-10-19, by bulwahn
removing quickcheck tester SML-inductive based on the old code generator
2011-10-19, by bulwahn
removing old code generator setup for inductive sets in the inductive set package
2011-10-19, by bulwahn
removing old code generator setup of inductive predicates
2011-10-19, by bulwahn
removing old code generator setup for product types
2011-10-19, by bulwahn
removing old code generator setup for function types
2011-10-19, by bulwahn
removing old code generator setup for datatypes
2011-10-19, by bulwahn
removing old code generator for recursive functions
2011-10-19, by bulwahn
removing old code generator setup in the HOL theory
2011-10-19, by bulwahn
removing invocations of the evaluation method based on the old code generator
2011-10-19, by bulwahn
removing invocations of the old code generator
2011-10-19, by bulwahn
freeze conjecture schematics before applying lambda-translation, which sometimes calls "close_form" and ruins it for freezing
2011-10-18, by blanchet
gracefully handle quantifiers of the form "All $ t" where "t" is not a lambda-abstraction in higher-order translations
2011-10-18, by blanchet
tuned
2011-10-18, by bulwahn
adding testing of quickcheck narrowing with finite types to mutabelle script; modified is_executable in mutabelle_extra
2011-10-18, by bulwahn
mira: collect size of heap images
2011-10-18, by krauss
updated doc related to Satallax
2011-10-17, by blanchet
parse Satallax unsat cores
2011-10-17, by blanchet
merged
2011-10-17, by wenzelm
(old) NEWS
2011-10-17, by noschinl
moving some common functions from quickcheck to the more HOL-specific quickcheck_common; renamed inductive_SML's configurations to more canonical names; adds automatically left and right hand sides of equations as evaluation terms
2011-10-17, by bulwahn
always use sockets on Windows/Cygwin;
2011-10-17, by wenzelm
mira configuration: use official polyml 5.4.1 on lxbroy10
2011-10-16, by krauss
added Term.dummy_pattern conveniences;
2011-10-16, by wenzelm
slightly more standard-conformant XML parsing (see also 94033767ef9b);
2011-10-16, by wenzelm
tuned proof
2011-10-16, by haftmann
tuned type annnotation
2011-10-16, by haftmann
hide not_member as also member
2011-10-16, by haftmann
misc tuning and modernization;
2011-10-15, by wenzelm
updated to Scala 2.8.2.final;
2011-10-15, by wenzelm
prefer recent polyml-5.4.1, but retain potentially fragile polyml-5.2.1 as experimental test;
2011-10-15, by wenzelm
updated to polyml-5.4.1;
2011-10-15, by wenzelm
updated to polyml-5.4.1;
2011-10-15, by wenzelm
merged
2011-10-15, by haftmann
monadic bind
2011-10-14, by haftmann
moved sublists to More_List.thy
2011-10-14, by haftmann
NEWS
2011-10-14, by haftmann
more complete stats, including small sessions which provide some clues on main HOL baseline performance;
2011-10-14, by wenzelm
avoid very specific code equation for card; corrected spelling
2011-10-13, by haftmann
bouned transitive closure
2011-10-13, by haftmann
moved acyclic predicate up in hierarchy
2011-10-13, by haftmann
tuned
2011-10-13, by haftmann
modernized definitions
2011-10-13, by haftmann
static dummy_task (again) to avoid a few extra allocations;
2011-10-13, by wenzelm
tuned markup
2011-10-13, by noschinl
discontinued obsolete 'types' command;
2011-10-13, by wenzelm
modernized structure Induct_Tacs;
2011-10-12, by wenzelm
tuned signature;
2011-10-12, by wenzelm
misc tuning and clarification;
2011-10-12, by wenzelm
tuned ML style;
2011-10-12, by wenzelm
tuned proofs -- eliminated vacuous "induct arbitrary: ..." situations;
2011-10-12, by wenzelm
discontinued obsolete alias structure ProofContext;
2011-10-12, by wenzelm
separated monotonicity reasoning and defined narrowing with while_option
2011-10-12, by nipkow
include no-smlnj targets into library (cf. e54a985daa61);
2011-10-10, by wenzelm
increasing values_timeout to avoid SML_makeall failures on our current tests
2011-10-10, by bulwahn
merged
2011-10-10, by wenzelm
removed obsolete RC tags;
2011-10-10, by wenzelm
Int.thy: discontinued some legacy theorems
2011-10-09, by huffman
Set.thy: remove redundant [simp] declarations
2011-10-09, by huffman
removing code equation for card on finite types when loading the Executable_Set theory; should resolve a code generation issue with CoreC++
2011-10-03, by bulwahn
tune text for document generation
2011-10-03, by bulwahn
adding examples with relations to Quickcheck_Examples to show that quickcheck can actually handle operators on relations as well
2011-10-03, by bulwahn
adding code equations for cardinality and (reflexive) transitive closure on finite types
2011-10-03, by bulwahn
adding lemma about rel_pow in Transitive_Closure for executable equation of the (refl) transitive closure
2011-10-03, by bulwahn
adding lemma to List library for executable equation of the (refl) transitive closure
2011-10-03, by bulwahn
fixed typos in IMP
2011-09-29, by Jean Pichon
added nice interval syntax
2011-09-28, by nipkow
Added dependecies
2011-09-28, by nipkow
Added Hoare-like Abstract Interpretation
2011-09-28, by nipkow
moved IMP/AbsInt stuff into subdirectory Abs_Int_Den
2011-09-28, by nipkow
back to post-release mode;
2011-09-26, by wenzelm
Added tag Isabelle2011-1 for changeset 76fef3e57004
2011-10-09, by wenzelm
tuned;
Isabelle2011-1
2011-10-09, by wenzelm
updated ISABELLE_HOME_USER;
2011-10-09, by wenzelm
more explicit check of Java executable -- relevant for Linux x86/x86_64 mismatch and absence on Mac OS Lion;
2011-10-04, by wenzelm
Added tag Isabelle2011-1-RC2 for changeset a45121ffcfcb
2011-10-03, by wenzelm
some amendments due to Jean Pichon;
2011-10-03, by wenzelm
correct coercion generation in case of unknown map functions
2011-09-29, by traytel
proper platform_file_url for Windows UNC paths (server shares);
2011-09-28, by wenzelm
proper platform_file_url;
2011-09-27, by wenzelm
observe base URL of rendered document;
2011-09-27, by wenzelm
more README;
2011-09-27, by wenzelm
tuned README.html;
2011-09-27, by wenzelm
tuned;
2011-09-27, by wenzelm
retain output, which is required for non-existent JRE, for example (cf. b455e4f42c04);
2011-09-27, by wenzelm
tuned message, which is displayed after termination of Isabelle.app on Mac OS;
2011-09-27, by wenzelm
keep top-level "Isabelle" executable -- now an alias for "isabelle jedit";
2011-09-26, by wenzelm
tuned;
2011-09-26, by wenzelm
ensure Isabelle env;
2011-09-26, by wenzelm
Added tag Isabelle2011-1-RC1 for changeset 24ad77c3a147
2011-09-26, by wenzelm
tuned;
2011-09-26, by wenzelm
misc tuning for release;
2011-09-26, by wenzelm
reverted 09cdc4209d25 for formal reasons: it did not say what was "broken" nor "fixed", but broke IsaMakefile dependencies;
2011-09-26, by wenzelm
makedist for release;
2011-09-26, by wenzelm
put MiniSat back first -- Torlak's eval seemed to suggest that Crypto and Lingeling were better, but Crypto is slower on "Nitpick_Examples" and Crypto crashes
2011-09-26, by blanchet
require Java 1.6 in the Nitpick documentation -- technically 1.5 will also work with Kodkodi 1.2.16, but it won't work with Kodkodi 1.5.0
2011-09-26, by blanchet
put CryptoMiniSat first and remove warning about unsoundness now that it has been fixed in Kodkod
2011-09-26, by blanchet
adding an example with inductive predicates to quickcheck narrowing examples
2011-09-26, by bulwahn
importing the Generated_Code module qualified to reduce the probability of name clashes between the static code and the generated code in the narrowing-based Quickcheck
2011-09-26, by bulwahn
clarify platforms
2011-09-25, by blanchet
killed JNI version of zChaff, since Kodkod 1.5 does not support it anymore
2011-09-25, by blanchet
updated Nitpick SAT Solver doc
2011-09-25, by blanchet
update list of SAT solvers reflecting Kodkod 1.5
2011-09-25, by blanchet
tuned signature;
2011-09-25, by wenzelm
more uniform defaults;
2011-09-25, by wenzelm
Quotient_Set.thy is part of library
2011-09-25, by haftmann
fixed typo
2011-09-25, by nipkow
standardize drive letters -- important for proper document node identification;
2011-09-24, by wenzelm
more user aliases;
2011-09-24, by wenzelm
fixed IsaMakefile action for HOL-TPTP.
2011-09-24, by sultana
prefer socket comminication on Cygwin, which is more stable here than fifos;
2011-09-23, by wenzelm
tuned proof;
2011-09-23, by wenzelm
made SML/NJ happy;
2011-09-23, by wenzelm
discontinued stream-based Socket_IO, which causes too many problems with Poly/ML and SML/NJ (reverting major parts of 5c0b0d67f9b1);
2011-09-23, by wenzelm
updated header;
2011-09-23, by wenzelm
merged;
2011-09-23, by wenzelm
reintroduced E-SInE now that it's unexpectedly working again (thanks to Geoff)
2011-09-23, by blanchet
first step towards extending Minipick with more translations
2011-09-23, by blanchet
Include keywords print_coercions and print_coercion_maps
2011-09-23, by berghofe
local coercion insertion algorithm to support complex coercions
2011-08-17, by traytel
printing and deleting of coercions
2011-08-17, by traytel
raw unbuffered socket IO, which bypasses the fragile BinIO layer in Poly/ML 5.4.x;
2011-09-23, by wenzelm
default print mode for Isabelle/Scala, not just Isabelle/jEdit;
2011-09-23, by wenzelm
augment existing print mode;
2011-09-23, by wenzelm
explicit option for socket vs. fifo communication;
2011-09-23, by wenzelm
tuned proof;
2011-09-23, by wenzelm
synchronized section names with manual
2011-09-23, by blanchet
merged;
2011-09-23, by wenzelm
discontinued legacy theorem names from RealDef.thy
2011-09-22, by huffman
merged
2011-09-22, by huffman
discontinued HOLCF legacy theorem names
2011-09-22, by huffman
take out remote E-SInE -- it's broken and Geoff says it might take quite a while before he gets to it, plus it's fairly obsolete in the meantime
2011-09-22, by blanchet
Moved extraction part of Higman's lemma to separate theory to allow reuse in
2011-09-22, by berghofe
Removed hcentering and vcentering options, since they are not supported
2011-09-22, by berghofe
merged
2011-09-22, by berghofe
Added documentation for HOL-SPARK
2011-09-22, by berghofe
drop partial monomorphic instances in Metis, like in Sledgehammer
2011-09-22, by blanchet
better type reconstruction -- prevents ill-instantiations in proof replay
2011-09-22, by blanchet
NEWS: mention replacement lemmas for the removed ones in Complete_Lattices
2011-09-22, by hoelzl
changing quickcheck_timeout to 30 seconds in mutabelle's testing
2011-09-22, by bulwahn
adding post-processing of terms to narrowing-based Quickcheck
2011-09-22, by bulwahn
HOL/ex/ROOT.ML: only list BinEx once
2011-09-21, by huffman
merged
2011-09-21, by huffman
remove redundant instantiation ereal :: power
2011-09-21, by huffman
reintroduced Minipick as Nitpick example
2011-09-21, by blanchet
tuned comment
2011-09-21, by blanchet
merged
2011-09-21, by huffman
Extended_Real_Limits: generalize some lemmas
2011-09-20, by huffman
add lemmas within_empty and tendsto_bot;
2011-09-20, by huffman
made SML/NJ happy;
2011-09-22, by wenzelm
abstract System_Channel in ML (cf. Scala version);
2011-09-22, by wenzelm
alternative Socket_Channel;
2011-09-21, by wenzelm
more abstract wrapping of fifos as System_Channel;
2011-09-21, by wenzelm
slightly more general Socket_IO as part of Pure;
2011-09-21, by wenzelm
more hints on Z3 configuration;
2011-09-21, by wenzelm
reduced default thread stack, to increase the success rate especially on Windows (NB: the actor worker farm tends to produce 100-200 threads for big sessions);
2011-09-21, by wenzelm
renamed inv -> filter
2011-09-21, by nipkow
Added proofs about narowing
2011-09-21, by nipkow
added missing makefile dependence
2011-09-21, by nipkow
added example
2011-09-21, by nipkow
tuned
2011-09-21, by nipkow
refined comment
2011-09-21, by nipkow
fixed two typos in IMP (by Jean Pichon)
2011-09-21, by kleing
merged
2011-09-21, by nipkow
Updated IMP to use new induction method
2011-09-20, by nipkow
New proof method "induction" that gives induction hypotheses the name IH.
2011-09-20, by nipkow
official status for UN_singleton
2011-09-20, by haftmann
tuned specification and lemma distribution among theories; tuned proofs
2011-09-20, by haftmann
more careful treatment of initial update, similar to output panel;
2011-09-20, by wenzelm
proper fact binding;
2011-09-20, by wenzelm
syntactic improvements and tuning names in the code generator due to Florian's code review
2011-09-20, by bulwahn
match types when applying mono_thm -- previous export generalizes type variables;
2011-09-20, by krauss
fixed headers;
2011-09-19, by wenzelm
less ambiguous syntax;
2011-09-19, by wenzelm
tuned proofs;
2011-09-19, by wenzelm
merged
2011-09-19, by wenzelm
catch PatternMatchFail exceptions in narrowing-based quickcheck
2011-09-19, by bulwahn
removing superfluous definition in the quickcheck narrowing invocation as the code generator now generates valid Haskell code with necessary type annotations without a separate definition
2011-09-19, by bulwahn
ensuring that some constants are generated in the source code by adding calls in ensure_testable
2011-09-19, by bulwahn
adding abstraction layer; more precise function names
2011-09-19, by bulwahn
adding type annotations more aggressively and redundantly to make code generation more reliable even when special printers for some constants are used
2011-09-19, by bulwahn
determining the fastype of a case-pattern but ignoring dummy type constructors that were added as markers for type annotations
2011-09-19, by bulwahn
only annotating constants with sort constraints
2011-09-19, by bulwahn
also adding type annotations for the dynamic invocation
2011-09-19, by bulwahn
removed legacy lemmas in Complete_Lattices
2011-09-19, by noschinl
increasing quickcheck timeout to reduce spurious test failures due to massive parallel invocations and bad scheduling
2011-09-19, by bulwahn
more isatest stats;
2011-09-19, by wenzelm
refined Symbol.is_symbolic -- cover recoded versions as well;
2011-09-19, by wenzelm
double clicks switch to document node buffer;
2011-09-19, by wenzelm
tuned;
2011-09-19, by wenzelm
explicit border independent of UI (cf. ad5883642a83, 2bec3b7514cf);
2011-09-19, by wenzelm
at least 2 worker threads to ensure some degree of lifeness, notably for asynchronous Document.print_state;
2011-09-19, by wenzelm
instantaneous cleanup (NB: VIEWER should be synchronous, cf. dd25b3055c4e);
2011-09-19, by wenzelm
unique file names via serial numbers, to allow files like "root" or multiple files with same base name;
2011-09-19, by wenzelm
imitate Apple in setting initial shell PATH -- especially relevant for MacTeX, MacPorts etc.;
2011-09-19, by wenzelm
merged
2011-09-18, by huffman
numeral_simprocs.ML: use HOL_basic_ss instead of HOL_ss for internal normalization proofs of cancel_factor simprocs, to avoid splitting if-then-else
2011-09-15, by huffman
removed obsolete patches for PG 4.1;
2011-09-18, by wenzelm
additional space for borderless UI;
2011-09-18, by wenzelm
more robust treatment of empty insets (NB: border may be null on some UIs, e.g. Windows);
2011-09-18, by wenzelm
explicit master_dir as part of header -- still required (for Cygwin) since Scala layer does not pass file content yet;
2011-09-18, by wenzelm
isatest settings for macbroy6 (Mac OS X Lion);
2011-09-18, by wenzelm
more Mac OS reference hardware;
2011-09-18, by wenzelm
updated to SML/NJ 110.73;
2011-09-18, by wenzelm
tentative announcement based on current NEWS;
2011-09-18, by wenzelm
tuned;
2011-09-18, by wenzelm
separated NEWS for Isabelle2011 from Isabelle2011-1 (cf. e1139e612b55);
2011-09-18, by wenzelm
updated for release;
2011-09-18, by wenzelm
tuned;
2011-09-18, by wenzelm
updated generated file;
2011-09-18, by wenzelm
updated Complete_Lattices;
2011-09-18, by wenzelm
some tuning and re-ordering for release;
2011-09-18, by wenzelm
misc tuning for release;
2011-09-18, by wenzelm
more contributors;
2011-09-18, by wenzelm
tuned proofs;
2011-09-18, by wenzelm
tweak keyboard shortcuts for Mac OS X;
2011-09-18, by wenzelm
explicit check_file wrt. jEdit VFS, to avoid slightly confusing empty buffer after IO error;
2011-09-18, by wenzelm
finite sequences as useful as introductory example;
2011-09-18, by wenzelm
discontinued hard-wired JAVA_HOME treatment for Mac OS X (cf. f471a2fb9a95), which can cause confusions of "isabelle java" vs. "isabelle scala" -- moved settings to external component;
2011-09-18, by wenzelm
graph traversal in topological order;
2011-09-18, by wenzelm
Document.Node.Name convenience;
2011-09-17, by wenzelm
more precise painting;
2011-09-17, by wenzelm
more elaborate Node_Renderer, which paints node_name.theory only;
2011-09-17, by wenzelm
raised default log level -- to avoid confusing warning about scala.tools.nsc.plugins.Plugin, which is mistaken as jEdit plugin;
2011-09-17, by wenzelm
tuned signature;
2011-09-17, by wenzelm
more careful traversal of theory dependencies to retain standard import order;
2011-09-17, by wenzelm
sane default for class Thy_Load;
2011-09-17, by wenzelm
removed obsolete patches for PG 4.1;
2011-09-17, by wenzelm
specific bundle for x86_64-linux, which is especially important for JRE due to its extra library dependencies;
2011-09-17, by wenzelm
added "isabelle scalac" convenience;
2011-09-17, by wenzelm
Symbol.explode as in ML;
2011-09-17, by wenzelm
ignore OUTPUT to avoid spam -- jEdit menu "Troubleshooting / Activity Log" should be sufficient;
2011-09-17, by wenzelm
dropped unused argument – avoids problem with SML/NJ
2011-09-17, by haftmann
tuned spacing
2011-09-17, by haftmann
tuned
2011-09-17, by haftmann
tuned post fixpoint setup
2011-09-17, by nipkow
merged
2011-09-17, by nipkow
when applying induction rules, remove names of assumptions that come
2011-09-16, by nipkow
remove stray "using [[simp_trace]]"
2011-09-16, by noschinl
tune indenting
2011-09-16, by noschinl
removed unused legacy lemma names, some comment cleanup.
2011-09-16, by kleing
removed word_neq_0_conv from simpset, it's almost never wanted.
2011-09-16, by kleing
removed further legacy rules from Complete_Lattices
2011-09-15, by hoelzl
NEWS on Complete_Lattices, Lattices
2011-09-15, by noschinl
tail recursive proof preprocessing (needed for huge proofs)
2011-09-15, by blanchet
tuning
2011-09-15, by blanchet
merged
2011-09-15, by nipkow
revised AbsInt and added widening and narrowing
2011-09-15, by nipkow
updated comment
2011-09-14, by haftmann
updated generated code
2011-09-14, by haftmann
tuned
2011-09-13, by haftmann
renamed Complete_Lattices lemmas, removed legacy names
2011-09-14, by hoelzl
merged
2011-09-14, by noschinl
create central list for language extensions used by the haskell code generator
2011-09-14, by noschinl
observe distinction between sets and predicates
2011-09-14, by boehmes
merged
2011-09-14, by nipkow
cleand up AbsInt fixpoint iteration; tuned syntax
2011-09-14, by nipkow
tuned proofs
2011-09-13, by huffman
tuned proofs
2011-09-13, by huffman
remove some redundant [simp] declarations;
2011-09-13, by huffman
tune proofs
2011-09-13, by noschinl
tune simpset for Complete_Lattices
2011-09-13, by noschinl
merged
2011-09-13, by bulwahn
added lemma motivated by a more specific lemma in the AFP-KBPs theories
2011-09-13, by bulwahn
simplified unsound proof detection by removing impossible case
2011-09-13, by blanchet
correcting NEWS
2011-09-13, by bulwahn
correcting theory name and dependencies
2011-09-13, by bulwahn
renamed AList_Impl to AList
2011-09-13, by bulwahn
fastsimp -> fastforce in doc
2011-09-13, by nipkow
fix typo
2011-09-12, by huffman
shorten proof of frontier_straddle
2011-09-12, by huffman
NEWS and CONTRIBUTORS
2011-09-12, by huffman
remove redundant lemma Lim_sequentially in favor of lemma LIMSEQ_def
2011-09-12, by huffman
simplify proofs using LIMSEQ lemmas
2011-09-12, by huffman
remove trivial lemma Lim_at_iff_LIM
2011-09-12, by huffman
fix typos
2011-09-12, by huffman
NEWS for euclidean_space class
2011-09-12, by huffman
move lemmas about complex number 'i' to Complex.thy and Library/Inner_Product.thy
2011-09-12, by huffman
adding NEWS and CONTRIBUTORS
2011-09-12, by hoelzl
merged
2011-09-12, by bulwahn
correcting imports after splitting and renaming AssocList
2011-09-12, by bulwahn
tuned
2011-09-12, by bulwahn
moving connection of association lists to Mappings into a separate theory
2011-09-12, by bulwahn
adding NEWS and CONTRIBUTORS
2011-09-12, by bulwahn
tuned some symbol that probably went there by some strange encoding issue
2011-09-12, by bulwahn
added my contributions to NEWS and CONTRIBUTORS
2011-09-12, by blanchet
fixed type intersection (again)
2011-09-12, by blanchet
consistent option naming
2011-09-12, by blanchet
NEWS fastsimp -> fastforce
2011-09-12, by nipkow
new fastforce replacing fastsimp - less confusing name
2011-09-12, by nipkow
merged
2011-09-11, by wenzelm
NEWS for Library/Product_Lattice.thy
2011-09-11, by huffman
misc tuning and clarification;
2011-09-11, by wenzelm
merged
2011-09-11, by wenzelm
merged
2011-09-11, by huffman
tuned proofs
2011-09-11, by huffman
Library/Saturated.thy: 'Sat' abbreviates 'of_nat'
2011-09-11, by huffman
more CONTRIBUTORS;
2011-09-11, by wenzelm
persistent ISABELLE_INTERFACE_CHOICE;
2011-09-11, by wenzelm
explicit choice of interface;
2011-09-11, by wenzelm
more orthogonal signature;
2011-09-11, by wenzelm
updates for release;
2011-09-11, by wenzelm
misc tuning and clarification (NB: settings are already local for named snapshots/releases);
2011-09-11, by wenzelm
some updates of PLATFORMS;
2011-09-11, by wenzelm
more README;
2011-09-11, by wenzelm
merged
2011-09-10, by wenzelm
mem_prs and mem_rsp in accordance with sets-as-predicates representation (backported from AFP/Coinductive)
2011-09-10, by krauss
misc tuning;
2011-09-10, by wenzelm
misc tuning and clarification;
2011-09-10, by wenzelm
speed up slow proof;
2011-09-10, by wenzelm
merged
2011-09-10, by wenzelm
more modularization
2011-09-10, by haftmann
stronger colors (as background);
2011-09-10, by wenzelm
some color scheme for theory status;
2011-09-10, by wenzelm
some keyboard shortcuts for important actions;
2011-09-10, by wenzelm
explicit jEdit actions -- to enable key mappings, for example;
2011-09-10, by wenzelm
more symbolic file positions via smart replacement of ISABELLE_HOME -- allows Isabelle distribution to be moved later on;
2011-09-10, by wenzelm
tuned usage;
2011-09-10, by wenzelm
simplified default Isabelle application wrapper (NB: build process is already part of isabelle jedit tool);
2011-09-10, by wenzelm
renamed theory Complete_Lattice to Complete_Lattices, in accordance with Lattices, Orderings etc.
2011-09-10, by haftmann
fixed definition of type intersection (soundness bug)
2011-09-10, by blanchet
continue with minimization in debug mode in spite of unsoundness
2011-09-10, by blanchet
generalize lemma of_nat_number_of_eq to class number_semiring
2011-09-09, by huffman
merged
2011-09-09, by bulwahn
stating more explicitly our expectation that these two terms have the same term structure
2011-09-09, by bulwahn
revisiting type annotations for Haskell: necessary type annotations are not inferred on the provided theorems but using the arguments and right hand sides, as these might differ in the case of constants with abstract code types
2011-09-09, by bulwahn
made SML/NJ happy
2011-09-09, by blanchet
call ghc with -XEmptyDataDecls
2011-09-08, by noschinl
merged
2011-09-09, by nipkow
tuned headers
2011-09-09, by nipkow
Library/Saturated.thy: number_semiring class instance
2011-09-08, by huffman
remove lemmas nat_add_min_{left,right} in favor of generic lemmas min_add_distrib_{left,right}
2011-09-08, by huffman
merged
2011-09-08, by huffman
remove unnecessary intermediate lemmas
2011-09-08, by huffman
added syntactic classes for "inf" and "sup"
2011-09-09, by krauss
prove existence, uniqueness, and other properties of complex arg function
2011-09-08, by huffman
tuned
2011-09-08, by huffman
remove obsolete intermediate lemma complex_inverse_complex_split
2011-09-08, by huffman
tuned
2011-09-08, by huffman
merged
2011-09-08, by haftmann
tuned
2011-09-08, by haftmann
merged
2011-09-08, by haftmann
merged
2011-09-07, by haftmann
merged
2011-09-06, by haftmann
merged
2011-09-06, by haftmann
merged
2011-09-06, by haftmann
tuned
2011-09-05, by haftmann
merged
2011-09-05, by haftmann
tuned
2011-09-05, by haftmann
tuned
2011-09-04, by haftmann
fixed computation of "in_conj" for polymorphic encodings
2011-09-08, by blanchet
add some new lemmas about cis and rcis;
2011-09-07, by huffman
Complex.thy: move theorems into appropriate subsections
2011-09-07, by huffman
merged
2011-09-07, by huffman
remove redundant lemma complex_of_real_minus_one
2011-09-07, by huffman
simplify proof of lemma DeMoivre, removing unnecessary intermediate lemma
2011-09-07, by huffman
removed unused lemma sin_cos_squared_add2_mult
2011-09-07, by huffman
remove duplicate lemma real_of_int_real_of_nat in favor of real_of_int_of_nat_eq
2011-09-07, by huffman
avoid using legacy theorem names
2011-09-07, by huffman
merged
2011-09-08, by wenzelm
theory of saturated naturals contributed by Peter Gammie
2011-09-07, by haftmann
theory of saturated naturals contributed by Peter Gammie
2011-09-07, by haftmann
lemmas about +, *, min, max on nat
2011-09-07, by haftmann
update Sledgehammer docs
2011-09-07, by blanchet
added new tagged encodings to Metis tests
2011-09-07, by blanchet
also implemented ghost version of the tagged encodings
2011-09-07, by blanchet
added new guards encoding to test
2011-09-07, by blanchet
smarter explicit apply business
2011-09-07, by blanchet
started work on ghost type arg encoding
2011-09-07, by blanchet
stricted type encoding parsing
2011-09-07, by blanchet
more substructural sharing to gain significant compression;
2011-09-08, by wenzelm
XML.cache for partial sharing (strings only);
2011-09-07, by wenzelm
platform-specific look and feel;
2011-09-07, by wenzelm
more README;
2011-09-07, by wenzelm
clarified terminology;
2011-09-07, by wenzelm
no print_state for final proof commands, which return to theory state;
2011-09-07, by wenzelm
NEWS on IsabelleText font;
2011-09-07, by wenzelm
explicit join_syntax ensures command transaction integrity of 'theory';
2011-09-07, by wenzelm
some updates for release;
2011-09-07, by wenzelm
some tuning for release;
2011-09-07, by wenzelm
updated file locations;
2011-09-07, by wenzelm
merged
2011-09-07, by wenzelm
merged
2011-09-07, by bulwahn
removing previously used function locally_monomorphic in the code generator
2011-09-07, by bulwahn
setting const_sorts to false in the type inference of the code generator
2011-09-07, by bulwahn
adapting Imperative HOL serializer to changes of the iterm datatype in the code generator
2011-09-07, by bulwahn
removing previous crude approximation to add type annotations to disambiguate types
2011-09-07, by bulwahn
adding minimalistic implementation for printing the type annotations
2011-09-07, by bulwahn
adding call to disambiguation annotations
2011-09-07, by bulwahn
adding type inference for disambiguation annotations in code equation
2011-09-07, by bulwahn
adding the body type as well to the code generation for constants as it is required for type annotations of constants
2011-09-07, by bulwahn
changing const type to pass along if typing annotations are necessary for disambigous terms
2011-09-07, by bulwahn
fixed THF type constructor syntax
2011-09-07, by blanchet
tweaking polymorphic TFF and THF output
2011-09-07, by blanchet
parse new experimental '@' encodings
2011-09-07, by blanchet
tuning
2011-09-07, by blanchet
tuning
2011-09-07, by blanchet
tuning
2011-09-07, by blanchet
clarified import;
2011-09-07, by wenzelm
tuned/simplified proofs;
2011-09-07, by wenzelm
tuned proofs;
2011-09-07, by wenzelm
deactivate unfinished charset provider for now, to avoid user confusion;
2011-09-07, by wenzelm
more NEWS;
2011-09-07, by wenzelm
added "check" button: adhoc change to full buffer perspective;
2011-09-07, by wenzelm
added "cancel" button based on cancel_execution, not interrupt (cf. 156be0e43336);
2011-09-07, by wenzelm
separate mangling, which can (and should) be done before the formulas are first-orderized, and type arg filtering, which must be done after once the min arities have been computed
2011-09-07, by blanchet
perform mangling before computing symbol arity, to avoid needless "hAPP"s and "hBOOL"s
2011-09-07, by blanchet
tuning
2011-09-07, by blanchet
make mangling sound w.r.t. type arguments
2011-09-07, by blanchet
make "filter_type_args" more robust if the actual arity is higher than the declared one
2011-09-07, by blanchet
updated Sledgehammer documentation
2011-09-07, by blanchet
rationalize uniform encodings
2011-09-07, by blanchet
merged
2011-09-06, by huffman
avoid using legacy theorem names
2011-09-06, by huffman
merged
2011-09-06, by huffman
remove redundant lemmas i_mult_eq and i_mult_eq2 in favor of i_squared
2011-09-06, by huffman
HOL/Import: Update HOL4 generated files to current Isabelle.
2011-09-07, by Cezary Kaliszyk
tuned proofs;
2011-09-07, by wenzelm
remove some unnecessary simp rules from simpset
2011-09-06, by huffman
some Isabelle/jEdit NEWS;
2011-09-06, by wenzelm
more README;
2011-09-06, by wenzelm
merged
2011-09-06, by wenzelm
merged
2011-09-06, by huffman
simplify proof of tan_half, removing unused assumptions
2011-09-06, by huffman
convert some proofs to Isar-style
2011-09-06, by huffman
added dummy polymorphic THF system
2011-09-06, by blanchet
added some examples for pattern and weight annotations
2011-09-06, by boehmes
merged
2011-09-06, by bulwahn
avoid "Code" as structure name (cf. 3bc39cfe27fe)
2011-09-06, by bulwahn
remove duplicate copy of lemma sqrt_add_le_add_sqrt
2011-09-06, by huffman
remove redundant lemma real_sum_squared_expand in favor of power2_sum
2011-09-06, by huffman
remove redundant lemma LIMSEQ_Complex in favor of tendsto_Complex
2011-09-06, by huffman
merged
2011-09-06, by huffman
add lemmas about arctan;
2011-09-05, by huffman
convert lemma cos_total to Isar-style proof
2011-09-05, by huffman
added new lemmas
2011-09-06, by nipkow
updated Sledgehammer's docs
2011-09-06, by blanchet
cleanup "simple" type encodings
2011-09-06, by blanchet
merge
2011-09-06, by Cezary Kaliszyk
HOL/Import: Make HOL4 Import work with current Isabelle. Updated constant maps, added bool type map, and tuned compat theorem.
2011-09-06, by Cezary Kaliszyk
tuning
2011-09-06, by blanchet
drop more type arguments soundly, when they can be deduced from the arg types
2011-09-06, by blanchet
bulk reports for improved message throughput;
2011-09-06, by wenzelm
bulk reports for improved message throughput;
2011-09-06, by wenzelm
tuned signature;
2011-09-06, by wenzelm
more specific message channels to avoid potential bottle-neck of raw_messages;
2011-09-06, by wenzelm
buffer prover messages to prevent overloading of session_actor input channel -- which is critical due to synchronous messages wrt. GUI thread;
2011-09-06, by wenzelm
more abstract receiver interface;
2011-09-06, by wenzelm
flush after Output.raw_message (and init message) for reduced latency of important protocol events;
2011-09-06, by wenzelm
convert lemma cos_is_zero to Isar-style
2011-09-05, by huffman
merged
2011-09-05, by huffman
convert lemma sin_gt_zero to Isar style;
2011-09-05, by huffman
modify lemma sums_group, and shorten proofs that use it
2011-09-05, by huffman
generalize some lemmas
2011-09-05, by huffman
add lemmas cos_arctan and sin_arctan
2011-09-05, by huffman
tuned indentation
2011-09-05, by huffman
more visible outdated_color;
2011-09-05, by wenzelm
commands_change_delay within main actor -- prevents overloading of commands_change_buffer input channel;
2011-09-05, by wenzelm
tuned imports;
2011-09-05, by wenzelm
fixed handling of "sledgehammer_params", so that "sledgehammer_params [e]" is really the same as "sledgehammer_params [provers = e]"
2011-09-05, by blanchet
tuned
2011-09-05, by boehmes
tuned
2011-09-05, by boehmes
filter out all schematic theorems if the problem contains no ground constants
2011-09-05, by boehmes
merged
2011-09-04, by huffman
tuned comments
2011-09-04, by huffman
simplify proof of Bseq_mono_convergent
2011-09-04, by huffman
merged
2011-09-04, by wenzelm
replace lemma expi_imaginary with reoriented lemma cis_conv_exp
2011-09-04, by huffman
remove redundant lemmas expi_add and expi_zero
2011-09-04, by huffman
remove redundant lemmas about LIMSEQ
2011-09-04, by huffman
introduce abbreviation 'int' earlier in Int.thy
2011-09-04, by huffman
remove unused assumptions from natceiling lemmas
2011-09-04, by huffman
move lemmas nat_le_iff and nat_mono into Int.thy
2011-09-04, by huffman
eliminated markup for plain identifiers (frequent but insignificant);
2011-09-04, by wenzelm
simplified signatures;
2011-09-04, by wenzelm
synchronous XML.Cache without actor -- potentially more efficient on machines with few cores;
2011-09-04, by wenzelm
tuned document;
2011-09-04, by wenzelm
improved handling of extended styles and hard tabs when prover is inactive;
2011-09-04, by wenzelm
mark hard tabs as single chunks, as required by jEdit;
2011-09-04, by wenzelm
updated READMEs;
2011-09-04, by wenzelm
property "tooltip-dismiss-delay" is edited in ms, not seconds;
2011-09-04, by wenzelm
moved XML/YXML to src/Pure/PIDE;
2011-09-04, by wenzelm
pass raw messages through xml_cache actor, which is important to retain ordering of results (e.g. read_command reports before assign, cf. 383c9d758a56);
2011-09-04, by wenzelm
pseudo-definition for perms on sets; tuned
2011-09-04, by haftmann
remove duplicate lemma nat_zero in favor of nat_0
2011-09-03, by huffman
merged
2011-09-03, by huffman
merged
2011-09-03, by huffman
modify nominal packages to better respect set/pred distinction
2011-09-03, by huffman
merged
2011-09-03, by huffman
remove unused assumption from lemma posreal_complete
2011-09-03, by huffman
tuned specifications
2011-09-03, by haftmann
merged
2011-09-03, by haftmann
tuned proof
2011-09-03, by haftmann
merged
2011-09-03, by haftmann
assert Pure equations for theorem references; avoid dynamic reference to fact
2011-09-03, by haftmann
assert Pure equations for theorem references; tuned
2011-09-03, by haftmann
tuned specifications and proofs
2011-09-03, by haftmann
merged
2011-09-03, by wenzelm
remove duplicate lemma finite_choice in favor of finite_set_choice
2011-09-03, by huffman
simplify proof
2011-09-03, by huffman
shorten some proofs
2011-09-03, by huffman
remove redundant simp rules ceiling_floor and floor_ceiling
2011-09-02, by huffman
misc tuning and simplification of proofs;
2011-09-03, by wenzelm
Document.removed_versions on Scala side;
2011-09-03, by wenzelm
discontinued predefined empty command (obsolete!?);
2011-09-03, by wenzelm
discontinued global execs: store exec value directly within entries;
2011-09-03, by wenzelm
Document.remove_versions on ML side;
2011-09-03, by wenzelm
some support to prune_history;
2011-09-03, by wenzelm
merged
2011-09-02, by huffman
speed up extremely slow metis proof of Sup_real_iff
2011-09-02, by huffman
remove redundant lemma reals_complete2 in favor of complete_real
2011-09-02, by huffman
simplify proof of Rats_dense_in_real;
2011-09-02, by huffman
remove unused, unnecessary lemmas
2011-09-02, by huffman
remove more duplicate lemmas
2011-09-02, by huffman
merged
2011-09-02, by wenzelm
merged
2011-09-02, by haftmann
avoid "Code" as structure name
2011-09-02, by haftmann
more robust chunk painting wrt. hard tabs, when chunk.str == null;
2011-09-02, by wenzelm
raw message function "assign_execs" avoids full overhead of decoding and caching message body;
2011-09-02, by wenzelm
less agressive parsing of commands (priority ~1);
2011-09-02, by wenzelm
tuned;
2011-09-02, by wenzelm
more direct Token.range_pos and Outer_Syntax.read_command, bypassing Thy_Syntax.span;
2011-09-02, by wenzelm
merged
2011-09-02, by nipkow
Added Abstract Interpretation theories
2011-09-02, by nipkow
tuned proofs;
2011-09-02, by wenzelm
proper config option linarith_trace;
2011-09-02, by wenzelm
discontinued slightly odd "Defining record ..." message and corresponding quiet_mode;
2011-09-02, by wenzelm
merged
2011-09-02, by wenzelm
renamed "Metis_Tactics" to "Metis_Tactic", now that there is only one Metis tactic ("metisFT" is legacy)
2011-09-02, by blanchet
use new syntax for Pi binder in TFF1 output
2011-09-02, by blanchet
fewer TPTP important messages
2011-09-02, by blanchet
simplify some proofs about uniform continuity, and add some new ones;
2011-09-01, by huffman
modernize lemmas about 'continuous' and 'continuous_on';
2011-09-01, by huffman
add lemma tendsto_infnorm
2011-09-01, by huffman
more precise iterate_entries_after if start refers to last entry;
2011-09-02, by wenzelm
clarified define_command: store name as structural information;
2011-09-02, by wenzelm
amended last_common, if that happens to the very last entry (important to load HOL/Auth, for example);
2011-09-01, by wenzelm
more redable Document.Node.toString;
2011-09-01, by wenzelm
sort wrt. theory name;
2011-09-01, by wenzelm
modernized theory name;
2011-09-01, by wenzelm
repaired benchmarks;
2011-09-01, by wenzelm
merged
2011-09-01, by wenzelm
tuning
2011-09-01, by blanchet
always measure time for ATPs -- auto minimization relies on it
2011-09-01, by blanchet
added two lemmas about "distinct" to help Sledgehammer
2011-09-01, by blanchet
make "sound" sound and "unsound" more sound, based on evaluation
2011-09-01, by blanchet
HOL/Import: observe distinction between sets and predicates (where possible)
2011-09-01, by Cezary Kaliszyk
simplify/generalize some proofs
2011-08-31, by huffman
generalize lemma isCont_vec_nth
2011-08-31, by huffman
convert proof to Isar-style
2011-08-31, by huffman
remove redundant lemma card_enum
2011-08-31, by huffman
move lemmas from Topology_Euclidean_Space to Euclidean_Space
2011-08-31, by huffman
convert to Isar-style proof
2011-08-31, by huffman
make SML/NJ happy
2011-08-31, by blanchet
more tuning
2011-08-31, by blanchet
more tuning
2011-08-31, by blanchet
tuning
2011-08-31, by blanchet
avoid relying on dubious TFF1 feature
2011-08-31, by blanchet
killed FIXME (the ATP exporter outputs TPTP FOF, which is first-order)
2011-08-31, by blanchet
fixed explicit declaration of TFF1 types
2011-08-31, by blanchet
adding list_size_append (thanks to Rene Thiemann)
2011-08-30, by bulwahn
strengthening list_size_pointwise (thanks to Rene Thiemann)
2011-08-30, by bulwahn
more flexible sorting;
2011-09-01, by wenzelm
tuned signature;
2011-09-01, by wenzelm
more abstract Document.Node.Name;
2011-09-01, by wenzelm
more careful treatment of interrupts, to retain them within forked/joined boundary of command transactions;
2011-09-01, by wenzelm
crude display of node status;
2011-08-31, by wenzelm
explicit cancel_execution before queueing new edits -- potential performance improvement for machines with few cores;
2011-08-31, by wenzelm
explicit running_color;
2011-08-31, by wenzelm
tuned join_commands: avoid traversing cumulative table;
2011-08-31, by wenzelm
some support for theory status overview;
2011-08-31, by wenzelm
tuned Commands_Changed: cover nodes as well;
2011-08-31, by wenzelm
maintain name of *the* enclosing node as part of command -- avoid full document traversal;
2011-08-31, by wenzelm
improved auto loading: selectable file list;
2011-08-31, by wenzelm
tuned document;
2011-08-30, by wenzelm
tuned import;
2011-08-30, by wenzelm
tuned document;
2011-08-30, by wenzelm
tuned color for Mac OS X (very light color profile?);
2011-08-30, by wenzelm
tuned document;
2011-08-30, by wenzelm
merged;
2011-08-30, by wenzelm
fixed just introduced silly bug
2011-08-30, by blanchet
"simple" was renamed "mono_simple" and there's now "poly_simple" as well -- but they are not needed here since for Metis they amount to the same as guards
2011-08-30, by blanchet
tuning
2011-08-30, by blanchet
cleaner "pff" dummy TFF0 prover
2011-08-30, by blanchet
generate properly typed TFF1 (PFF) problems in the presence of type class predicates
2011-08-30, by blanchet
added type abstractions (for declaring polymorphic constants) to TFF syntax
2011-08-30, by blanchet
implement more of the polymorphic simply typed format TFF(1)
2011-08-30, by blanchet
flip logic of boolean option so it's off by default
2011-08-30, by blanchet
extended simple types with polymorphism -- the implementation still needs some work though
2011-08-30, by blanchet
added dummy PFF prover, for debugging purposes
2011-08-30, by blanchet
first step towards polymorphic TFF + changed defaults for Vampire
2011-08-30, by blanchet
tuning
2011-08-30, by blanchet
removed explicit reliance on Hilbert_Choice.Eps
2011-08-30, by nik
improved handling of induction rules in Sledgehammer
2011-08-30, by nik
added generation of induction rules
2011-08-30, by nik
simplify some proofs
2011-08-29, by huffman
restrict perspective to actual buffer_range, to avoid spurious edits due to faulty last_exec_offset (NB: jEdit screenlines may be silently extended by trailing newline);
2011-08-30, by wenzelm
tuned signature;
2011-08-30, by wenzelm
dynamic exec state lookup for implicit position information (e.g. 'definition' without binding);
2011-08-30, by wenzelm
some support for hyperlinks between different buffers;
2011-08-30, by wenzelm
tuned colors -- more distance between outdated_color and quoted_color;
2011-08-30, by wenzelm
do not normalized extra file dependencies for now -- still loaded by prover process;
2011-08-30, by wenzelm
separate module for jEdit primitives for loading theory files;
2011-08-30, by wenzelm
merged
2011-08-29, by wenzelm
Product_Vector.thy: clean up some proofs
2011-08-29, by huffman
actual auto loading of required files;
2011-08-29, by wenzelm
some dialog for auto loading of required files (still inactive);
2011-08-29, by wenzelm
invoke in Swing thread to make double sure;
2011-08-29, by wenzelm
move class perfect_space into RealVector.thy;
2011-08-28, by huffman
generalize LIM_zero lemmas to arbitrary filters
2011-08-28, by huffman
merged
2011-08-28, by huffman
discontinue many legacy theorems about LIM and LIMSEQ, in favor of tendsto theorems
2011-08-28, by huffman
tuned
2011-08-28, by haftmann
split timeout among ATPs in and add Metis to the mix as backup
2011-08-28, by blanchet
more portable cp options, e.g. for non-GNU version on Mac OS X Leopard;
2011-08-28, by wenzelm
tuned positions of ambiguity messages -- less intrusive in IDE view;
2011-08-28, by wenzelm
tuned
2011-08-28, by haftmann
merged
2011-08-28, by haftmann
avoid loading List_Cset and Dlist_Cet at the same time
2011-08-28, by haftmann
corrected slip
2011-08-28, by haftmann
Cset, Dlist_Cset, List_Cset: restructured
2011-08-27, by haftmann
Cset, Dlist_Cset, List_Cset: restructured
2011-08-27, by haftmann
adapted to changes in Cset.thy
2011-08-27, by haftmann
adapted to changes in Cset.thy
2011-08-26, by haftmann
separating predicates and sets syntactically
2011-08-26, by haftmann
merged
2011-08-26, by haftmann
avoid intermixing set and predicates; dropped lemmas mem_rsp and mem_prs (now in Quotient_Set.thy)
2011-08-26, by haftmann
updated generated files
2011-08-25, by haftmann
merged
2011-08-25, by haftmann
updated generated files
2011-08-25, by haftmann
explicit markup for legacy warnings;
2011-08-27, by wenzelm
updated generated files;
2011-08-27, by wenzelm
less aggressive warning icon;
2011-08-27, by wenzelm
tuned colors;
2011-08-27, by wenzelm
transparent foreground color for quoted entities;
2011-08-27, by wenzelm
more precise treatment of nodes that are fully required for partially visible ones;
2011-08-27, by wenzelm
de-assigned commands also count as changed;
2011-08-27, by wenzelm
beef up sledgehammer_tac in Mirabelle some more
2011-08-27, by blanchet
merged
2011-08-27, by blanchet
change default for generation of tag idempotence and tag argument equations
2011-08-26, by blanchet
merged
2011-08-26, by huffman
NEWS entry for setsum_norm ~> norm_setsum
2011-08-26, by huffman
make HOL-Probability respect set/pred distinction
2011-08-26, by huffman
merged
2011-08-26, by wenzelm
use rename_tac to make proof script more robust (with separate set type, 'clarify' yields different variable names)
2010-09-08, by huffman
merged
2011-08-26, by huffman
generalize and simplify proof of continuous_within_sequentially
2011-08-26, by huffman
add lemma sequentially_imp_eventually_within;
2011-08-26, by huffman
replace some continuous_on lemmas with more general versions
2011-08-25, by huffman
remove legacy theorem Lim_inner
2011-08-25, by huffman
arrange everything related to ordered_euclidean_space class together
2011-08-25, by huffman
generalize and shorten proof of basis_orthogonal
2011-08-25, by huffman
remove dot_lsum and dot_rsum in favor of inner_setsum_{left,right}
2011-08-25, by huffman
merged
2011-08-25, by huffman
generalize lemma finite_imp_compact_convex_hull and related lemmas
2011-08-25, by huffman
generalize some lemmas
2011-08-25, by huffman
generalize lemma convex_cone_hull
2011-08-25, by huffman
rename subset_{interior,closure} to {interior,closure}_mono;
2011-08-25, by huffman
simplify many proofs about subspace and span;
2011-08-25, by huffman
remove duplicate simp declaration
2011-08-25, by huffman
simplify definition of 'interior';
2011-08-25, by huffman
add lemma closure_union;
2011-08-24, by huffman
minimize imports
2011-08-24, by huffman
move everything related to 'norm' method into new theory file Norm_Arith.thy
2011-08-24, by huffman
remove unused lemmas dimensionI, dimension_eq
2011-08-24, by huffman
move geometric progression lemmas from Linear_Algebra.thy to Integration.thy where they are used
2011-08-24, by huffman
merge
2011-08-26, by Cezary Kaliszyk
FSet: Explicit proof without mem_def
2011-08-26, by Cezary Kaliszyk
merged
2011-08-26, by nipkow
added lemma
2011-08-26, by nipkow
added a component in generated file names reflecting whether the minimizer is used -- needed for evaluation to keep these files separated from the main problem files
2011-08-26, by blanchet
comment
2011-08-26, by blanchet
disable TFF for Vampire 1.8 until they've fixed the soundness issues and it's back on SystemOnTPTP
2011-08-26, by blanchet
improve completeness of polymorphic encodings
2011-08-26, by blanchet
mangle tag bound declarations properly
2011-08-26, by blanchet
fixed inverted logic and improve precision when handling monotonic types in polymorphic encodings
2011-08-26, by blanchet
make sure that if slicing is disabled, a non-SOS slice is chosen
2011-08-25, by blanchet
honor TFF Implicit
2011-08-25, by blanchet
make polymorphic encodings more complete
2011-08-25, by blanchet
make default unsound mode less unsound
2011-08-25, by blanchet
make TFF output less explicit where possible
2011-08-25, by blanchet
use more appropriate encoding for Z3 TPTP, as confirmed by evaluation
2011-08-25, by blanchet
added one more known Z3 failure
2011-08-25, by blanchet
added config options to control two aspects of the translation, for evaluation purposes
2011-08-25, by blanchet
added choice operator output for
2011-08-25, by nik
rationalized option names -- mono becomes raw_mono and mangled becomes mono
2011-08-25, by blanchet
handle nonmangled monomorphich the same way as mangled monomorphic when it comes to helper -- otherwise we can end up generating too tight type guards
2011-08-25, by blanchet
avoid using ":" for anything but systematic type tag annotations, because Hurd's Metis gives it that special semantics
2011-08-25, by blanchet
fixed bang encoding detection of which types to encode
2011-08-25, by blanchet
lemma Compl_insert: "- insert x A = (-A) - {x}"
2011-08-25, by krauss
avoid variable clashes by properly incrementing indices
2011-08-25, by boehmes
improved completeness and efficiency of Z3 proof reconstruction, especially by an improved handling of Skolemization
2011-08-25, by boehmes
include chained facts for minimizer, otherwise it won't work
2011-08-25, by blanchet
remove Vampire imconplete proof detection -- the bug it was trying to work around has been fixed in version 1.8, and the check is too sensitive anyway
2011-08-24, by blanchet
back to tradition Scratch.thy default -- execution wrt. perspective overcomes the main problems of 226563829580;
2011-08-26, by wenzelm
tuned Session.edit_node: update_perspective based on last_exec_offset;
2011-08-26, by wenzelm
tuned signature -- iterate subsumes both fold and get_first;
2011-08-26, by wenzelm
further clarification of Document.updated, based on last_common and after_entry;
2011-08-26, by wenzelm
tuned signature;
2011-08-26, by wenzelm
improved Document.edit: more accurate update_start and no_execs;
2011-08-26, by wenzelm
refined document state assignment: observe perspective, more explicit assignment message;
2011-08-26, by wenzelm
tuned signature -- emphasize traditional read/eval/print terminology, which is still relevant here;
2011-08-25, by wenzelm
maintain last_execs assignment on Scala side;
2011-08-25, by wenzelm
propagate information about last command with exec state assignment through document model;
2011-08-25, by wenzelm
tuned signature;
2011-08-25, by wenzelm
slightly more abstract Command.Perspective;
2011-08-25, by wenzelm
slightly more abstract Text.Perspective;
2011-08-25, by wenzelm
tuned proofs;
2011-08-24, by wenzelm
tuned syntax -- avoid ambiguities;
2011-08-24, by wenzelm
more accurate treatment of index syntax constants, for proper entity references in concrete notation (e.g. infix "\<oplus>\<index>");
2011-08-24, by wenzelm
delete commented-out dead code
2011-08-24, by huffman
merged
2011-08-24, by huffman
change some subsection headings to subsubsection
2011-08-24, by huffman
remove unnecessary lemma card_ge1
2011-08-23, by huffman
move connected_real_lemma to the one place it is used
2011-08-23, by huffman
merged
2011-08-24, by wenzelm
make sure that all facts are passed to ATP from minimizer
2011-08-24, by blanchet
more reliable "sledgehammer\_tac" reconstruction, by avoiding "insert_tac"
2011-08-24, by blanchet
specify timeout for "sledgehammer_tac"
2011-08-24, by blanchet
tuning
2011-08-24, by blanchet
Quotient Package: add mem_rsp, mem_prs, tune proofs.
2011-08-24, by Cezary Kaliszyk
merged
2011-08-23, by huffman
declare euclidean_simps [simp] at the point they are proved;
2011-08-23, by huffman
merged
2011-08-23, by huffman
merged
2011-08-22, by huffman
avoid warnings
2011-08-22, by huffman
comment out dead code to avoid compiler warnings
2011-08-22, by huffman
legacy theorem names
2011-08-22, by huffman
remove duplicate lemma
2011-08-22, by huffman
fixed "hBOOL" of existential variables, and generate more helpers
2011-08-23, by blanchet
don't select facts when using sledgehammer_tac for reconstruction
2011-08-23, by blanchet
don't perform a triviality check if the goal is skipped anyway
2011-08-23, by blanchet
optional reconstructor
2011-08-23, by blanchet
misc tuning and simplification;
2011-08-24, by wenzelm
tuned pri: prefer purging of canceled execution;
2011-08-24, by wenzelm
tuned Document.node: maintain "touched" flag to indicate changes in entries etc.;
2011-08-24, by wenzelm
clarified Document.Node.clear -- retain header (cf. ML version);
2011-08-24, by wenzelm
clarified norm_header/header_edit -- disallow update of loaded theories;
2011-08-24, by wenzelm
misc tuning and simplification;
2011-08-24, by wenzelm
ignore irrelevant timings;
2011-08-24, by wenzelm
print state only for visible command, to avoid wasting resources for the larger part of the text;
2011-08-24, by wenzelm
early filtering of unchanged perspective;
2011-08-24, by wenzelm
more reliable update_perspective handler based on actual text visibility (e.g. on startup or when resizing without scrolling);
2011-08-24, by wenzelm
update_perspective without actual edits, bypassing the full state assignment protocol;
2011-08-24, by wenzelm
tuned;
2011-08-23, by wenzelm
handle potentially more approriate BufferUpdate.LOADED event;
2011-08-23, by wenzelm
special treatment of structure index 1 in Pure, including legacy warning;
2011-08-22, by wenzelm
compile
2011-08-23, by blanchet
added "max_calls" option to get a fixed number of Sledgehammer calls per theory
2011-08-23, by blanchet
beef up "sledgehammer_tac" reconstructor
2011-08-23, by blanchet
clean up Sledgehammer tactic
2011-08-23, by blanchet
fixed document;
2011-08-23, by wenzelm
tuned signature;
2011-08-23, by wenzelm
merged
2011-08-23, by wenzelm
always use TFF if possible
2011-08-23, by blanchet
clearer separator in generated file names
2011-08-23, by blanchet
exploit TFF format in Z3 used as ATP, and renamed it "z3_tptp"
2011-08-23, by blanchet
updated known failures for Z3 3.0 TPTP
2011-08-23, by blanchet
updated Z3 docs
2011-08-23, by blanchet
avoid TFF format with older Vampire versions
2011-08-23, by blanchet
update the Vampire related parts of the documentation
2011-08-23, by blanchet
fixed TFF slicing
2011-08-23, by blanchet
kindly ask Vampire to output axiom names
2011-08-23, by blanchet
added formats to the slice and use TFF for remote Vampire
2011-08-23, by blanchet
tuned specifications, syntax and proofs
2011-08-23, by haftmann
tuned specifications and syntax
2011-08-22, by haftmann
Quotient Package: some infrastructure for lifting inside sets
2011-08-23, by Cezary Kaliszyk
include all encodings in tests, now that the incompleteness of some encodings has been addressed
2011-08-22, by blanchet
change Metis's default settings if type information axioms are generated
2011-08-22, by blanchet
we must tag any type whose ground types intersect a nonmonotonic type
2011-08-22, by blanchet
prefer the lighter, slightly unsound monotonicity-based encodings for Metis
2011-08-22, by blanchet
made reconstruction of type tag equalities "\?x = \?x" reliable
2011-08-22, by blanchet
tuning ATP problem output
2011-08-22, by blanchet
revert guard logic -- make sure that typing information is generated for existentials
2011-08-22, by blanchet
generate tag equations for existential variables
2011-08-22, by blanchet
tuning, plus started implementing tag equation generation for existential variables
2011-08-22, by blanchet
precisely distinguish between universal and existential quantifiers, instead of assuming the worst (universal), for monotonicity analysis
2011-08-22, by blanchet
clearer terminology
2011-08-22, by blanchet
renamed "heavy" to "uniform", based on discussion with Nick Smallbone
2011-08-22, by blanchet
removed unused configuration option
2011-08-22, by blanchet
added caching for (in)finiteness checks
2011-08-22, by blanchet
remove needless typing information
2011-08-22, by blanchet
cleaner handling of polymorphic monotonicity inference
2011-08-22, by blanchet
started cleaning up polymorphic monotonicity-based encodings, based on discussions with Nick Smallbone
2011-08-22, by blanchet
more precise warning
2011-08-22, by blanchet
added option to control soundness of encodings more precisely, for evaluation purposes
2011-08-22, by blanchet
make sound mode more sound (and clean up code)
2011-08-22, by blanchet
reintroduced slightly unsound optimization taken out in 717880e98e6b, but only if "sound" is false
2011-08-22, by blanchet
gracefully handle empty SPASS problems
2011-08-22, by blanchet
pass sound option to Sledgehammer tactic
2011-08-22, by blanchet
tuned signature -- contrast physical output primitives versus Output.raw_message;
2011-08-23, by wenzelm
tuned signature;
2011-08-23, by wenzelm
discontinued slightly odd Future/Lazy.get_finished, which do not really fit into the execution model of Future.cancel/join_tasks (canceled tasks need to be dequeued and terminated explicitly);
2011-08-23, by wenzelm
some support for toplevel printing wrt. editor perspective (still inactive);
2011-08-23, by wenzelm
propagate editor perspective through document model;
2011-08-23, by wenzelm
some support for editor perspective;
2011-08-22, by wenzelm
discontinued redundant Edit_Command_ID;
2011-08-22, by wenzelm
reduced warnings;
2011-08-22, by wenzelm
tuned message;
2011-08-22, by wenzelm
less
more
|
(0)
-30000
-10000
-3000
-1000
-960
+960
+1000
+3000
+10000
+30000
tip