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