Mercurial
Mercurial
>
repos
>
isabelle
/ graph
summary
|
shortlog
|
changelog
| graph |
tags
|
bookmarks
|
branches
|
files
|
gz
|
help
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+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.
updated Sign.add_type, Name_Space.declare;
2012-03-28, by wenzelm
updated comments;
2012-03-28, by wenzelm
merged
2012-03-28, by huffman
remove unnecessary rules from the simpset
2012-03-27, by huffman
remove unused premises
2012-03-27, by huffman
remove duplicate lemmas
2012-03-27, by huffman
mark some duplicate lemmas for deletion
2012-03-27, by huffman
remove more redundant lemmas
2012-03-27, by huffman
tuned proofs
2012-03-27, by huffman
remove redundant lemmas
2012-03-27, by huffman
generalized lemma zpower_zmod
2012-03-27, by huffman
remove redundant lemma
2012-03-27, by huffman
remove redundant lemma
2012-03-27, by huffman
remove duplicate [algebra] declarations
2012-03-27, by huffman
generalize more div/mod lemmas
2012-03-27, by huffman
generalize some theorems about div/mod
2012-03-27, by huffman
updated to jedit-4.5.1;
2012-03-28, by wenzelm
merged
2012-03-27, by kuncar
note a code eqn in quotient_def
2012-03-27, by kuncar
dropped support for List.distinct in binding to SMT solvers: only few applications benefited from this support, and in some cases the smt method fails due to its support for List.distinct
2012-03-27, by boehmes
more robustness in case a theorem cannot be retrieved (which typically happens with backtick facts)
2012-03-27, by blanchet
fixed eta-extension of higher-order quantifiers in THF output
2012-03-27, by blanchet
renamed "smt_fixed" to "smt_read_only_certificates"
2012-03-27, by blanchet
tuning
2012-03-27, by blanchet
tuning (in particular, Symtab instead of AList)
2012-03-27, by blanchet
tweak slices, based on eval by Daniel Wand
2012-03-27, by blanchet
be less forceful about ":lt" to make infinite loops less likely (could still fail with mutually recursive tail rec functions)
2012-03-27, by blanchet
print a hint
2012-03-27, by blanchet
avoid DL
2012-03-27, by blanchet
TFF: declare free types as types
2012-03-27, by blanchet
merged
2012-03-27, by bulwahn
association lists with distinct keys uses the quotient infrastructure to obtain code certificates;
2012-03-27, by bulwahn
remove redundant lemmas
2012-03-27, by huffman
move int::ring_div instance upward, simplify several proofs
2012-03-27, by huffman
rename lemmas {divmod_int_rel_{div,mod} -> {div,mod}_int_unique, for consistency with nat lemma names
2012-03-27, by huffman
extend definition of divmod_int_rel to handle denominator=0 case
2012-03-27, by huffman
tuned proofs
2012-03-27, by huffman
shorten a proof
2012-03-27, by huffman
simplify some proofs
2012-03-27, by huffman
rename lemmas {div,mod}_eq -> {div,mod}_nat_unique, for consistency with minus_unique, inverse_unique, etc.
2012-03-27, by huffman
simplify some proofs
2012-03-27, by huffman
merged
2012-03-26, by wenzelm
merged
2012-03-26, by nipkow
reverted to canonical name
2012-03-26, by nipkow
merged
2012-03-26, by wenzelm
merged
2012-03-26, by huffman
revert changeset 500a5d97511a, re-enabling HOL-Proofs-Lambda
2012-03-26, by huffman
merged
2012-03-26, by huffman
fix incorrect code_modulename declarations
2012-03-26, by huffman
code lemma for function 'nat' that doesn't go into an infinite loop (fixes problem with non-terminating HOL-Proofs-Lambda)
2012-03-26, by huffman
remove old-style semicolon
2012-03-26, by huffman
merged
2012-03-26, by nipkow
Functions and lemmas by Christian Sternagel
2012-03-26, by nipkow
more precise treatment of \r\n as blank symbol (cf. 2bf29095d26f), e.g. relevant for loading theory headers in Isabelle/jEdit -- NB: jEdit and Isabelle/ML normalize newline variants to \n, but Isabelle/Scala retains them literally;
2012-03-26, by wenzelm
disabled HOL-Proofs-Lambda temporarily, which causes problems with 2a1953f0d20d;
2012-03-26, by wenzelm
tuned comment
2012-03-26, by kuncar
merged
2012-03-26, by kuncar
merged
2012-03-26, by kuncar
tuned proof - no smt call
2012-03-26, by kuncar
more robust command invocation via ISABELLE_JDK_HOME or SCALA_HOME (NB: bash exec requires genuine executable, not function);
2012-03-26, by wenzelm
updated theory header syntax and related details;
2012-03-26, by wenzelm
ISABELLE_JDK_HOME settings variable points to JDK with javac and jar (not just JRE);
2012-03-24, by wenzelm
merged
2012-03-26, by wenzelm
reintroduced broken proofs and regenerated certificates
2012-03-26, by blanchet
merged, resolving trivial conflict;
2012-03-26, by wenzelm
fixed Nitpick after numeral representation change (2a1953f0d20d)
2012-03-26, by blanchet
merged fork with new numeral representation (see NEWS)
2012-03-25, by huffman
merged
2012-03-24, by kuncar
use Thm.transfer for thms stored in generic context data storage
2012-03-23, by kuncar
hide invariant constant
2012-03-23, by kuncar
explicit SMTP server (appears to be required after recent change of system configuration);
2012-03-24, by wenzelm
more isatest subscribers;
2012-03-24, by wenzelm
merged
2012-03-23, by paulson
proof tidying
2012-03-23, by paulson
updated comment
2012-01-16, by kuncar
resolve invariant constant name clash
2012-03-23, by kuncar
update etc/isar-keywords.el
2012-03-23, by kuncar
fix example files
2012-03-23, by kuncar
generation of a code certificate from a respectfulness theorem for constants lifted by the quotient_definition command & setup_lifting command: setups Quotient infrastructure from a typedef theorem
2012-03-23, by kuncar
simplified code of generation of aggregate relations
2012-03-23, by kuncar
store the relational theorem for every relator
2012-03-23, by kuncar
store the quotient theorem for every quotient
2012-03-23, by kuncar
fix Quotient_Examples
2012-03-23, by kuncar
respectfulness theorem has to be proved if a new constant is lifted by quotient_definition
2012-03-23, by kuncar
adjusting to longer names in PNF_Narrowing_Engine, which was overlooked in 4106258260b3
2012-03-23, by bulwahn
tuned;
2012-03-23, by wenzelm
merged;
2012-03-22, by wenzelm
fixed typo
2012-03-22, by haftmann
more instructive NEWS
2012-03-22, by haftmann
more structured proofs
2012-03-22, by paulson
New Message
2012-03-22, by paulson
No longer treat "title" as FDL keyword
2012-03-22, by berghofe
tuned proofs;
2012-03-22, by wenzelm
uniform Generic_Target.standard_declaration, which uses the standard morphism for each context (NB: targets like "interpretation" appear like "theory" but declare local type parameters);
2012-03-22, by wenzelm
tuned;
2012-03-22, by wenzelm
synchronize syntax uniformly for target stack and aux. context;
2012-03-22, by wenzelm
tuned;
2012-03-22, by wenzelm
merged
2012-03-21, by wenzelm
removed Satallax option, now that this is the default
2012-03-21, by blanchet
doc update
2012-03-21, by blanchet
improve "remote_satallax" by exploiting unsat core
2012-03-21, by blanchet
generate weights and precedences for predicates as well
2012-03-21, by blanchet
refinements to constructibility
2012-03-21, by paulson
More structured proofs for infinite cardinalities
2012-03-21, by paulson
actually expose target context;
2012-03-21, by wenzelm
more explicit Toplevel.open_target/close_target;
2012-03-21, by wenzelm
tuned signature;
2012-03-21, by wenzelm
optional 'includes' element for long theorem statements;
2012-03-21, by wenzelm
basic support for nested contexts including bundles;
2012-03-21, by wenzelm
tuned messages;
2012-03-21, by wenzelm
basic support for nested local theory targets;
2012-03-21, by wenzelm
try apple.laf.useScreenMenuBar=false to make menus stay closer to the editor views they belong to -- potentially less confusing for jEdit newcomers;
2012-03-21, by wenzelm
improved isatest arguments for macbroy2;
2012-03-21, by wenzelm
clarified Local_Theory.init: avoid hardwired naming policy, discontinued odd/unused group argument (cf. 5ee13e0428d2);
2012-03-21, by wenzelm
prefer explicitly qualified exception List.Empty;
2012-03-21, by wenzelm
merged
2012-03-20, by wenzelm
refined init_model: allow change of buffer name as caused by "Save as", for example;
2012-03-20, by wenzelm
basic support for bundled declarations;
2012-03-20, by wenzelm
doc update
2012-03-20, by blanchet
made "spass" a "metaprover" that uses either the new SPASS or the old SPASS, to preserve backward compatibility and prepare for the upcoming release
2012-03-20, by blanchet
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip