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.
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
less
more
|
(0)
-30000
-10000
-3000
-1000
-120
+120
+1000
+3000
+10000
+30000
tip