Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-480
+480
+1000
+3000
+10000
+30000
tip
Find changesets by keywords (author, files, the commit message), revision number or hash, or
revset expression
.
The revision graph only works with JavaScript-enabled browsers.
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
less
more
|
(0)
-30000
-10000
-3000
-1000
-480
+480
+1000
+3000
+10000
+30000
tip