| author | wenzelm | 
| Sun, 23 May 2021 18:04:35 +0200 | |
| changeset 73768 | c73c22c62d08 | 
| parent 73526 | a3cc9fa1295d | 
| child 73935 | 269b2f976100 | 
| permissions | -rw-r--r-- | 
| 24799 | 1 | For the purposes of the license agreement in the file COPYRIGHT, a | 
| 62098 | 2 | 'contributor' is anybody who is listed in this file (CONTRIBUTORS) or who is | 
| 3 | listed as an author in one of the source files of this Isabelle distribution. | |
| 4 | ||
| 23382 | 5 | |
| 73126 | 6 | Contributions to this Isabelle version | 
| 7 | -------------------------------------- | |
| 8 | ||
| 73526 
a3cc9fa1295d
new automatic order prover: stateless, complete, verified
 nipkow parents: 
73477diff
changeset | 9 | * March 2021: Lukas Stevens | 
| 
a3cc9fa1295d
new automatic order prover: stateless, complete, verified
 nipkow parents: 
73477diff
changeset | 10 | New order prover | 
| 
a3cc9fa1295d
new automatic order prover: stateless, complete, verified
 nipkow parents: 
73477diff
changeset | 11 | |
| 73477 | 12 | * March 2021: Florian Haftmann | 
| 13 | Dedicated session for combinatorics. | |
| 14 | ||
| 73455 | 15 | * March 2021: Simon Foster and Leo Freitas | 
| 16 | More symbol definitions for Z Notation: Isabelle fonts and LaTeX macros. | |
| 73446 
d1c4c2395650
more Isabelle symbol definitions for Z Notation, based on https://github.com/isabelle-utp/Z_Toolkit 998c9f7880d3 by Simon Foster;
 wenzelm parents: 
73253diff
changeset | 17 | |
| 73253 
f6bb31879698
HOL-Analysis/Probability: Hoeffding's inequality, negative binomial distribution, etc.
 Manuel Eberl <eberlm@in.tum.de> parents: 
73213diff
changeset | 18 | * February 2021: Manuel Eberl | 
| 
f6bb31879698
HOL-Analysis/Probability: Hoeffding's inequality, negative binomial distribution, etc.
 Manuel Eberl <eberlm@in.tum.de> parents: 
73213diff
changeset | 19 | New material in HOL-Analysis/HOL-Probability, most notably Hoeffding's | 
| 
f6bb31879698
HOL-Analysis/Probability: Hoeffding's inequality, negative binomial distribution, etc.
 Manuel Eberl <eberlm@in.tum.de> parents: 
73213diff
changeset | 20 | inequality and the negative binomial distribution | 
| 
f6bb31879698
HOL-Analysis/Probability: Hoeffding's inequality, negative binomial distribution, etc.
 Manuel Eberl <eberlm@in.tum.de> parents: 
73213diff
changeset | 21 | |
| 73127 
4c4d479b097d
new magerial from Jakub Kądziołka
 paulson <lp15@cam.ac.uk> parents: 
73126diff
changeset | 22 | * January 2021: Jakub Kądziołka | 
| 
4c4d479b097d
new magerial from Jakub Kądziołka
 paulson <lp15@cam.ac.uk> parents: 
73126diff
changeset | 23 | Some lemmas for HOL-Computational_Algebra. | 
| 
4c4d479b097d
new magerial from Jakub Kądziołka
 paulson <lp15@cam.ac.uk> parents: 
73126diff
changeset | 24 | |
| 73213 
bb35f7f60d6c
contributors
 Andreas Lochbihler <mail@andreas-lochbihler.de> parents: 
73183diff
changeset | 25 | * January 2021: Martin Rasyzk | 
| 
bb35f7f60d6c
contributors
 Andreas Lochbihler <mail@andreas-lochbihler.de> parents: 
73183diff
changeset | 26 | Fast set operations for red-black trees. | 
| 73126 | 27 | |
| 73446 
d1c4c2395650
more Isabelle symbol definitions for Z Notation, based on https://github.com/isabelle-utp/Z_Toolkit 998c9f7880d3 by Simon Foster;
 wenzelm parents: 
73253diff
changeset | 28 | |
| 72972 | 29 | Contributions to Isabelle2021 | 
| 30 | ----------------------------- | |
| 72971 
162b71f7e554
rebuild component with proper ZIPPERPOSITION_HOME for sledgehammer;
 wenzelm parents: 
72806diff
changeset | 31 | |
| 73108 
981a383610df
HOL-Data_Structures: added Selection and time functions for list functions
 Manuel Eberl <eberlm@in.tum.de> parents: 
73079diff
changeset | 32 | * January 2021: Manuel Eberl | 
| 73124 | 33 | Characteristic of a semiring. | 
| 73108 
981a383610df
HOL-Data_Structures: added Selection and time functions for list functions
 Manuel Eberl <eberlm@in.tum.de> parents: 
73079diff
changeset | 34 | |
| 
981a383610df
HOL-Data_Structures: added Selection and time functions for list functions
 Manuel Eberl <eberlm@in.tum.de> parents: 
73079diff
changeset | 35 | * January 2021: Manuel Eberl | 
| 73124 | 36 | Algebraic integers in HOL-Computational_Algebra. | 
| 73108 
981a383610df
HOL-Data_Structures: added Selection and time functions for list functions
 Manuel Eberl <eberlm@in.tum.de> parents: 
73079diff
changeset | 37 | |
| 73018 | 38 | * December 2020: Stepan Holub | 
| 73079 | 39 | Contributed lemmas for theory HOL.List. | 
| 73018 | 40 | |
| 72971 
162b71f7e554
rebuild component with proper ZIPPERPOSITION_HOME for sledgehammer;
 wenzelm parents: 
72806diff
changeset | 41 | * December 2020: Martin Desharnais | 
| 72972 | 42 | Zipperposition 2.0 as external prover for Sledgehammer. | 
| 72971 
162b71f7e554
rebuild component with proper ZIPPERPOSITION_HOME for sledgehammer;
 wenzelm parents: 
72806diff
changeset | 43 | |
| 72972 | 44 | * December 2020: Walter Guttmann | 
| 45 | Extension of session HOL-Hoare with total correctness proof system. | |
| 72806 
4fa08e083865
Extension of session HOL/Hoare with total correctness proof system by Walter Guttmann
 nipkow parents: 
72732diff
changeset | 46 | |
| 73007 | 47 | * November / December 2020: Makarius Wenzel | 
| 48 | Improved HTML presentation and PDF document preparation, using mostly | |
| 49 | Isabelle/Scala instead of Isabelle/ML. | |
| 50 | ||
| 72732 | 51 | * November 2020: Stepan Holub | 
| 72972 | 52 | Removed preconditions from lemma comm_append_are_replicate. | 
| 71557 | 53 | |
| 72606 | 54 | * November 2020: Florian Haftmann | 
| 55 | Bundle mixins for locale and class expressions. | |
| 56 | ||
| 72630 
4167d3d3d478
Jakub Kądziołka's stronger version of generate_pow_card (required some restructuring)
 paulson <lp15@cam.ac.uk> parents: 
72606diff
changeset | 57 | * November 2020: Jakub Kądziołka | 
| 72972 | 58 | Stronger lemmas about orders of group elements (generate_pow_card). | 
| 72630 
4167d3d3d478
Jakub Kądziołka's stronger version of generate_pow_card (required some restructuring)
 paulson <lp15@cam.ac.uk> parents: 
72606diff
changeset | 59 | |
| 72518 
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
 desharna parents: 
72495diff
changeset | 60 | * October 2020: Jasmin Blanchette, Martin Desharnais, Mathias Fleury | 
| 72972 | 61 | Support veriT as external prover in Sledgehammer. | 
| 72518 
4be6ae020fc4
Added smt (verit) to Sledgehammer's proof preplay.
 desharna parents: 
72495diff
changeset | 62 | |
| 72478 
b452242dce36
proper Isabelle component settings: prefer standard terminology "ISABELLE_VERIT", avoid conflict of "VERIT_VERSION" with processing of implicit options by veriT;
 wenzelm parents: 
72292diff
changeset | 63 | * October 2020: Mathias Fleury | 
| 
b452242dce36
proper Isabelle component settings: prefer standard terminology "ISABELLE_VERIT", avoid conflict of "VERIT_VERSION" with processing of implicit options by veriT;
 wenzelm parents: 
72292diff
changeset | 64 | Updated proof reconstruction for the SMT solver veriT in the smt method. | 
| 
b452242dce36
proper Isabelle component settings: prefer standard terminology "ISABELLE_VERIT", avoid conflict of "VERIT_VERSION" with processing of implicit options by veriT;
 wenzelm parents: 
72292diff
changeset | 65 | |
| 72495 | 66 | * October 2020: Jasmin Blanchette, Martin Desharnais | 
| 72972 | 67 | Support E prover 2.5 as external prover in Sledgehammer. | 
| 72495 | 68 | |
| 72606 | 69 | * September 2020: Florian Haftmann | 
| 73007 | 70 | Substantial reworking and modularization of Word library, with generic type | 
| 71 | conversions. | |
| 72 | ||
| 73 | * August 2020: Makarius Wenzel | |
| 74 | Finally enable PIDE protocol for batch-builds, with various consequences of | |
| 75 | handling session build databases, Isabelle/Scala within Isabelle/ML etc. | |
| 72606 | 76 | |
| 72150 | 77 | * August 2020: Makarius Wenzel | 
| 78 | Improved monitoring of runtime statistics: ML GC progress and Java. | |
| 79 | ||
| 72004 | 80 | * July 2020: Martin Desharnais | 
| 72972 | 81 | Update to Metis 2.4. | 
| 72004 | 82 | |
| 71980 | 83 | * June 2020: Makarius Wenzel | 
| 72103 | 84 | Batch-builds via "isabelle build" allow to invoke Scala from ML. | 
| 71980 | 85 | |
| 72606 | 86 | * June 2020: Florian Haftmann | 
| 87 | Simproc defined_all for more aggressive substitution with variables | |
| 88 | from assumptions. | |
| 89 | ||
| 71980 | 90 | * May 2020: Makarius Wenzel | 
| 91 |   Antiquotations for Isabelle systems programming, notably @{scala_function}
 | |
| 92 |   and @{scala} to invoke Scala from ML.
 | |
| 93 | ||
| 71956 | 94 | * May 2020: Florian Haftmann | 
| 71957 
3e162c63371a
build bit operations on word on library theory on bit operations
 haftmann parents: 
71956diff
changeset | 95 | Generic algebraically founded bit operations NOT, AND, OR, XOR. | 
| 71956 | 96 | |
| 71557 | 97 | |
| 71485 | 98 | Contributions to Isabelle2020 | 
| 99 | ----------------------------- | |
| 71431 | 100 | |
| 71437 | 101 | * February 2020: E. Gunther, M. Pagano and P. Sánchez Terraf | 
| 102 | Simplified, generalised version of ZF/Constructible. | |
| 103 | ||
| 104 | * January 2020: LC Paulson | |
| 105 | The full finite Ramsey's theorem and elements of finite and infinite | |
| 106 | Ramsey theory. | |
| 70265 | 107 | |
| 71438 | 108 | * December 2019: Basil Fürer, Andreas Lochbihler, Joshua Schneider, Dmitriy | 
| 109 | Traytel | |
| 71264 | 110 | Extension of lift_bnf to support quotient types. | 
| 111 | ||
| 71473 
be84312a2d53
update to WebviewPanel API, following initial version by Peter Zeller;
 wenzelm parents: 
71438diff
changeset | 112 | * November 2019: Peter Zeller, TU Kaiserslautern | 
| 
be84312a2d53
update to WebviewPanel API, following initial version by Peter Zeller;
 wenzelm parents: 
71438diff
changeset | 113 | Update of Isabelle/VSCode to WebviewPanel API. | 
| 
be84312a2d53
update to WebviewPanel API, following initial version by Peter Zeller;
 wenzelm parents: 
71438diff
changeset | 114 | |
| 71438 | 115 | * October..December 2019: Makarius Wenzel | 
| 116 | Isabelle/Phabrictor server setup, including Linux platform support in | |
| 117 | Isabelle/Scala. Client-side tool "isabelle hg_setup". | |
| 118 | ||
| 70955 | 119 | * October 2019: Maximilian Schäffeler | 
| 120 | Port of the HOL Light decision procedure for metric spaces. | |
| 70265 | 121 | |
| 71437 | 122 | * October 2019: Makarius Wenzel | 
| 123 | More scalable Isabelle dump and underlying headless PIDE session. | |
| 71435 
d8fb621fea02
some lemmas about the lex ordering on lists, etc.
 paulson <lp15@cam.ac.uk> parents: 
71431diff
changeset | 124 | |
| 71438 | 125 | * August 2019: Makarius Wenzel | 
| 126 | Better support for proof terms in Isabelle/Pure, notably via method | |
| 127 | combinator SUBPROOFS (ML) and "subproofs" (Isar). | |
| 128 | ||
| 71436 | 129 | * July 2019: Alexander Krauss, Makarius Wenzel | 
| 130 | Minimal support for a soft-type system within the Isabelle logical | |
| 131 | framework. | |
| 132 | ||
| 71435 
d8fb621fea02
some lemmas about the lex ordering on lists, etc.
 paulson <lp15@cam.ac.uk> parents: 
71431diff
changeset | 133 | |
| 70024 | 134 | Contributions to Isabelle2019 | 
| 135 | ----------------------------- | |
| 69814 | 136 | |
| 70164 
1f163f772da3
Group theory developments towards proving algebraic closure (by de Vilhena and Baillon)
 paulson <lp15@cam.ac.uk> parents: 
70024diff
changeset | 137 | * April 2019: LC Paulson | 
| 
1f163f772da3
Group theory developments towards proving algebraic closure (by de Vilhena and Baillon)
 paulson <lp15@cam.ac.uk> parents: 
70024diff
changeset | 138 | Homology and supporting lemmas on topology and group theory | 
| 
1f163f772da3
Group theory developments towards proving algebraic closure (by de Vilhena and Baillon)
 paulson <lp15@cam.ac.uk> parents: 
70024diff
changeset | 139 | |
| 
1f163f772da3
Group theory developments towards proving algebraic closure (by de Vilhena and Baillon)
 paulson <lp15@cam.ac.uk> parents: 
70024diff
changeset | 140 | * April 2019: Paulo de Vilhena and Martin Baillon | 
| 70216 | 141 | Group theory developments, esp. algebraic closure of a field | 
| 70164 
1f163f772da3
Group theory developments towards proving algebraic closure (by de Vilhena and Baillon)
 paulson <lp15@cam.ac.uk> parents: 
70024diff
changeset | 142 | |
| 70024 | 143 | * February/March 2019: Makarius Wenzel | 
| 144 | Stateless management of export artifacts in the Isabelle/HOL code generator. | |
| 69791 
195aeee8b30a
Formal Laurent series and overhaul of Formal power series (due to Jeremy Sylvestre)
 Manuel Eberl <eberlm@in.tum.de> parents: 
69790diff
changeset | 145 | |
| 69785 
9e326f6f8a24
More material for HOL-Number_Theory: ord, Carmichael's function, primitive roots
 Manuel Eberl <eberlm@in.tum.de> parents: 
69568diff
changeset | 146 | * February 2019: Manuel Eberl | 
| 69790 
154cf64e403e
Exponentiation by squaring, fast modular exponentiation
 Manuel Eberl <eberlm@in.tum.de> parents: 
69785diff
changeset | 147 | Exponentiation by squaring, used to implement "power" in monoid_mult and | 
| 
154cf64e403e
Exponentiation by squaring, fast modular exponentiation
 Manuel Eberl <eberlm@in.tum.de> parents: 
69785diff
changeset | 148 | fast modular exponentiation. | 
| 
154cf64e403e
Exponentiation by squaring, fast modular exponentiation
 Manuel Eberl <eberlm@in.tum.de> parents: 
69785diff
changeset | 149 | |
| 
154cf64e403e
Exponentiation by squaring, fast modular exponentiation
 Manuel Eberl <eberlm@in.tum.de> parents: 
69785diff
changeset | 150 | * February 2019: Manuel Eberl | 
| 70024 | 151 | Carmichael's function, primitive roots in residue rings, more properties of | 
| 152 | the order in residue rings. | |
| 153 | ||
| 154 | * February 2019: Jeremy Sylvestre | |
| 155 | Formal Laurent Series and overhaul of Formal power series. | |
| 156 | ||
| 157 | * January 2019: Florian Haftmann | |
| 158 | Clarified syntax and congruence rules for big operators on sets involving | |
| 159 | the image operator. | |
| 160 | ||
| 161 | * January 2019: Florian Haftmann | |
| 162 | Renovation of code generation, particularly export into session data and | |
| 163 | proper strings and proper integers based on zarith for OCaml. | |
| 69785 
9e326f6f8a24
More material for HOL-Number_Theory: ord, Carmichael's function, primitive roots
 Manuel Eberl <eberlm@in.tum.de> parents: 
69568diff
changeset | 164 | |
| 69568 
de09a7261120
new implementation for case_of_simps based on Code_Lazy's pattern matching elimination algorithm
 Andreas Lochbihler parents: 
69205diff
changeset | 165 | * January 2019: Andreas Lochbihler | 
| 70024 | 166 | New implementation for case_of_simps based on Code_Lazy's pattern matching | 
| 167 | elimination algorithm. | |
| 168 | ||
| 169 | * November/December 2018: Makarius Wenzel | |
| 170 | Support for Isabelle/Haskell applications of Isabelle/PIDE. | |
| 171 | ||
| 172 | * August/September 2018: Makarius Wenzel | |
| 173 | Improvements of headless Isabelle/PIDE session and server, and systematic | |
| 174 | exports from theory documents. | |
| 69568 
de09a7261120
new implementation for case_of_simps based on Code_Lazy's pattern matching elimination algorithm
 Andreas Lochbihler parents: 
69205diff
changeset | 175 | |
| 69814 | 176 | * December 2018: Florian Haftmann | 
| 177 | Generic executable sorting algorithms based on executable comparators. | |
| 178 | ||
| 69205 
8050734eee3e
add reconstruction by veriT in method smt
 fleury <Mathias.Fleury@mpi-inf.mpg.de> parents: 
68683diff
changeset | 179 | * October 2018: Mathias Fleury | 
| 69814 | 180 | Proof reconstruction for the SMT solver veriT in the smt method. | 
| 69205 
8050734eee3e
add reconstruction by veriT in method smt
 fleury <Mathias.Fleury@mpi-inf.mpg.de> parents: 
68683diff
changeset | 181 | |
| 68683 | 182 | |
| 68391 | 183 | Contributions to Isabelle2018 | 
| 184 | ----------------------------- | |
| 66651 | 185 | |
| 68630 | 186 | * July 2018: Manuel Eberl | 
| 187 | "real_asymp" proof method for automatic proofs of real limits, "Big-O" | |
| 188 | statements, etc. | |
| 189 | ||
| 68522 
d9cbc1e8644d
example for Types_To_Sets: transfer from type-based linear algebra to subspaces
 immler parents: 
68466diff
changeset | 190 | * June 2018: Fabian Immler | 
| 
d9cbc1e8644d
example for Types_To_Sets: transfer from type-based linear algebra to subspaces
 immler parents: 
68466diff
changeset | 191 | More tool support for HOL-Types_To_Sets. | 
| 
d9cbc1e8644d
example for Types_To_Sets: transfer from type-based linear algebra to subspaces
 immler parents: 
68466diff
changeset | 192 | |
| 68466 | 193 | * June 2018: Martin Baillon and Paulo Emílio de Vilhena | 
| 194 | A variety of contributions to HOL-Algebra. | |
| 195 | ||
| 68532 
f8b98d31ad45
Incorporating new/strengthened proofs from Library and AFP entries
 paulson <lp15@cam.ac.uk> parents: 
68522diff
changeset | 196 | * June 2018: Wenda Li | 
| 
f8b98d31ad45
Incorporating new/strengthened proofs from Library and AFP entries
 paulson <lp15@cam.ac.uk> parents: 
68522diff
changeset | 197 | New/strengthened results involving analysis, topology, etc. | 
| 
f8b98d31ad45
Incorporating new/strengthened proofs from Library and AFP entries
 paulson <lp15@cam.ac.uk> parents: 
68522diff
changeset | 198 | |
| 68545 | 199 | * May/June 2018: Makarius Wenzel | 
| 200 | System infrastructure to export blobs as theory presentation, and to dump | |
| 201 | PIDE database content in batch mode. | |
| 202 | ||
| 68246 
b48bab511939
Moved Landau_Symbols from the AFP to HOL-Library
 Manuel Eberl <eberlm@in.tum.de> parents: 
68200diff
changeset | 203 | * May 2018: Manuel Eberl | 
| 68391 | 204 | Landau symbols and asymptotic equivalence (moved from the AFP). | 
| 68246 
b48bab511939
Moved Landau_Symbols from the AFP to HOL-Library
 Manuel Eberl <eberlm@in.tum.de> parents: 
68200diff
changeset | 205 | |
| 68073 
fad29d2a17a5
merged; resolved conflicts manually (esp. lemmas that have been moved from Linear_Algebra and Cartesian_Euclidean_Space)
 immlerdiff
changeset | 206 | * May 2018: Jose Divasón (Universidad de la Rioja), | 
| 68072 
493b818e8e10
added Johannes' generalizations Modules.thy and Vector_Spaces.thy; adapted HOL and HOL-Analysis accordingly
 immler parents: 
67928diff
changeset | 207 | Jesús Aransay (Universidad de la Rioja), Johannes Hölzl (VU Amsterdam), | 
| 
493b818e8e10
added Johannes' generalizations Modules.thy and Vector_Spaces.thy; adapted HOL and HOL-Analysis accordingly
 immler parents: 
67928diff
changeset | 208 | Fabian Immler (TUM) | 
| 
493b818e8e10
added Johannes' generalizations Modules.thy and Vector_Spaces.thy; adapted HOL and HOL-Analysis accordingly
 immler parents: 
67928diff
changeset | 209 | Generalizations in the formalization of linear algebra. | 
| 
493b818e8e10
added Johannes' generalizations Modules.thy and Vector_Spaces.thy; adapted HOL and HOL-Analysis accordingly
 immler parents: 
67928diff
changeset | 210 | |
| 68028 | 211 | * May 2018: Florian Haftmann | 
| 212 | Consolidation of string-like types in HOL. | |
| 213 | ||
| 68200 
5859c688102a
NEWS and CONTRIBUTORS for 8b50f29a1992
 Andreas Lochbihler parents: 
68073diff
changeset | 214 | * May 2018: Andreas Lochbihler (Digital Asset), | 
| 
5859c688102a
NEWS and CONTRIBUTORS for 8b50f29a1992
 Andreas Lochbihler parents: 
68073diff
changeset | 215 | Pascal Stoop (ETH Zurich) | 
| 
5859c688102a
NEWS and CONTRIBUTORS for 8b50f29a1992
 Andreas Lochbihler parents: 
68073diff
changeset | 216 | Code generation with lazy evaluation semantics. | 
| 
5859c688102a
NEWS and CONTRIBUTORS for 8b50f29a1992
 Andreas Lochbihler parents: 
68073diff
changeset | 217 | |
| 67928 | 218 | * March 2018: Florian Haftmann | 
| 68391 | 219 | Abstract bit operations push_bit, take_bit, drop_bit, alongside with an | 
| 220 | algebraic foundation for bit strings and word types in HOL-ex. | |
| 67928 | 221 | |
| 67831 
07f5588f2735
Removed stray 'sledgehammer' invocation
 Manuel Eberl <eberlm@in.tum.de> parents: 
67456diff
changeset | 222 | * March 2018: Viorel Preoteasa | 
| 
07f5588f2735
Removed stray 'sledgehammer' invocation
 Manuel Eberl <eberlm@in.tum.de> parents: 
67456diff
changeset | 223 | Generalisation of complete_distrib_lattice | 
| 
07f5588f2735
Removed stray 'sledgehammer' invocation
 Manuel Eberl <eberlm@in.tum.de> parents: 
67456diff
changeset | 224 | |
| 68531 | 225 | * February 2018: Wenda Li | 
| 68548 | 226 | A unified definition for the order of zeros and poles. Improved reasoning | 
| 227 | around non-essential singularities. | |
| 68531 | 228 | |
| 67456 | 229 | * January 2018: Sebastien Gouezel | 
| 230 | Various small additions to HOL-Analysis | |
| 231 | ||
| 67224 | 232 | * December 2017: Jan Gilcher, Andreas Lochbihler, Dmitriy Traytel | 
| 67279 | 233 | A new conditional parametricity prover. | 
| 67224 | 234 | |
| 66893 
ced164fe3bbd
derived axiom iffI as a lemma (thanks to Alexander Maletzky)
 nipkow parents: 
66651diff
changeset | 235 | * October 2017: Alexander Maletzky | 
| 68391 | 236 | Derivation of axiom "iff" in theory HOL.HOL from the other axioms. | 
| 237 | ||
| 66651 | 238 | |
| 66475 | 239 | Contributions to Isabelle2017 | 
| 66482 | 240 | ----------------------------- | 
| 64439 | 241 | |
| 66648 | 242 | * September 2017: Lawrence Paulson | 
| 243 | HOL-Analysis, e.g. simplicial complexes, Jordan Curve Theorem. | |
| 244 | ||
| 245 | * September 2017: Jasmin Blanchette | |
| 246 | Further integration of Nunchaku model finder. | |
| 247 | ||
| 66475 | 248 | * November 2016 - June 2017: Makarius Wenzel | 
| 249 | New Isabelle/VSCode, with underlying restructuring of Isabelle/PIDE. | |
| 250 | ||
| 251 | * 2017: Makarius Wenzel | |
| 252 | Session-qualified theory names (theory imports and ROOT files). | |
| 253 | Prover IDE improvements. | |
| 254 | Support for SQL databases in Isabelle/Scala: SQLite and PostgreSQL. | |
| 255 | ||
| 66563 | 256 | * August 2017: Andreas Lochbihler, ETH Zurich | 
| 257 | type of unordered pairs (HOL-Library.Uprod) | |
| 258 | ||
| 66480 
4b8d1df8933b
HOL-Analysis: Convergent FPS and infinite sums
 Manuel Eberl <eberlm@in.tum.de> parents: 
66475diff
changeset | 259 | * August 2017: Manuel Eberl, TUM | 
| 
4b8d1df8933b
HOL-Analysis: Convergent FPS and infinite sums
 Manuel Eberl <eberlm@in.tum.de> parents: 
66475diff
changeset | 260 | HOL-Analysis: infinite products over natural numbers, | 
| 
4b8d1df8933b
HOL-Analysis: Convergent FPS and infinite sums
 Manuel Eberl <eberlm@in.tum.de> parents: 
66475diff
changeset | 261 | infinite sums over arbitrary sets, connection between formal | 
| 
4b8d1df8933b
HOL-Analysis: Convergent FPS and infinite sums
 Manuel Eberl <eberlm@in.tum.de> parents: 
66475diff
changeset | 262 | power series and analytic complex functions | 
| 
4b8d1df8933b
HOL-Analysis: Convergent FPS and infinite sums
 Manuel Eberl <eberlm@in.tum.de> parents: 
66475diff
changeset | 263 | |
| 65330 | 264 | * March 2017: Alasdair Armstrong, University of Sheffield and | 
| 265 | Simon Foster, University of York | |
| 65099 
30d0b2f1df76
Knaster-Tarski fixed point theorem and Galois Connections.
 ballarin parents: 
65042diff
changeset | 266 | Fixed-point theory and Galois Connections in HOL-Algebra. | 
| 
30d0b2f1df76
Knaster-Tarski fixed point theorem and Galois Connections.
 ballarin parents: 
65042diff
changeset | 267 | |
| 65041 | 268 | * February 2017: Florian Haftmann, TUM | 
| 65042 | 269 | Statically embedded computations implemented by generated code. | 
| 65041 | 270 | |
| 64439 | 271 | |
| 64072 | 272 | Contributions to Isabelle2016-1 | 
| 273 | ------------------------------- | |
| 62216 | 274 | |
| 64551 | 275 | * December 2016: Ondřej Kunčar, TUM | 
| 276 | Types_To_Sets: experimental extension of Higher-Order Logic to allow | |
| 277 | translation of types to sets. | |
| 278 | ||
| 64393 | 279 | * October 2016: Jasmin Blanchette | 
| 280 | Integration of Nunchaku model finder. | |
| 281 | ||
| 282 | * October 2016: Jaime Mendizabal Roche, TUM | |
| 283 | Ported remaining theories of session Old_Number_Theory to the new | |
| 284 | Number_Theory and removed Old_Number_Theory. | |
| 285 | ||
| 286 | * September 2016: Sascha Boehme | |
| 287 | Proof method "argo" based on SMT technology for a combination of | |
| 288 | quantifier-free propositional logic, equality and linear real arithmetic | |
| 289 | ||
| 290 | * July 2016: Daniel Stuewe | |
| 291 | Height-size proofs in HOL-Data_Structures. | |
| 292 | ||
| 293 | * July 2016: Manuel Eberl, TUM | |
| 294 | Algebraic foundation for primes; generalization from nat to general | |
| 295 | factorial rings. | |
| 296 | ||
| 297 | * June 2016: Andreas Lochbihler, ETH Zurich | |
| 298 | Formalisation of discrete subprobability distributions. | |
| 299 | ||
| 300 | * June 2016: Florian Haftmann, TUM | |
| 301 | Improvements to code generation: optional timing measurements, more succint | |
| 302 | closures for static evaluation, less ambiguities concering Scala implicits. | |
| 303 | ||
| 304 | * May 2016: Manuel Eberl, TUM | |
| 305 | Code generation for Probability Mass Functions. | |
| 62343 
24106dc44def
prefer abbreviations for compound operators INFIMUM and SUPREMUM
 haftmann parents: 
62284diff
changeset | 306 | |
| 64011 | 307 | * March 2016: Florian Haftmann, TUM | 
| 62499 | 308 | Abstract factorial rings with unique factorization. | 
| 309 | ||
| 64011 | 310 | * March 2016: Florian Haftmann, TUM | 
| 64393 | 311 | Reworking of the HOL char type as special case of a finite numeral type. | 
| 62216 | 312 | |
| 64393 | 313 | * March 2016: Andreas Lochbihler, ETH Zurich | 
| 314 | Reasoning support for monotonicity, continuity and admissibility in | |
| 315 | chain-complete partial orders. | |
| 64011 | 316 | |
| 64393 | 317 | * February - October 2016: Makarius Wenzel | 
| 318 | Prover IDE improvements. | |
| 319 | ML IDE improvements: bootstrap of Pure. | |
| 320 | Isar language consolidation. | |
| 321 | Notational modernization of HOL. | |
| 322 | Tight Poly/ML integration. | |
| 323 | More Isabelle/Scala system programming modules (e.g. SSH, Mercurial). | |
| 63552 | 324 | |
| 64433 | 325 | * Winter 2016: Jasmin Blanchette, Inria & LORIA & MPII, Aymeric Bouzy, | 
| 326 | Ecole polytechnique, Andreas Lochbihler, ETH Zurich, Andrei Popescu, | |
| 327 | Middlesex University, and Dmitriy Traytel, ETH Zurich | |
| 328 | 'corec' command and friends. | |
| 329 | ||
| 64393 | 330 | * January 2016: Florian Haftmann, TUM | 
| 331 | Abolition of compound operators INFIMUM and SUPREMUM for complete lattices. | |
| 64389 | 332 | |
| 333 | ||
| 62016 | 334 | Contributions to Isabelle2016 | 
| 335 | ----------------------------- | |
| 60138 | 336 | |
| 62201 
eca7b38c8ee5
Added approximation of powr to NEWS/CONTRIBUTORS
 Manuel Eberl <eberlm@in.tum.de> parents: 
62138diff
changeset | 337 | * Winter 2016: Manuel Eberl, TUM | 
| 
eca7b38c8ee5
Added approximation of powr to NEWS/CONTRIBUTORS
 Manuel Eberl <eberlm@in.tum.de> parents: 
62138diff
changeset | 338 |   Support for real exponentiation ("powr") in the "approximation" method.
 | 
| 62693 | 339 | (This was removed in Isabelle 2015 due to a changed definition of "powr".) | 
| 62201 
eca7b38c8ee5
Added approximation of powr to NEWS/CONTRIBUTORS
 Manuel Eberl <eberlm@in.tum.de> parents: 
62138diff
changeset | 340 | |
| 62138 | 341 | * Summer 2015 - Winter 2016: Lawrence C Paulson, Cambridge | 
| 342 | General, homology form of Cauchy's integral theorem and supporting material | |
| 62205 | 343 | (ported from HOL Light). | 
| 62138 | 344 | |
| 62118 | 345 | * Winter 2015/16: Gerwin Klein, NICTA | 
| 62205 | 346 | New print_record command. | 
| 62118 | 347 | |
| 62236 | 348 | * May - December 2015: Makarius Wenzel | 
| 349 | Prover IDE improvements. | |
| 350 | More Isar language elements. | |
| 351 | Document language refinements. | |
| 352 | Poly/ML debugger integration. | |
| 353 | Improved multi-platform and multi-architecture support. | |
| 354 | ||
| 62060 
b75764fc4c35
Added summability/Gamma/etc. to NEWS and CONTRIBUTORS
 eberlm parents: 
62016diff
changeset | 355 | * Winter 2015: Manuel Eberl, TUM | 
| 
b75764fc4c35
Added summability/Gamma/etc. to NEWS and CONTRIBUTORS
 eberlm parents: 
62016diff
changeset | 356 | The radius of convergence of power series and various summability tests. | 
| 62064 | 357 | Harmonic numbers and the Euler-Mascheroni constant. | 
| 62060 
b75764fc4c35
Added summability/Gamma/etc. to NEWS and CONTRIBUTORS
 eberlm parents: 
62016diff
changeset | 358 | The Generalised Binomial Theorem. | 
| 62064 | 359 | The complex and real Gamma/log-Gamma/Digamma/Polygamma functions and their | 
| 360 | most important properties. | |
| 62138 | 361 | |
| 62086 
1c0246456ab9
Added formal power series updates to NEWS/CONTRIBUTORS
 Manuel Eberl <eberlm@in.tum.de> parents: 
62084diff
changeset | 362 | * Autumn 2015: Manuel Eberl, TUM | 
| 
1c0246456ab9
Added formal power series updates to NEWS/CONTRIBUTORS
 Manuel Eberl <eberlm@in.tum.de> parents: 
62084diff
changeset | 363 | Proper definition of division (with remainder) for formal power series; | 
| 
1c0246456ab9
Added formal power series updates to NEWS/CONTRIBUTORS
 Manuel Eberl <eberlm@in.tum.de> parents: 
62084diff
changeset | 364 | Euclidean Ring and GCD instance for formal power series. | 
| 62060 
b75764fc4c35
Added summability/Gamma/etc. to NEWS and CONTRIBUTORS
 eberlm parents: 
62016diff
changeset | 365 | |
| 61891 
76189756ff65
documentation on last state of the art concerning interpretation
 haftmann parents: 
61766diff
changeset | 366 | * Autumn 2015: Florian Haftmann, TUM | 
| 62064 | 367 | Rewrite definitions for global interpretations and sublocale declarations. | 
| 61891 
76189756ff65
documentation on last state of the art concerning interpretation
 haftmann parents: 
61766diff
changeset | 368 | |
| 61766 
507b39df1a57
add formalisation of Bourbaki-Witt fixpoint theorem
 Andreas Lochbihler parents: 
61552diff
changeset | 369 | * Autumn 2015: Andreas Lochbihler | 
| 62064 | 370 | Bourbaki-Witt fixpoint theorem for increasing functions on chain-complete | 
| 371 | partial orders. | |
| 61766 
507b39df1a57
add formalisation of Bourbaki-Witt fixpoint theorem
 Andreas Lochbihler parents: 
61552diff
changeset | 372 | |
| 61552 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
60920diff
changeset | 373 | * Autumn 2015: Chaitanya Mangla, Lawrence C Paulson, and Manuel Eberl | 
| 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
60920diff
changeset | 374 | A large number of additional binomial identities. | 
| 
980dd46a03fb
Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
 eberlm parents: 
60920diff
changeset | 375 | |
| 60632 | 376 | * Summer 2015: Daniel Matichuk, NICTA and Makarius Wenzel | 
| 62064 | 377 | Isar subgoal command for proof structure within unstructured proof scripts. | 
| 60632 | 378 | |
| 60434 | 379 | * Summer 2015: Florian Haftmann, TUM | 
| 60632 | 380 | Generic partial division in rings as inverse operation of multiplication. | 
| 60434 | 381 | |
| 60517 
f16e4fb20652
separate class for notions specific for integral (semi)domains, in contrast to fields where these are trivial
 haftmann parents: 
60434diff
changeset | 382 | * Summer 2015: Manuel Eberl and Florian Haftmann, TUM | 
| 62064 | 383 | Type class hierarchy with common algebraic notions of integral (semi)domains | 
| 384 | like units, associated elements and normalization wrt. units. | |
| 60517 
f16e4fb20652
separate class for notions specific for integral (semi)domains, in contrast to fields where these are trivial
 haftmann parents: 
60434diff
changeset | 385 | |
| 60804 | 386 | * Summer 2015: Florian Haftmann, TUM | 
| 387 | Fundamentals of abstract type class for factorial rings. | |
| 388 | ||
| 60920 | 389 | * Summer 2015: Julian Biendarra, TUM and Dmitriy Traytel, ETH Zurich | 
| 62064 | 390 | Command to lift a BNF structure on the raw type to the abstract type for | 
| 391 | typedefs. | |
| 60920 | 392 | |
| 62236 | 393 | * Summer 2014: Jeremy Avigad, Luke Serafin, CMU, and Johannes Hölzl, TUM | 
| 394 | Proof of the central limit theorem: includes weak convergence, | |
| 395 | characteristic functions, and Levy's uniqueness and continuity theorem. | |
| 396 | ||
| 60138 | 397 | |
| 60012 | 398 | Contributions to Isabelle2015 | 
| 399 | ----------------------------- | |
| 57695 | 400 | |
| 60119 
54bea620e54f
added Eisbach, using version 3752768caa17 of its Bitbucket repository;
 wenzelm parents: 
60012diff
changeset | 401 | * 2014/2015: Daniel Matichuk, Toby Murray, NICTA and Makarius Wenzel | 
| 
54bea620e54f
added Eisbach, using version 3752768caa17 of its Bitbucket repository;
 wenzelm parents: 
60012diff
changeset | 402 | The Eisbach proof method language and "match" method. | 
| 
54bea620e54f
added Eisbach, using version 3752768caa17 of its Bitbucket repository;
 wenzelm parents: 
60012diff
changeset | 403 | |
| 60260 | 404 | * Winter 2014 and Spring 2015: Ondrej Kuncar, TUM | 
| 60261 | 405 | Extension of lift_definition to execute lifted functions that have as a | 
| 406 | return type a datatype containing a subtype. | |
| 60260 | 407 | |
| 59980 | 408 | * March 2015: Jasmin Blanchette, Inria & LORIA & MPII, Mathias Fleury, MPII, | 
| 409 | and Dmitriy Traytel, TUM | |
| 59813 | 410 | More multiset theorems, syntax, and operations. | 
| 411 | ||
| 59980 | 412 | * December 2014: Johannes Hölzl, Manuel Eberl, Sudeep Kanav, TUM, and | 
| 413 | Jeremy Avigad, Luke Serafin, CMU | |
| 414 | Various integration theorems: mostly integration on intervals and | |
| 415 | substitution. | |
| 59092 
d469103c0737
add integral substitution theorems from Manuel Eberl, Jeremy Avigad, Luke Serafin, and Sudeep Kanav
 hoelzl parents: 
58626diff
changeset | 416 | |
| 58196 
1b3fbfb85980
theory about lexicographic ordering on functions
 haftmann parents: 
58023diff
changeset | 417 | * September 2014: Florian Haftmann, TUM | 
| 
1b3fbfb85980
theory about lexicographic ordering on functions
 haftmann parents: 
58023diff
changeset | 418 | Lexicographic order on functions and | 
| 
1b3fbfb85980
theory about lexicographic ordering on functions
 haftmann parents: 
58023diff
changeset | 419 | sum/product over function bodies. | 
| 
1b3fbfb85980
theory about lexicographic ordering on functions
 haftmann parents: 
58023diff
changeset | 420 | |
| 58626 | 421 | * August 2014: Andreas Lochbihler, ETH Zurich | 
| 59980 | 422 | Test infrastructure for executing generated code in target languages. | 
| 58626 | 423 | |
| 58023 
62826b36ac5e
generic euclidean algorithm (due to Manuel Eberl)
 haftmann parents: 
57882diff
changeset | 424 | * August 2014: Manuel Eberl, TUM | 
| 59980 | 425 | Generic euclidean algorithms for GCD et al. | 
| 58023 
62826b36ac5e
generic euclidean algorithm (due to Manuel Eberl)
 haftmann parents: 
57882diff
changeset | 426 | |
| 57695 | 427 | |
| 57452 | 428 | Contributions to Isabelle2014 | 
| 429 | ----------------------------- | |
| 54055 | 430 | |
| 57513 | 431 | * July 2014: Thomas Sewell, NICTA | 
| 57516 | 432 | Preserve equality hypotheses in "clarify" and friends. New | 
| 433 | "hypsubst_thin" method configuration option. | |
| 57513 | 434 | |
| 57519 | 435 | * Summer 2014: Florian Haftmann, TUM | 
| 436 | Consolidation and generalization of facts concerning (abelian) | |
| 437 | semigroups and monoids, particularly products (resp. sums) on | |
| 438 | finite sets. | |
| 57419 | 439 | |
| 57216 | 440 | * Summer 2014: Mathias Fleury, ENS Rennes, and Albert Steckermeier, TUM | 
| 57452 | 441 | Work on exotic automatic theorem provers for Sledgehammer (LEO-II, | 
| 442 | veriT, Waldmeister, etc.). | |
| 57216 | 443 | |
| 57875 | 444 | * June 2014: Florian Haftmann, TUM | 
| 445 | Internal reorganisation of the local theory / named target stack. | |
| 446 | ||
| 57254 
d3d91422f408
lemmas about the moments of the normal distribution
 hoelzl parents: 
57252diff
changeset | 447 | * June 2014: Sudeep Kanav, TUM, Jeremy Avigad, CMU, and Johannes Hölzl, TUM | 
| 57452 | 448 | Various properties of exponentially, Erlang, and normal distributed | 
| 449 | random variables. | |
| 57235 
b0b9a10e4bf4
properties of Erlang and exponentially distributed random variables (by Sudeep Kanav)
 hoelzl parents: 
57216diff
changeset | 450 | |
| 57452 | 451 | * May 2014: Cezary Kaliszyk, University of Innsbruck, and | 
| 452 | Jasmin Blanchette, TUM | |
| 57030 | 453 | SML-based engines for MaSh. | 
| 454 | ||
| 55913 | 455 | * March 2014: René Thiemann | 
| 55895 | 456 | Improved code generation for multisets. | 
| 457 | ||
| 56416 | 458 | * February 2014: Florian Haftmann, TUM | 
| 57452 | 459 | Permanent interpretation inside theory, locale and class targets | 
| 460 | with mixin definitions. | |
| 461 | ||
| 57474 | 462 | * Spring 2014: Lawrence C Paulson, Cambridge | 
| 463 | Theory Complex_Basic_Analysis. Tidying up Number_Theory vs Old_Number_Theory | |
| 464 | ||
| 57827 | 465 | * Winter 2013 and Spring 2014: Ondrej Kuncar, TUM | 
| 466 | Various improvements to Lifting/Transfer, integration with the BNF package. | |
| 467 | ||
| 57452 | 468 | * Winter 2013 and Spring 2014: Makarius Wenzel, Université Paris-Sud / LRI | 
| 469 | Improvements of Isabelle/Scala and Isabelle/jEdit Prover IDE. | |
| 56416 | 470 | |
| 57452 | 471 | * Fall 2013 and Winter 2014: Martin Desharnais, Lorenz Panny, | 
| 472 | Dmitriy Traytel, and Jasmin Blanchette, TUM | |
| 473 | Various improvements to the BNF-based (co)datatype package, | |
| 474 | including a more polished "primcorec" command, optimizations, and | |
| 475 | integration in the "HOL" session. | |
| 56118 
d3967fdc800a
updated NEWS and CONTRIBUTORS (BNF, SMT2, Sledgehammer)
 blanchet parents: 
55913diff
changeset | 476 | |
| 57452 | 477 | * Winter/Spring 2014: Sascha Boehme, QAware GmbH, and | 
| 478 | Jasmin Blanchette, TUM | |
| 479 | "SMT2" module and "smt2" proof method, based on SMT-LIB 2 and | |
| 480 | Z3 4.3. | |
| 56118 
d3967fdc800a
updated NEWS and CONTRIBUTORS (BNF, SMT2, Sledgehammer)
 blanchet parents: 
55913diff
changeset | 481 | |
| 55316 
885500f4aa6a
interactive simplifier trace: new panel in Isabelle/jEdit to inspect and modify simplification state
 Lars Hupel <lars.hupel@mytum.de> parents: 
54384diff
changeset | 482 | * January 2014: Lars Hupel, TUM | 
| 
885500f4aa6a
interactive simplifier trace: new panel in Isabelle/jEdit to inspect and modify simplification state
 Lars Hupel <lars.hupel@mytum.de> parents: 
54384diff
changeset | 483 | An improved, interactive simplifier trace with integration into the | 
| 
885500f4aa6a
interactive simplifier trace: new panel in Isabelle/jEdit to inspect and modify simplification state
 Lars Hupel <lars.hupel@mytum.de> parents: 
54384diff
changeset | 484 | Isabelle/jEdit Prover IDE. | 
| 54055 | 485 | |
| 56416 | 486 | * December 2013: Florian Haftmann, TUM | 
| 487 | Consolidation of abstract interpretations concerning min and max. | |
| 488 | ||
| 489 | * November 2013: Florian Haftmann, TUM | |
| 56418 | 490 | Abolition of negative numeral literals in the logic. | 
| 56416 | 491 | |
| 55913 | 492 | |
| 53984 | 493 | Contributions to Isabelle2013-1 | 
| 494 | ------------------------------- | |
| 50994 | 495 | |
| 54363 | 496 | * September 2013: Lars Noschinski, TUM | 
| 54364 | 497 | Conversion between function definitions as list of equations and | 
| 498 | case expressions in HOL. | |
| 499 | New library Simps_Case_Conv with commands case_of_simps, | |
| 500 | simps_of_case. | |
| 54363 | 501 | |
| 53396 | 502 | * September 2013: Nik Sultana, University of Cambridge | 
| 503 | Improvements to HOL/TPTP parser and import facilities. | |
| 504 | ||
| 54029 | 505 | * September 2013: Johannes Hölzl and Dmitriy Traytel, TUM | 
| 506 | New "coinduction" method (residing in HOL-BNF) to avoid boilerplate. | |
| 507 | ||
| 53984 | 508 | * Summer 2013: Makarius Wenzel, Université Paris-Sud / LRI | 
| 509 | Improvements of Isabelle/Scala and Isabelle/jEdit Prover IDE. | |
| 510 | ||
| 53613 | 511 | * Summer 2013: Manuel Eberl, TUM | 
| 512 | Generation of elimination rules in the function package. | |
| 513 | New command "fun_cases". | |
| 514 | ||
| 54051 | 515 | * Summer 2013: Christian Sternagel, JAIST | 
| 516 | Improved support for ad hoc overloading of constants, including | |
| 517 | documentation and examples. | |
| 518 | ||
| 53396 | 519 | * Spring and Summer 2013: Lorenz Panny, Dmitriy Traytel, and | 
| 520 | Jasmin Blanchette, TUM | |
| 56118 
d3967fdc800a
updated NEWS and CONTRIBUTORS (BNF, SMT2, Sledgehammer)
 blanchet parents: 
55913diff
changeset | 521 | Various improvements to the BNF-based (co)datatype package, including | 
| 54010 | 522 | "primrec_new" and "primcorec" commands and a compatibility layer. | 
| 53307 | 523 | |
| 54021 | 524 | * Spring and Summer 2013: Ondrej Kuncar, TUM | 
| 54035 | 525 | Various improvements of Lifting and Transfer packages. | 
| 54021 | 526 | |
| 527 | * Spring 2013: Brian Huffman, Galois Inc. | |
| 54035 | 528 | Improvements of the Transfer package. | 
| 54051 | 529 | |
| 53728 | 530 | * Summer 2013: Daniel Kühlwein, ICIS, Radboud University Nijmegen | 
| 531 | Jasmin Blanchette, TUM | |
| 532 | Various improvements to MaSh, including a server mode. | |
| 533 | ||
| 534 | * First half of 2013: Steffen Smolka, TUM | |
| 535 | Further improvements to Sledgehammer's Isar proof generator. | |
| 536 | ||
| 52485 | 537 | * May 2013: Florian Haftmann, TUM | 
| 538 | Ephemeral interpretation in local theories. | |
| 539 | ||
| 52266 | 540 | * May 2013: Lukas Bulwahn and Nicolai Schaffroth, TUM | 
| 53164 
beb4ee344c22
clarified position of Spec_Check for Isabelle/ML -- it is unrelated to Isabelle/HOL;
 wenzelm parents: 
52896diff
changeset | 541 | Spec_Check: A Quickcheck tool for Isabelle/ML. | 
| 52266 | 542 | |
| 51682 | 543 | * April 2013: Stefan Berghofer, secunet Security Networks AG | 
| 544 | Dmitriy Traytel, TUM | |
| 545 | Makarius Wenzel, Université Paris-Sud / LRI | |
| 546 | Case translations as a separate check phase independent of the | |
| 547 | datatype package. | |
| 548 | ||
| 51487 | 549 | * March 2013: Florian Haftmann, TUM | 
| 51489 | 550 | Reform of "big operators" on sets. | 
| 551 | ||
| 552 | * March 2013: Florian Haftmann, TUM | |
| 51487 | 553 | Algebraic locale hierarchy for orderings and (semi)lattices. | 
| 554 | ||
| 52503 | 555 | * February 2013: Florian Haftmann, TUM | 
| 556 | Reworking and consolidation of code generation for target language | |
| 557 | numerals. | |
| 51167 | 558 | |
| 52503 | 559 | * February 2013: Florian Haftmann, TUM | 
| 51173 | 560 | Sieve of Eratosthenes. | 
| 561 | ||
| 51167 | 562 | |
| 50993 | 563 | Contributions to Isabelle2013 | 
| 564 | ----------------------------- | |
| 47887 | 565 | |
| 49532 | 566 | * 2012: Makarius Wenzel, Université Paris-Sud / LRI | 
| 567 | Improvements of Isabelle/Scala and Isabelle/jEdit Prover IDE. | |
| 568 | ||
| 50648 | 569 | * Fall 2012: Daniel Kühlwein, ICIS, Radboud University Nijmegen | 
| 50222 | 570 | Jasmin Blanchette, TUM | 
| 571 | Implemented Machine Learning for Sledgehammer (MaSh). | |
| 572 | ||
| 50219 | 573 | * Fall 2012: Steffen Smolka, TUM | 
| 50648 | 574 | Various improvements to Sledgehammer's Isar proof generator, | 
| 575 | including a smart type annotation algorithm and proof shrinking. | |
| 50219 | 576 | |
| 50573 | 577 | * December 2012: Alessandro Coglio, Kestrel | 
| 50991 | 578 | Contributions to HOL's Lattice library. | 
| 50573 | 579 | |
| 50142 | 580 | * November 2012: Fabian Immler, TUM | 
| 50184 | 581 | "Symbols" dockable for Isabelle/jEdit. | 
| 582 | ||
| 583 | * November 2012: Fabian Immler, TUM | |
| 584 | Proof of the Daniell-Kolmogorov theorem: the existence of the limit | |
| 585 | of projective families. | |
| 50142 | 586 | |
| 49770 
cf6a78acf445
efficient construction of red black trees from sorted associative lists
 Andreas Lochbihler parents: 
49532diff
changeset | 587 | * October 2012: Andreas Lochbihler, KIT | 
| 50184 | 588 | Efficient construction of red-black trees from sorted associative | 
| 589 | lists. | |
| 49770 
cf6a78acf445
efficient construction of red black trees from sorted associative lists
 Andreas Lochbihler parents: 
49532diff
changeset | 590 | |
| 49190 | 591 | * September 2012: Florian Haftmann, TUM | 
| 592 | Lattice instances for type option. | |
| 593 | ||
| 49145 | 594 | * September 2012: Christian Sternagel, JAIST | 
| 595 | Consolidated HOL/Library (theories: Prefix_Order, Sublist, and | |
| 596 | Sublist_Order) w.r.t. prefixes, suffixes, and embedding on lists. | |
| 597 | ||
| 48977 | 598 | * August 2012: Dmitriy Traytel, Andrei Popescu, Jasmin Blanchette, TUM | 
| 49510 
ba50d204095e
renamed "Codatatype" directory "BNF" (and corresponding session) -- this opens the door to no-nonsense session names like "HOL-BNF-LFP"
 blanchet parents: 
49481diff
changeset | 599 | New BNF-based (co)datatype package. | 
| 48977 | 600 | |
| 601 | * August 2012: Andrei Popescu and Dmitriy Traytel, TUM | |
| 602 | Theories of ordinals and cardinals. | |
| 603 | ||
| 48585 
a82910dd2270
announce advanced support for Isabelle sessions and build management;
 wenzelm parents: 
48124diff
changeset | 604 | * July 2012: Makarius Wenzel, Université Paris-Sud / LRI | 
| 
a82910dd2270
announce advanced support for Isabelle sessions and build management;
 wenzelm parents: 
48124diff
changeset | 605 | Advanced support for Isabelle sessions and build management, notably | 
| 
a82910dd2270
announce advanced support for Isabelle sessions and build management;
 wenzelm parents: 
48124diff
changeset | 606 | "isabelle build". | 
| 
a82910dd2270
announce advanced support for Isabelle sessions and build management;
 wenzelm parents: 
48124diff
changeset | 607 | |
| 48111 | 608 | * June 2012: Felix Kuperjans, Lukas Bulwahn, TUM and Rafal Kolanski, NICTA | 
| 48585 
a82910dd2270
announce advanced support for Isabelle sessions and build management;
 wenzelm parents: 
48124diff
changeset | 609 | Simproc for rewriting set comprehensions into pointfree expressions. | 
| 47887 | 610 | |
| 49481 
818bf31759e7
NEWS and CONTRIBUTORS for a5377f6d9f14 and f0ecc1550998
 Andreas Lochbihler parents: 
49190diff
changeset | 611 | * May 2012: Andreas Lochbihler, KIT | 
| 
818bf31759e7
NEWS and CONTRIBUTORS for a5377f6d9f14 and f0ecc1550998
 Andreas Lochbihler parents: 
49190diff
changeset | 612 | Theory of almost everywhere constant functions. | 
| 48124 | 613 | |
| 50648 | 614 | * 2010-2012: Markus Kaiser and Lukas Bulwahn, TUM | 
| 615 | Graphview in Scala/Swing. | |
| 616 | ||
| 617 | ||
| 47462 | 618 | Contributions to Isabelle2012 | 
| 619 | ----------------------------- | |
| 45109 | 620 | |
| 47695 | 621 | * April 2012: Johannes Hölzl, TUM | 
| 47808 | 622 | Probability: Introduced type to represent measures instead of | 
| 623 | locales. | |
| 47695 | 624 | |
| 625 | * April 2012: Johannes Hölzl, Fabian Immler, TUM | |
| 626 | Float: Moved to Dyadic rationals to represent floating point numers. | |
| 627 | ||
| 47808 | 628 | * April 2012: Thomas Sewell, NICTA and | 
| 629 | 2010: Sascha Boehme, TUM | |
| 630 | Theory HOL/Word/WordBitwise: logic/circuit expansion of bitvector | |
| 631 | equalities/inequalities. | |
| 47567 
407cabf66f21
New tactic "word_bitwise" expands word equalities/inequalities into logic.
 Thomas Sewell <thomas.sewell@nicta.com.au> parents: 
47563diff
changeset | 632 | |
| 47808 | 633 | * March 2012: Christian Sternagel, JAIST | 
| 47448 | 634 | Consolidated theory of relation composition. | 
| 635 | ||
| 47413 | 636 | * March 2012: Nik Sultana, University of Cambridge | 
| 637 | HOL/TPTP parser and import facilities. | |
| 638 | ||
| 47462 | 639 | * March 2012: Cezary Kaliszyk, University of Innsbruck and | 
| 640 | Alexander Krauss, QAware GmbH | |
| 641 | Faster and more scalable Import mechanism for HOL Light proofs. | |
| 642 | ||
| 47563 | 643 | * January 2012: Florian Haftmann, TUM, et al. | 
| 46596 | 644 | (Re-)Introduction of the "set" type constructor. | 
| 645 | ||
| 47700 | 646 | * 2012: Ondrej Kuncar, TUM | 
| 47808 | 647 | New package Lifting, various improvements and refinements to the | 
| 648 | Quotient package. | |
| 47700 | 649 | |
| 47563 | 650 | * 2011/2012: Jasmin Blanchette, TUM | 
| 651 | Various improvements to Sledgehammer, notably: tighter integration | |
| 47808 | 652 | with SPASS, support for more provers (Alt-Ergo, iProver, | 
| 653 | iProver-Eq). | |
| 47563 | 654 | |
| 47462 | 655 | * 2011/2012: Makarius Wenzel, Université Paris-Sud / LRI | 
| 47485 | 656 | Various refinements of local theory infrastructure. | 
| 47462 | 657 | Improvements of Isabelle/Scala layer and Isabelle/jEdit Prover IDE. | 
| 47265 | 658 | |
| 45109 | 659 | |
| 44801 | 660 | Contributions to Isabelle2011-1 | 
| 661 | ------------------------------- | |
| 41651 | 662 | |
| 44818 
27ba81ad0890
theory of saturated naturals contributed by Peter Gammie
 haftmann parents: 
41651diff
changeset | 663 | * September 2011: Peter Gammie | 
| 44908 | 664 | Theory HOL/Library/Saturated: numbers with saturated arithmetic. | 
| 44818 
27ba81ad0890
theory of saturated naturals contributed by Peter Gammie
 haftmann parents: 
41651diff
changeset | 665 | |
| 
27ba81ad0890
theory of saturated naturals contributed by Peter Gammie
 haftmann parents: 
41651diff
changeset | 666 | * August 2011: Florian Haftmann, Johannes Hölzl and Lars Noschinski, TUM | 
| 
27ba81ad0890
theory of saturated naturals contributed by Peter Gammie
 haftmann parents: 
41651diff
changeset | 667 | Refined theory on complete lattices. | 
| 
27ba81ad0890
theory of saturated naturals contributed by Peter Gammie
 haftmann parents: 
41651diff
changeset | 668 | |
| 44967 | 669 | * August 2011: Brian Huffman, Portland State University | 
| 670 | Miscellaneous cleanup of Complex_Main and Multivariate_Analysis. | |
| 671 | ||
| 672 | * June 2011: Brian Huffman, Portland State University | |
| 673 | Proof method "countable_datatype" for theory Library/Countable. | |
| 674 | ||
| 675 | * 2011: Jasmin Blanchette, TUM | |
| 676 | Various improvements to Sledgehammer, notably: use of sound | |
| 677 | translations, support for more provers (Waldmeister, LEO-II, | |
| 678 | Satallax). Further development of Nitpick and 'try' command. | |
| 679 | ||
| 680 | * 2011: Andreas Lochbihler, Karlsruhe Institute of Technology | |
| 681 | Theory HOL/Library/Cset_Monad allows do notation for computable sets | |
| 682 | (cset) via the generic monad ad-hoc overloading facility. | |
| 683 | ||
| 684 | * 2011: Johannes Hölzl, Armin Heller, TUM and | |
| 685 | Bogdan Grechuk, University of Edinburgh | |
| 686 | Theory HOL/Library/Extended_Reals: real numbers extended with plus | |
| 687 | and minus infinity. | |
| 688 | ||
| 44882 | 689 | * 2011: Makarius Wenzel, Université Paris-Sud / LRI | 
| 690 | Various building blocks for Isabelle/Scala layer and Isabelle/jEdit | |
| 691 | Prover IDE. | |
| 692 | ||
| 44908 | 693 | |
| 41512 | 694 | Contributions to Isabelle2011 | 
| 695 | ----------------------------- | |
| 37383 | 696 | |
| 41567 | 697 | * January 2011: Stefan Berghofer, secunet Security Networks AG | 
| 698 | HOL-SPARK: an interactive prover back-end for SPARK. | |
| 699 | ||
| 40379 | 700 | * October 2010: Bogdan Grechuk, University of Edinburgh | 
| 701 | Extended convex analysis in Multivariate Analysis. | |
| 702 | ||
| 40287 | 703 | * October 2010: Dmitriy Traytel, TUM | 
| 704 | Coercive subtyping via subtype constraints. | |
| 705 | ||
| 41531 | 706 | * October 2010: Alexander Krauss, TUM | 
| 707 | Command partial_function for function definitions based on complete | |
| 708 | partial orders in HOL. | |
| 709 | ||
| 39644 | 710 | * September 2010: Florian Haftmann, TUM | 
| 41596 | 711 | Refined concepts for evaluation, i.e., normalization of terms using | 
| 41531 | 712 | different techniques. | 
| 40120 | 713 | |
| 714 | * September 2010: Florian Haftmann, TUM | |
| 39644 | 715 | Code generation for Scala. | 
| 716 | ||
| 38656 | 717 | * August 2010: Johannes Hoelzl, Armin Heller, and Robert Himmelmann, TUM | 
| 41596 | 718 | Improved Probability theory in HOL. | 
| 38656 | 719 | |
| 38461 | 720 | * July 2010: Florian Haftmann, TUM | 
| 39644 | 721 | Reworking and extension of the Imperative HOL framework. | 
| 38461 | 722 | |
| 41596 | 723 | * July 2010: Alexander Krauss, TUM and Christian Sternagel, University | 
| 724 | of Innsbruck | |
| 41531 | 725 | Ad-hoc overloading. Generic do notation for monads. | 
| 726 | ||
| 37383 | 727 | |
| 37144 | 728 | Contributions to Isabelle2009-2 | 
| 41512 | 729 | ------------------------------- | 
| 33951 | 730 | |
| 37303 | 731 | * 2009/2010: Stefan Berghofer, Alexander Krauss, and Andreas Schropp, TUM, | 
| 732 | Makarius Wenzel, TUM / LRI | |
| 733 | Elimination of type classes from proof terms. | |
| 734 | ||
| 37144 | 735 | * April 2010: Florian Haftmann, TUM | 
| 36416 | 736 | Reorganization of abstract algebra type classes. | 
| 737 | ||
| 37144 | 738 | * April 2010: Florian Haftmann, TUM | 
| 36416 | 739 | Code generation for data representations involving invariants; | 
| 740 | various collections avaiable in theories Fset, Dlist, RBT, | |
| 741 | Mapping and AssocList. | |
| 742 | ||
| 37144 | 743 | * March 2010: Sascha Boehme, TUM | 
| 744 | Efficient SHA1 library for Poly/ML. | |
| 745 | ||
| 37282 | 746 | * February 2010: Cezary Kaliszyk and Christian Urban, TUM | 
| 747 | Quotient type package for Isabelle/HOL. | |
| 748 | ||
| 26874 | 749 | |
| 33842 | 750 | Contributions to Isabelle2009-1 | 
| 751 | ------------------------------- | |
| 33649 
854173fcd21c
added a tabled implementation of the reflexive transitive closure
 bulwahn parents: 
33627diff
changeset | 752 | |
| 33862 | 753 | * November 2009, Brian Huffman, PSU | 
| 754 | New definitional domain package for HOLCF. | |
| 755 | ||
| 33759 
b369324fc244
Added the contributions of Robert Himmelmann to CONTRIBUTIONS and NEWS
 hoelzl parents: 
33649diff
changeset | 756 | * November 2009: Robert Himmelmann, TUM | 
| 33862 | 757 | Derivation and Brouwer's fixpoint theorem in Multivariate Analysis. | 
| 33759 
b369324fc244
Added the contributions of Robert Himmelmann to CONTRIBUTIONS and NEWS
 hoelzl parents: 
33649diff
changeset | 758 | |
| 33842 | 759 | * November 2009: Stefan Berghofer and Lukas Bulwahn, TUM | 
| 760 | A tabled implementation of the reflexive transitive closure. | |
| 33649 
854173fcd21c
added a tabled implementation of the reflexive transitive closure
 bulwahn parents: 
33627diff
changeset | 761 | |
| 33627 
ffb4a811e34d
announcing the predicate compiler in NEWS and CONTRIBUTORS
 bulwahn parents: 
33419diff
changeset | 762 | * November 2009: Lukas Bulwahn, TUM | 
| 33842 | 763 | Predicate Compiler: a compiler for inductive predicates to | 
| 33843 | 764 | equational specifications. | 
| 48977 | 765 | |
| 33897 | 766 | * November 2009: Sascha Boehme, TUM and Burkhart Wolff, LRI Paris | 
| 33842 | 767 | HOL-Boogie: an interactive prover back-end for Boogie and VCC. | 
| 33419 | 768 | |
| 33192 
08a39a957ed7
added Nitpick's theory and ML files to Isabelle/HOL;
 blanchet parents: 
33010diff
changeset | 769 | * October 2009: Jasmin Blanchette, TUM | 
| 33842 | 770 | Nitpick: yet another counterexample generator for Isabelle/HOL. | 
| 33192 
08a39a957ed7
added Nitpick's theory and ML files to Isabelle/HOL;
 blanchet parents: 
33010diff
changeset | 771 | |
| 33010 | 772 | * October 2009: Sascha Boehme, TUM | 
| 33182 | 773 | Extension of SMT method: proof-reconstruction for the SMT solver Z3. | 
| 33010 | 774 | |
| 775 | * October 2009: Florian Haftmann, TUM | |
| 33182 | 776 | Refinement of parts of the HOL datatype package. | 
| 33005 | 777 | |
| 33010 | 778 | * October 2009: Florian Haftmann, TUM | 
| 33182 | 779 | Generic term styles for term antiquotations. | 
| 33005 | 780 | |
| 32762 
5f485f98652f
Thomas Sewell, NICTA: more efficient HOL/record implementation;
 wenzelm parents: 
32618diff
changeset | 781 | * September 2009: Thomas Sewell, NICTA | 
| 33182 | 782 | More efficient HOL/record implementation. | 
| 32762 
5f485f98652f
Thomas Sewell, NICTA: more efficient HOL/record implementation;
 wenzelm parents: 
32618diff
changeset | 783 | |
| 32618 
42865636d006
added new method "smt": an oracle-based connection to external SMT solvers
 boehmes parents: 
32600diff
changeset | 784 | * September 2009: Sascha Boehme, TUM | 
| 33182 | 785 | SMT method using external SMT solvers. | 
| 32618 
42865636d006
added new method "smt": an oracle-based connection to external SMT solvers
 boehmes parents: 
32600diff
changeset | 786 | |
| 32600 | 787 | * September 2009: Florian Haftmann, TUM | 
| 33182 | 788 | Refinement of sets and lattices. | 
| 32600 | 789 | |
| 790 | * July 2009: Jeremy Avigad and Amine Chaieb | |
| 33182 | 791 | New number theory. | 
| 32600 | 792 | |
| 32268 
d50f0cb67578
Functionality for sum of squares to call a remote csdp prover
 Philipp Meyer parents: 
31997diff
changeset | 793 | * July 2009: Philipp Meyer, TUM | 
| 33182 | 794 | HOL/Library/Sum_Of_Squares: functionality to call a remote csdp | 
| 795 | prover. | |
| 32268 
d50f0cb67578
Functionality for sum of squares to call a remote csdp prover
 Philipp Meyer parents: 
31997diff
changeset | 796 | |
| 31997 | 797 | * July 2009: Florian Haftmann, TUM | 
| 33182 | 798 | New quickcheck implementation using new code generator. | 
| 31997 | 799 | |
| 800 | * July 2009: Florian Haftmann, TUM | |
| 39644 | 801 | HOL/Library/Fset: an explicit type of sets; finite sets ready to use | 
| 33182 | 802 | for code generation. | 
| 31466 | 803 | |
| 804 | * June 2009: Florian Haftmann, TUM | |
| 33843 | 805 | HOL/Library/Tree: search trees implementing mappings, ready to use | 
| 33182 | 806 | for code generation. | 
| 30978 | 807 | |
| 32268 
d50f0cb67578
Functionality for sum of squares to call a remote csdp prover
 Philipp Meyer parents: 
31997diff
changeset | 808 | * March 2009: Philipp Meyer, TUM | 
| 33843 | 809 | Minimization tool for results from Sledgehammer. | 
| 33182 | 810 | |
| 32268 
d50f0cb67578
Functionality for sum of squares to call a remote csdp prover
 Philipp Meyer parents: 
31997diff
changeset | 811 | |
| 30978 | 812 | Contributions to Isabelle2009 | 
| 813 | ----------------------------- | |
| 814 | ||
| 30383 | 815 | * March 2009: Robert Himmelmann, TUM and Amine Chaieb, University of | 
| 816 | Cambridge | |
| 817 | Elementary topology in Euclidean space. | |
| 818 | ||
| 30886 
dda08b76fa99
updated official title of contribution by Johannes Hoelzl;
 wenzelm parents: 
30383diff
changeset | 819 | * March 2009: Johannes Hoelzl, TUM | 
| 
dda08b76fa99
updated official title of contribution by Johannes Hoelzl;
 wenzelm parents: 
30383diff
changeset | 820 | Method "approximation", which proves real valued inequalities by | 
| 
dda08b76fa99
updated official title of contribution by Johannes Hoelzl;
 wenzelm parents: 
30383diff
changeset | 821 | computation. | 
| 
dda08b76fa99
updated official title of contribution by Johannes Hoelzl;
 wenzelm parents: 
30383diff
changeset | 822 | |
| 30179 | 823 | * February 2009: Filip Maric, Univ. of Belgrade | 
| 824 | A Serbian theory. | |
| 825 | ||
| 30162 | 826 | * February 2009: Jasmin Christian Blanchette, TUM | 
| 30154 | 827 | Misc cleanup of HOL/refute. | 
| 828 | ||
| 30162 | 829 | * February 2009: Timothy Bourke, NICTA | 
| 29883 | 830 | New find_consts command. | 
| 831 | ||
| 30162 | 832 | * February 2009: Timothy Bourke, NICTA | 
| 29861 
3c348f5873f3
updated NEWS etc with "solves" criterion and auto_solves
 kleing parents: 
29398diff
changeset | 833 | "solves" criterion for find_theorems and auto_solve option | 
| 
3c348f5873f3
updated NEWS etc with "solves" criterion and auto_solves
 kleing parents: 
29398diff
changeset | 834 | |
| 29398 | 835 | * December 2008: Clemens Ballarin, TUM | 
| 836 | New locale implementation. | |
| 837 | ||
| 29182 | 838 | * December 2008: Armin Heller, TUM and Alexander Krauss, TUM | 
| 839 | Method "sizechange" for advanced termination proofs. | |
| 840 | ||
| 28901 | 841 | * November 2008: Timothy Bourke, NICTA | 
| 842 | Performance improvement (factor 50) for find_theorems. | |
| 843 | ||
| 29398 | 844 | * 2008: Florian Haftmann, TUM | 
| 845 | Various extensions and restructurings in HOL, improvements | |
| 846 | in evaluation mechanisms, new module binding.ML for name bindings. | |
| 847 | ||
| 28604 
f36496b73227
generic ATP manager based on threads (by Fabian Immler);
 wenzelm parents: 
28474diff
changeset | 848 | * October 2008: Fabian Immler, TUM | 
| 
f36496b73227
generic ATP manager based on threads (by Fabian Immler);
 wenzelm parents: 
28474diff
changeset | 849 | ATP manager for Sledgehammer, based on ML threads instead of Posix | 
| 
f36496b73227
generic ATP manager based on threads (by Fabian Immler);
 wenzelm parents: 
28474diff
changeset | 850 | processes. Additional ATP wrappers, including remote SystemOnTPTP | 
| 
f36496b73227
generic ATP manager based on threads (by Fabian Immler);
 wenzelm parents: 
28474diff
changeset | 851 | services. | 
| 
f36496b73227
generic ATP manager based on threads (by Fabian Immler);
 wenzelm parents: 
28474diff
changeset | 852 | |
| 30162 | 853 | * September 2008: Stefan Berghofer, TUM and Marc Bezem, Univ. Bergen | 
| 854 | Prover for coherent logic. | |
| 855 | ||
| 28474 
d0b8b0a1fca5
Vampire wrapper script for remote SystemOnTPTP service (by Fabian Immler);
 wenzelm parents: 
27009diff
changeset | 856 | * August 2008: Fabian Immler, TUM | 
| 
d0b8b0a1fca5
Vampire wrapper script for remote SystemOnTPTP service (by Fabian Immler);
 wenzelm parents: 
27009diff
changeset | 857 | Vampire wrapper script for remote SystemOnTPTP service. | 
| 
d0b8b0a1fca5
Vampire wrapper script for remote SystemOnTPTP service (by Fabian Immler);
 wenzelm parents: 
27009diff
changeset | 858 | |
| 
d0b8b0a1fca5
Vampire wrapper script for remote SystemOnTPTP service (by Fabian Immler);
 wenzelm parents: 
27009diff
changeset | 859 | |
| 
d0b8b0a1fca5
Vampire wrapper script for remote SystemOnTPTP service (by Fabian Immler);
 wenzelm parents: 
27009diff
changeset | 860 | Contributions to Isabelle2008 | 
| 
d0b8b0a1fca5
Vampire wrapper script for remote SystemOnTPTP service (by Fabian Immler);
 wenzelm parents: 
27009diff
changeset | 861 | ----------------------------- | 
| 
d0b8b0a1fca5
Vampire wrapper script for remote SystemOnTPTP service (by Fabian Immler);
 wenzelm parents: 
27009diff
changeset | 862 | |
| 27009 | 863 | * 2007/2008: | 
| 864 | Alexander Krauss, TUM and Florian Haftmann, TUM and Stefan Berghofer, TUM | |
| 865 | HOL library improvements. | |
| 25468 | 866 | |
| 27009 | 867 | * 2007/2008: Brian Huffman, PSU | 
| 868 | HOLCF library improvements. | |
| 869 | ||
| 870 | * 2007/2008: Stefan Berghofer, TUM | |
| 30179 | 871 | HOL-Nominal package improvements. | 
| 27009 | 872 | |
| 873 | * March 2008: Markus Reiter, TUM | |
| 874 | HOL/Library/RBT: red-black trees. | |
| 26728 | 875 | |
| 26874 | 876 | * February 2008: Alexander Krauss, TUM and Florian Haftmann, TUM and | 
| 877 | Lukas Bulwahn, TUM and John Matthews, Galois: | |
| 878 | HOL/Library/Imperative_HOL: Haskell-style imperative data structures | |
| 879 | for HOL. | |
| 26728 | 880 | |
| 27009 | 881 | * December 2007: Norbert Schirmer, Uni Saarbruecken | 
| 882 | Misc improvements of record package in HOL. | |
| 883 | ||
| 884 | * December 2007: Florian Haftmann, TUM | |
| 885 | Overloading and class instantiation target. | |
| 886 | ||
| 887 | * December 2007: Florian Haftmann, TUM | |
| 888 | New version of primrec package for local theories. | |
| 889 | ||
| 890 | * December 2007: Alexander Krauss, TUM | |
| 891 | Method "induction_scheme" in HOL. | |
| 892 | ||
| 893 | * November 2007: Peter Lammich, Uni Muenster | |
| 894 | HOL-Lattice: some more lemmas. | |
| 26198 | 895 | |
| 26874 | 896 | |
| 25454 | 897 | Contributions to Isabelle2007 | 
| 898 | ----------------------------- | |
| 23252 | 899 | |
| 25409 | 900 | * October 2007: Norbert Schirmer, TUM / Uni Saarbruecken | 
| 25398 | 901 | State Spaces: The Locale Way (in HOL). | 
| 902 | ||
| 25057 
021fcbe2aaa5
Mark A. Hillebrand, DFKI: Robust sub/superscripts in LaTeX document output.
 wenzelm parents: 
24803diff
changeset | 903 | * October 2007: Mark A. Hillebrand, DFKI | 
| 
021fcbe2aaa5
Mark A. Hillebrand, DFKI: Robust sub/superscripts in LaTeX document output.
 wenzelm parents: 
24803diff
changeset | 904 | Robust sub/superscripts in LaTeX document output. | 
| 
021fcbe2aaa5
Mark A. Hillebrand, DFKI: Robust sub/superscripts in LaTeX document output.
 wenzelm parents: 
24803diff
changeset | 905 | |
| 24799 | 906 | * August 2007: Jeremy Dawson, NICTA and Paul Graunke, Galois and Brian | 
| 907 | Huffman, PSU and Gerwin Klein, NICTA and John Matthews, Galois | |
| 24333 | 908 | HOL-Word: a library for fixed-size machine words in Isabelle. | 
| 909 | ||
| 24332 
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
 kleing parents: 
23449diff
changeset | 910 | * August 2007: Brian Huffman, PSU | 
| 24799 | 911 | HOL/Library/Boolean_Algebra and HOL/Library/Numeral_Type. | 
| 24332 
e3a2b75b1cf9
boolean algebras as locales and numbers as types by Brian Huffman
 kleing parents: 
23449diff
changeset | 912 | |
| 23252 | 913 | * June 2007: Amine Chaieb, TUM | 
| 24799 | 914 | Semiring normalization and Groebner Bases. | 
| 25449 | 915 | Support for dense linear orders. | 
| 17866 | 916 | |
| 23449 | 917 | * June 2007: Joe Hurd, Oxford | 
| 24799 | 918 | Metis theorem-prover. | 
| 919 | ||
| 920 | * 2007: Kong W. Susanto, Cambridge | |
| 921 | HOL: Metis prover integration. | |
| 23449 | 922 | |
| 24799 | 923 | * 2007: Stefan Berghofer, TUM | 
| 25449 | 924 | HOL: inductive predicates and sets. | 
| 24799 | 925 | |
| 24803 | 926 | * 2007: Norbert Schirmer, TUM | 
| 927 | HOL/record: misc improvements. | |
| 928 | ||
| 24799 | 929 | * 2006/2007: Alexander Krauss, TUM | 
| 930 | HOL: function package and related theories on termination. | |
| 23449 | 931 | |
| 22449 | 932 | * 2006/2007: Florian Haftmann, TUM | 
| 933 | Pure: generic code generator framework. | |
| 934 | Pure: class package. | |
| 24799 | 935 | HOL: theory reorganization, code generator setup. | 
| 936 | ||
| 25449 | 937 | * 2006/2007: Christian Urban, TUM and Stefan Berghofer, TUM and | 
| 938 | Julien Narboux, TUM | |
| 24799 | 939 | HOL/Nominal package and related tools. | 
| 22449 | 940 | |
| 21242 
d73735bb33c1
* November 2006: Lukas Bulwahn, TUM -- HOL/function: method "lexicographic_order".
 wenzelm parents: 
21169diff
changeset | 941 | * November 2006: Lukas Bulwahn, TUM | 
| 24799 | 942 | HOL: method "lexicographic_order" for function package. | 
| 21242 
d73735bb33c1
* November 2006: Lukas Bulwahn, TUM -- HOL/function: method "lexicographic_order".
 wenzelm parents: 
21169diff
changeset | 943 | |
| 21169 | 944 | * October 2006: Stefan Hohe, TUM | 
| 945 | HOL-Algebra: ideals and quotients over rings. | |
| 946 | ||
| 20340 
6afc1c133b86
Amine Chaieb: experimental generic reflection and reification in HOL;
 wenzelm parents: 
20067diff
changeset | 947 | * August 2006: Amine Chaieb, TUM | 
| 
6afc1c133b86
Amine Chaieb: experimental generic reflection and reification in HOL;
 wenzelm parents: 
20067diff
changeset | 948 | Experimental support for generic reflection and reification in HOL. | 
| 
6afc1c133b86
Amine Chaieb: experimental generic reflection and reification in HOL;
 wenzelm parents: 
20067diff
changeset | 949 | |
| 20067 
26bac504ef90
hex and binary numerals (contributed by Rafal Kolanski)
 kleing parents: 
19896diff
changeset | 950 | * July 2006: Rafal Kolanski, NICTA | 
| 
26bac504ef90
hex and binary numerals (contributed by Rafal Kolanski)
 kleing parents: 
19896diff
changeset | 951 | Hex (0xFF) and binary (0b1011) numerals. | 
| 
26bac504ef90
hex and binary numerals (contributed by Rafal Kolanski)
 kleing parents: 
19896diff
changeset | 952 | |
| 19896 | 953 | * May 2006: Klaus Aehlig, LMU | 
| 954 | Command 'normal_form': normalization by evaluation. | |
| 955 | ||
| 19650 | 956 | * May 2006: Amine Chaieb, TUM | 
| 957 | HOL-Complex: Ferrante and Rackoff Algorithm for linear real | |
| 958 | arithmetic. | |
| 19470 | 959 | |
| 960 | * February 2006: Benjamin Porter, NICTA | |
| 23382 | 961 | HOL and HOL-Complex: generalised mean value theorem, continuum is | 
| 19470 | 962 | not denumerable, harmonic and arithmetic series, and denumerability | 
| 963 | of rationals. | |
| 17532 | 964 | |
| 19650 | 965 | * October 2005: Martin Wildmoser, TUM | 
| 966 | Sketch for Isar 'guess' element. | |
| 967 | ||
| 968 | ||
| 25454 | 969 | Contributions to Isabelle2005 | 
| 970 | ----------------------------- | |
| 17382 | 971 | |
| 17640 | 972 | * September 2005: Lukas Bulwahn and Bernhard Haeupler, TUM | 
| 973 | HOL-Complex: Formalization of Taylor series. | |
| 974 | ||
| 975 | * September 2005: Stephan Merz, Alwen Tiu, QSL Loria | |
| 976 | Components for SAT solver method using zChaff. | |
| 977 | ||
| 17534 | 978 | * September 2005: Ning Zhang and Christian Urban, LMU Munich | 
| 979 | A Chinese theory. | |
| 980 | ||
| 17562 | 981 | * September 2005: Bernhard Haeupler, TUM | 
| 17382 | 982 | Method comm_ring for proving equalities in commutative rings. | 
| 16892 | 983 | |
| 17532 | 984 | * July/August 2005: Jeremy Avigad, Carnegie Mellon University | 
| 16892 | 985 | Various improvements of the HOL and HOL-Complex library. | 
| 16868 | 986 | |
| 16892 | 987 | * July 2005: Florian Zuleger, Johannes Hoelzl, and Simon Funke, TUM | 
| 988 | Some structured proofs about completeness of real numbers. | |
| 989 | ||
| 17532 | 990 | * May 2005: Rafal Kolanski and Gerwin Klein, NICTA | 
| 991 | Improved retrieval of facts from theory/proof context. | |
| 15994 | 992 | |
| 16252 | 993 | * February 2005: Lucas Dixon, University of Edinburgh | 
| 17532 | 994 | Improved subst method. | 
| 995 | ||
| 996 | * 2005: Brian Huffman, OGI | |
| 997 | Various improvements of HOLCF. | |
| 998 | Some improvements of the HOL-Complex library. | |
| 999 | ||
| 1000 | * 2005: Claire Quigley and Jia Meng, University of Cambridge | |
| 1001 | Some support for asynchronous communication with external provers | |
| 1002 | (experimental). | |
| 1003 | ||
| 1004 | * 2005: Florian Haftmann, TUM | |
| 17543 | 1005 | Contributions to document 'sugar'. | 
| 17532 | 1006 | Various ML combinators, notably linear functional transformations. | 
| 1007 | Some cleanup of ML legacy. | |
| 1008 | Additional antiquotations. | |
| 1009 | Improved Isabelle web site. | |
| 1010 | ||
| 1011 | * 2004/2005: David Aspinall, University of Edinburgh | |
| 1012 | Various elements of XML and PGIP based communication with user | |
| 1013 | interfaces (experimental). | |
| 1014 | ||
| 1015 | * 2004/2005: Gerwin Klein, NICTA | |
| 1016 | Contributions to document 'sugar'. | |
| 1017 | Improved Isabelle web site. | |
| 1018 | Improved HTML presentation of theories. | |
| 1019 | ||
| 1020 | * 2004/2005: Clemens Ballarin, TUM | |
| 1021 | Provers: tools for transitive relations and quasi orders. | |
| 1022 | Improved version of locales, notably interpretation of locales. | |
| 1023 | Improved version of HOL-Algebra. | |
| 1024 | ||
| 1025 | * 2004/2005: Amine Chaieb, TUM | |
| 1026 | Improved version of HOL presburger method. | |
| 1027 | ||
| 1028 | * 2004/2005: Steven Obua, TUM | |
| 1029 | Improved version of HOL/Import, support for HOL-Light. | |
| 1030 | Improved version of HOL-Complex-Matrix. | |
| 17572 | 1031 | Pure/defs: more sophisticated checks on well-formedness of overloading. | 
| 17543 | 1032 | Pure/Tools: an experimental evaluator for lambda terms. | 
| 17532 | 1033 | |
| 1034 | * 2004/2005: Norbert Schirmer, TUM | |
| 1035 | Contributions to document 'sugar'. | |
| 1036 | Improved version of HOL/record. | |
| 1037 | ||
| 1038 | * 2004/2005: Sebastian Skalberg, TUM | |
| 1039 | Improved version of HOL/Import. | |
| 1040 | Some internal ML reorganizations. | |
| 1041 | ||
| 1042 | * 2004/2005: Tjark Weber, TUM | |
| 17640 | 1043 | SAT solver method using zChaff. | 
| 17532 | 1044 | Improved version of HOL/refute. | 
| 62098 | 1045 | |
| 1046 | :maxLineLen=78: |