CONTRIBUTORS
author Manuel Eberl <eberlm@in.tum.de>
Mon, 02 Dec 2019 14:22:28 +0100
changeset 71193 777d673fa672
parent 70955 73ae8c30c6cb
child 71264 0c454a5d125d
permissions -rw-r--r--
Removed duplicate theorems from HOL-Analysis
Ignore whitespace changes - Everywhere: Within whitespace: At end of lines:
24799
dff164b6f2a6 misc tuning and update;
wenzelm
parents: 24333
diff changeset
     1
For the purposes of the license agreement in the file COPYRIGHT, a
62098
wenzelm
parents: 62086
diff changeset
     2
'contributor' is anybody who is listed in this file (CONTRIBUTORS) or who is
wenzelm
parents: 62086
diff changeset
     3
listed as an author in one of the source files of this Isabelle distribution.
wenzelm
parents: 62086
diff changeset
     4
23382
0459ab90389a clarified who we consider to be a contributor
kleing
parents: 23252
diff changeset
     5
70265
a8238fd25541 back to post-release mode;
wenzelm
parents: 70216
diff changeset
     6
Contributions to this Isabelle version
a8238fd25541 back to post-release mode;
wenzelm
parents: 70216
diff changeset
     7
--------------------------------------
a8238fd25541 back to post-release mode;
wenzelm
parents: 70216
diff changeset
     8
70955
73ae8c30c6cb added contributor
immler
parents: 70265
diff changeset
     9
* October 2019: Maximilian Schäffeler
73ae8c30c6cb added contributor
immler
parents: 70265
diff changeset
    10
  Port of the HOL Light decision procedure for metric spaces.
70265
a8238fd25541 back to post-release mode;
wenzelm
parents: 70216
diff changeset
    11
70024
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    12
Contributions to Isabelle2019
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    13
-----------------------------
69814
5929b172c6fe CONTRIBUTORS
haftmann
parents: 69791
diff changeset
    14
70164
1f163f772da3 Group theory developments towards proving algebraic closure (by de Vilhena and Baillon)
paulson <lp15@cam.ac.uk>
parents: 70024
diff changeset
    15
* 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
    16
  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
    17
1f163f772da3 Group theory developments towards proving algebraic closure (by de Vilhena and Baillon)
paulson <lp15@cam.ac.uk>
parents: 70024
diff changeset
    18
* April 2019: Paulo de Vilhena and Martin Baillon
70216
40f19372a723 A bit of de-applying
paulson <lp15@cam.ac.uk>
parents: 70164
diff changeset
    19
  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
    20
70024
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    21
* February/March 2019: Makarius Wenzel
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    22
  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
    23
69785
9e326f6f8a24 More material for HOL-Number_Theory: ord, Carmichael's function, primitive roots
Manuel Eberl <eberlm@in.tum.de>
parents: 69568
diff changeset
    24
* February 2019: Manuel Eberl
69790
154cf64e403e Exponentiation by squaring, fast modular exponentiation
Manuel Eberl <eberlm@in.tum.de>
parents: 69785
diff changeset
    25
  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
    26
  fast modular exponentiation.
154cf64e403e Exponentiation by squaring, fast modular exponentiation
Manuel Eberl <eberlm@in.tum.de>
parents: 69785
diff changeset
    27
154cf64e403e Exponentiation by squaring, fast modular exponentiation
Manuel Eberl <eberlm@in.tum.de>
parents: 69785
diff changeset
    28
* February 2019: Manuel Eberl
70024
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    29
  Carmichael's function, primitive roots in residue rings, more properties of
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    30
  the order in residue rings.
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    31
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    32
* February 2019: Jeremy Sylvestre
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    33
  Formal Laurent Series and overhaul of Formal power series.
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    34
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    35
* January 2019: Florian Haftmann
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    36
  Clarified syntax and congruence rules for big operators on sets involving
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    37
  the image operator.
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    38
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    39
* January 2019: Florian Haftmann
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    40
  Renovation of code generation, particularly export into session data and
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    41
  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
    42
69568
de09a7261120 new implementation for case_of_simps based on Code_Lazy's pattern matching elimination algorithm
Andreas Lochbihler
parents: 69205
diff changeset
    43
* January 2019: Andreas Lochbihler
70024
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    44
  New implementation for case_of_simps based on Code_Lazy's pattern matching
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    45
  elimination algorithm.
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    46
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    47
* November/December 2018: Makarius Wenzel
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    48
  Support for Isabelle/Haskell applications of Isabelle/PIDE.
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    49
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    50
* August/September 2018: Makarius Wenzel
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    51
  Improvements of headless Isabelle/PIDE session and server, and systematic
f4843d791e70 more material for release;
wenzelm
parents: 69907
diff changeset
    52
  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
    53
69814
5929b172c6fe CONTRIBUTORS
haftmann
parents: 69791
diff changeset
    54
* December 2018: Florian Haftmann
5929b172c6fe CONTRIBUTORS
haftmann
parents: 69791
diff changeset
    55
  Generic executable sorting algorithms based on executable comparators.
5929b172c6fe CONTRIBUTORS
haftmann
parents: 69791
diff changeset
    56
69205
8050734eee3e add reconstruction by veriT in method smt
fleury <Mathias.Fleury@mpi-inf.mpg.de>
parents: 68683
diff changeset
    57
* October 2018: Mathias Fleury
69814
5929b172c6fe CONTRIBUTORS
haftmann
parents: 69791
diff changeset
    58
  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
    59
68683
d69127c6e80f back to post-release mode -- after fork point;
wenzelm
parents: 68630
diff changeset
    60
68391
9b4f60bdad54 updated for release;
wenzelm
parents: 68246
diff changeset
    61
Contributions to Isabelle2018
9b4f60bdad54 updated for release;
wenzelm
parents: 68246
diff changeset
    62
-----------------------------
66651
435cb8d69e27 back to post-release mode -- after fork point;
wenzelm
parents: 66648
diff changeset
    63
68630
c55f6f0b3854 Added Real_Asymp package
Manuel Eberl <eberlm@in.tum.de>
parents: 68548
diff changeset
    64
* July 2018: Manuel Eberl
c55f6f0b3854 Added Real_Asymp package
Manuel Eberl <eberlm@in.tum.de>
parents: 68548
diff changeset
    65
  "real_asymp" proof method for automatic proofs of real limits, "Big-O"
c55f6f0b3854 Added Real_Asymp package
Manuel Eberl <eberlm@in.tum.de>
parents: 68548
diff changeset
    66
  statements, etc.
c55f6f0b3854 Added Real_Asymp package
Manuel Eberl <eberlm@in.tum.de>
parents: 68548
diff changeset
    67
68522
d9cbc1e8644d example for Types_To_Sets: transfer from type-based linear algebra to subspaces
immler
parents: 68466
diff changeset
    68
* June 2018: Fabian Immler
d9cbc1e8644d example for Types_To_Sets: transfer from type-based linear algebra to subspaces
immler
parents: 68466
diff changeset
    69
  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
    70
68466
3d8241f4198b corrections to markup
paulson <lp15@cam.ac.uk>
parents: 68391
diff changeset
    71
* June 2018: Martin Baillon and Paulo Emílio de Vilhena
3d8241f4198b corrections to markup
paulson <lp15@cam.ac.uk>
parents: 68391
diff changeset
    72
  A variety of contributions to HOL-Algebra.
3d8241f4198b corrections to markup
paulson <lp15@cam.ac.uk>
parents: 68391
diff changeset
    73
68532
f8b98d31ad45 Incorporating new/strengthened proofs from Library and AFP entries
paulson <lp15@cam.ac.uk>
parents: 68522
diff changeset
    74
* June 2018: Wenda Li
f8b98d31ad45 Incorporating new/strengthened proofs from Library and AFP entries
paulson <lp15@cam.ac.uk>
parents: 68522
diff changeset
    75
  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
    76
68545
7922992c99ea misc tuning and updates for release;
wenzelm
parents: 68522
diff changeset
    77
* May/June 2018: Makarius Wenzel
7922992c99ea misc tuning and updates for release;
wenzelm
parents: 68522
diff changeset
    78
  System infrastructure to export blobs as theory presentation, and to dump
7922992c99ea misc tuning and updates for release;
wenzelm
parents: 68522
diff changeset
    79
  PIDE database content in batch mode.
7922992c99ea misc tuning and updates for release;
wenzelm
parents: 68522
diff changeset
    80
68246
b48bab511939 Moved Landau_Symbols from the AFP to HOL-Library
Manuel Eberl <eberlm@in.tum.de>
parents: 68200
diff changeset
    81
* May 2018: Manuel Eberl
68391
9b4f60bdad54 updated for release;
wenzelm
parents: 68246
diff changeset
    82
  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
    83
68073
fad29d2a17a5 merged; resolved conflicts manually (esp. lemmas that have been moved from Linear_Algebra and Cartesian_Euclidean_Space)
immler
parents: 68072 68028
diff changeset
    84
* 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
    85
  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
    86
  Fabian Immler (TUM)
493b818e8e10 added Johannes' generalizations Modules.thy and Vector_Spaces.thy; adapted HOL and HOL-Analysis accordingly
immler
parents: 67928
diff changeset
    87
  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
    88
68028
1f9f973eed2a proper datatype for 8-bit characters
haftmann
parents: 68027
diff changeset
    89
* May 2018: Florian Haftmann
1f9f973eed2a proper datatype for 8-bit characters
haftmann
parents: 68027
diff changeset
    90
  Consolidation of string-like types in HOL.
1f9f973eed2a proper datatype for 8-bit characters
haftmann
parents: 68027
diff changeset
    91
68200
5859c688102a NEWS and CONTRIBUTORS for 8b50f29a1992
Andreas Lochbihler
parents: 68073
diff changeset
    92
* May 2018: Andreas Lochbihler (Digital Asset),
5859c688102a NEWS and CONTRIBUTORS for 8b50f29a1992
Andreas Lochbihler
parents: 68073
diff changeset
    93
  Pascal Stoop (ETH Zurich)
5859c688102a NEWS and CONTRIBUTORS for 8b50f29a1992
Andreas Lochbihler
parents: 68073
diff changeset
    94
  Code generation with lazy evaluation semantics.
5859c688102a NEWS and CONTRIBUTORS for 8b50f29a1992
Andreas Lochbihler
parents: 68073
diff changeset
    95
67928
7f5b1b6f7f40 NEWS and CONTRIBUTORS
haftmann
parents: 67831
diff changeset
    96
* March 2018: Florian Haftmann
68391
9b4f60bdad54 updated for release;
wenzelm
parents: 68246
diff changeset
    97
  Abstract bit operations push_bit, take_bit, drop_bit, alongside with an
9b4f60bdad54 updated for release;
wenzelm
parents: 68246
diff changeset
    98
  algebraic foundation for bit strings and word types in HOL-ex.
67928
7f5b1b6f7f40 NEWS and CONTRIBUTORS
haftmann
parents: 67831
diff changeset
    99
67831
07f5588f2735 Removed stray 'sledgehammer' invocation
Manuel Eberl <eberlm@in.tum.de>
parents: 67456
diff changeset
   100
* March 2018: Viorel Preoteasa
07f5588f2735 Removed stray 'sledgehammer' invocation
Manuel Eberl <eberlm@in.tum.de>
parents: 67456
diff changeset
   101
  Generalisation of complete_distrib_lattice
07f5588f2735 Removed stray 'sledgehammer' invocation
Manuel Eberl <eberlm@in.tum.de>
parents: 67456
diff changeset
   102
68531
7c6f812afdc4 NEWS and CONTRIBUTORS
Wenda Li <wl302@cam.ac.uk>
parents: 68522
diff changeset
   103
* February 2018: Wenda Li
68548
wenzelm
parents: 68547
diff changeset
   104
  A unified definition for the order of zeros and poles. Improved reasoning
wenzelm
parents: 68547
diff changeset
   105
  around non-essential singularities.
68531
7c6f812afdc4 NEWS and CONTRIBUTORS
Wenda Li <wl302@cam.ac.uk>
parents: 68522
diff changeset
   106
67456
7895c159d7b1 added lemma
nipkow
parents: 67279
diff changeset
   107
* January 2018: Sebastien Gouezel
7895c159d7b1 added lemma
nipkow
parents: 67279
diff changeset
   108
  Various small additions to HOL-Analysis
7895c159d7b1 added lemma
nipkow
parents: 67279
diff changeset
   109
67224
341fbce5b26d a conditional paramitrecity prover
traytel
parents: 66893
diff changeset
   110
* December 2017: Jan Gilcher, Andreas Lochbihler, Dmitriy Traytel
67279
d327c11c9f3e spelling
haftmann
parents: 67224
diff changeset
   111
  A new conditional parametricity prover.
67224
341fbce5b26d a conditional paramitrecity prover
traytel
parents: 66893
diff changeset
   112
66893
ced164fe3bbd derived axiom iffI as a lemma (thanks to Alexander Maletzky)
nipkow
parents: 66651
diff changeset
   113
* October 2017: Alexander Maletzky
68391
9b4f60bdad54 updated for release;
wenzelm
parents: 68246
diff changeset
   114
  Derivation of axiom "iff" in theory HOL.HOL from the other axioms.
9b4f60bdad54 updated for release;
wenzelm
parents: 68246
diff changeset
   115
66651
435cb8d69e27 back to post-release mode -- after fork point;
wenzelm
parents: 66648
diff changeset
   116
66475
d8e0fd64216f misc updates for release;
wenzelm
parents: 65330
diff changeset
   117
Contributions to Isabelle2017
66482
wenzelm
parents: 66480
diff changeset
   118
-----------------------------
64439
2bafda87b524 back to post-release mode -- after fork point;
wenzelm
parents: 64433
diff changeset
   119
66648
wenzelm
parents: 66645
diff changeset
   120
* September 2017: Lawrence Paulson
wenzelm
parents: 66645
diff changeset
   121
  HOL-Analysis, e.g. simplicial complexes, Jordan Curve Theorem.
wenzelm
parents: 66645
diff changeset
   122
wenzelm
parents: 66645
diff changeset
   123
* September 2017: Jasmin Blanchette
wenzelm
parents: 66645
diff changeset
   124
  Further integration of Nunchaku model finder.
wenzelm
parents: 66645
diff changeset
   125
66475
d8e0fd64216f misc updates for release;
wenzelm
parents: 65330
diff changeset
   126
* November 2016 - June 2017: Makarius Wenzel
d8e0fd64216f misc updates for release;
wenzelm
parents: 65330
diff changeset
   127
  New Isabelle/VSCode, with underlying restructuring of Isabelle/PIDE.
d8e0fd64216f misc updates for release;
wenzelm
parents: 65330
diff changeset
   128
d8e0fd64216f misc updates for release;
wenzelm
parents: 65330
diff changeset
   129
* 2017: Makarius Wenzel
d8e0fd64216f misc updates for release;
wenzelm
parents: 65330
diff changeset
   130
  Session-qualified theory names (theory imports and ROOT files).
d8e0fd64216f misc updates for release;
wenzelm
parents: 65330
diff changeset
   131
  Prover IDE improvements.
d8e0fd64216f misc updates for release;
wenzelm
parents: 65330
diff changeset
   132
  Support for SQL databases in Isabelle/Scala: SQLite and PostgreSQL.
d8e0fd64216f misc updates for release;
wenzelm
parents: 65330
diff changeset
   133
66563
87b9eb69d5ba add type of unordered pairs
Andreas Lochbihler
parents: 66482
diff changeset
   134
* August 2017: Andreas Lochbihler, ETH Zurich
87b9eb69d5ba add type of unordered pairs
Andreas Lochbihler
parents: 66482
diff changeset
   135
  type of unordered pairs (HOL-Library.Uprod)
87b9eb69d5ba add type of unordered pairs
Andreas Lochbihler
parents: 66482
diff changeset
   136
66480
4b8d1df8933b HOL-Analysis: Convergent FPS and infinite sums
Manuel Eberl <eberlm@in.tum.de>
parents: 66475
diff changeset
   137
* August 2017: Manuel Eberl, TUM
4b8d1df8933b HOL-Analysis: Convergent FPS and infinite sums
Manuel Eberl <eberlm@in.tum.de>
parents: 66475
diff changeset
   138
  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
   139
  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
   140
  power series and analytic complex functions
4b8d1df8933b HOL-Analysis: Convergent FPS and infinite sums
Manuel Eberl <eberlm@in.tum.de>
parents: 66475
diff changeset
   141
65330
d83f709b7580 Corrected affiliation.
ballarin
parents: 65099
diff changeset
   142
* March 2017: Alasdair Armstrong, University of Sheffield and
d83f709b7580 Corrected affiliation.
ballarin
parents: 65099
diff changeset
   143
  Simon Foster, University of York
65099
30d0b2f1df76 Knaster-Tarski fixed point theorem and Galois Connections.
ballarin
parents: 65042
diff changeset
   144
  Fixed-point theory and Galois Connections in HOL-Algebra.
30d0b2f1df76 Knaster-Tarski fixed point theorem and Galois Connections.
ballarin
parents: 65042
diff changeset
   145
65041
2525e680f94f basic documentation for computations
haftmann
parents: 64555
diff changeset
   146
* February 2017: Florian Haftmann, TUM
65042
956ea00a162a more precise NEWS and CONTRIBUTORS
haftmann
parents: 65041
diff changeset
   147
  Statically embedded computations implemented by generated code.
65041
2525e680f94f basic documentation for computations
haftmann
parents: 64555
diff changeset
   148
64439
2bafda87b524 back to post-release mode -- after fork point;
wenzelm
parents: 64433
diff changeset
   149
64072
9f96e4da3064 updated for release;
wenzelm
parents: 64011
diff changeset
   150
Contributions to Isabelle2016-1
9f96e4da3064 updated for release;
wenzelm
parents: 64011
diff changeset
   151
-------------------------------
62216
5fb86150a579 back to post-release mode -- after fork point;
wenzelm
parents: 62205
diff changeset
   152
64551
79e9587dbcca proper session HOL-Types_To_Sets;
wenzelm
parents: 64433
diff changeset
   153
* December 2016: Ondřej Kunčar, TUM
79e9587dbcca proper session HOL-Types_To_Sets;
wenzelm
parents: 64433
diff changeset
   154
  Types_To_Sets: experimental extension of Higher-Order Logic to allow
79e9587dbcca proper session HOL-Types_To_Sets;
wenzelm
parents: 64433
diff changeset
   155
  translation of types to sets.
79e9587dbcca proper session HOL-Types_To_Sets;
wenzelm
parents: 64433
diff changeset
   156
64393
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   157
* October 2016: Jasmin Blanchette
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   158
  Integration of Nunchaku model finder.
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   159
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   160
* October 2016: Jaime Mendizabal Roche, TUM
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   161
  Ported remaining theories of session Old_Number_Theory to the new
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   162
  Number_Theory and removed Old_Number_Theory.
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   163
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   164
* September 2016: Sascha Boehme
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   165
  Proof method "argo" based on SMT technology for a combination of
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   166
  quantifier-free propositional logic, equality and linear real arithmetic
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   167
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   168
* July 2016: Daniel Stuewe
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   169
  Height-size proofs in HOL-Data_Structures.
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   170
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   171
* July 2016: Manuel Eberl, TUM
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   172
  Algebraic foundation for primes; generalization from nat to general
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   173
  factorial rings.
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   174
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   175
* June 2016: Andreas Lochbihler, ETH Zurich
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   176
  Formalisation of discrete subprobability distributions.
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   177
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   178
* June 2016: Florian Haftmann, TUM
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   179
  Improvements to code generation: optional timing measurements, more succint
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   180
  closures for static evaluation, less ambiguities concering Scala implicits.
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   181
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   182
* May 2016: Manuel Eberl, TUM
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   183
  Code generation for Probability Mass Functions.
62343
24106dc44def prefer abbreviations for compound operators INFIMUM and SUPREMUM
haftmann
parents: 62284
diff changeset
   184
64011
54b785efd547 CONTRIBUTORS
haftmann
parents: 63964
diff changeset
   185
* March 2016: Florian Haftmann, TUM
62499
4a5b81ff5992 constructive formulation of factorization
haftmann
parents: 62343
diff changeset
   186
  Abstract factorial rings with unique factorization.
4a5b81ff5992 constructive formulation of factorization
haftmann
parents: 62343
diff changeset
   187
64011
54b785efd547 CONTRIBUTORS
haftmann
parents: 63964
diff changeset
   188
* March 2016: Florian Haftmann, TUM
64393
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   189
  Reworking of the HOL char type as special case of a finite numeral type.
62216
5fb86150a579 back to post-release mode -- after fork point;
wenzelm
parents: 62205
diff changeset
   190
64393
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   191
* March 2016: Andreas Lochbihler, ETH Zurich
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   192
  Reasoning support for monotonicity, continuity and admissibility in
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   193
  chain-complete partial orders.
64011
54b785efd547 CONTRIBUTORS
haftmann
parents: 63964
diff changeset
   194
64393
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   195
* February - October 2016: Makarius Wenzel
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   196
  Prover IDE improvements.
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   197
  ML IDE improvements: bootstrap of Pure.
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   198
  Isar language consolidation.
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   199
  Notational modernization of HOL.
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   200
  Tight Poly/ML integration.
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   201
  More Isabelle/Scala system programming modules (e.g. SSH, Mercurial).
63552
2112e5fe9712 NEWS: Primes
Manuel Eberl <eberlm@in.tum.de>
parents: 63411
diff changeset
   202
64433
d4829dc875fb moved contribution to right release
blanchet
parents: 64393
diff changeset
   203
* Winter 2016: Jasmin Blanchette, Inria & LORIA & MPII, Aymeric Bouzy,
d4829dc875fb moved contribution to right release
blanchet
parents: 64393
diff changeset
   204
  Ecole polytechnique, Andreas Lochbihler, ETH Zurich, Andrei Popescu,
d4829dc875fb moved contribution to right release
blanchet
parents: 64393
diff changeset
   205
  Middlesex University, and Dmitriy Traytel, ETH Zurich
d4829dc875fb moved contribution to right release
blanchet
parents: 64393
diff changeset
   206
  'corec' command and friends.
d4829dc875fb moved contribution to right release
blanchet
parents: 64393
diff changeset
   207
64393
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   208
* January 2016: Florian Haftmann, TUM
17a7543fadad tuned and updated for release;
wenzelm
parents: 64389
diff changeset
   209
  Abolition of compound operators INFIMUM and SUPREMUM for complete lattices.
64389
6273d4c8325b added Nunchaku integration
blanchet
parents: 64363
diff changeset
   210
6273d4c8325b added Nunchaku integration
blanchet
parents: 64363
diff changeset
   211
62016
740c70a21523 misc updates for release;
wenzelm
parents: 61891
diff changeset
   212
Contributions to Isabelle2016
740c70a21523 misc updates for release;
wenzelm
parents: 61891
diff changeset
   213
-----------------------------
60138
b11401808dac back to post-release mode -- after fork point;
wenzelm
parents: 60119
diff changeset
   214
62201
eca7b38c8ee5 Added approximation of powr to NEWS/CONTRIBUTORS
Manuel Eberl <eberlm@in.tum.de>
parents: 62138
diff changeset
   215
* Winter 2016: Manuel Eberl, TUM
eca7b38c8ee5 Added approximation of powr to NEWS/CONTRIBUTORS
Manuel Eberl <eberlm@in.tum.de>
parents: 62138
diff changeset
   216
  Support for real exponentiation ("powr") in the "approximation" method.
62693
0ae225877b68 document addition of 'corec'
blanchet
parents: 62652
diff changeset
   217
  (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
   218
62138
d679e7d500ad crediting LCP in CONTRIBUTORS
paulson <lp15@cam.ac.uk>
parents: 62118
diff changeset
   219
* Summer 2015 - Winter 2016: Lawrence C Paulson, Cambridge
d679e7d500ad crediting LCP in CONTRIBUTORS
paulson <lp15@cam.ac.uk>
parents: 62118
diff changeset
   220
  General, homology form of Cauchy's integral theorem and supporting material
62205
wenzelm
parents: 62201
diff changeset
   221
  (ported from HOL Light).
62138
d679e7d500ad crediting LCP in CONTRIBUTORS
paulson <lp15@cam.ac.uk>
parents: 62118
diff changeset
   222
62118
e60f1a925b4d print_record NEWS and CONTRIBUTORS
kleing
parents: 62098
diff changeset
   223
* Winter 2015/16: Gerwin Klein, NICTA
62205
wenzelm
parents: 62201
diff changeset
   224
  New print_record command.
62118
e60f1a925b4d print_record NEWS and CONTRIBUTORS
kleing
parents: 62098
diff changeset
   225
62236
3a326bc9d4d8 more CONTRIBUTORS;
wenzelm
parents: 62205
diff changeset
   226
* May - December 2015: Makarius Wenzel
3a326bc9d4d8 more CONTRIBUTORS;
wenzelm
parents: 62205
diff changeset
   227
  Prover IDE improvements.
3a326bc9d4d8 more CONTRIBUTORS;
wenzelm
parents: 62205
diff changeset
   228
  More Isar language elements.
3a326bc9d4d8 more CONTRIBUTORS;
wenzelm
parents: 62205
diff changeset
   229
  Document language refinements.
3a326bc9d4d8 more CONTRIBUTORS;
wenzelm
parents: 62205
diff changeset
   230
  Poly/ML debugger integration.
3a326bc9d4d8 more CONTRIBUTORS;
wenzelm
parents: 62205
diff changeset
   231
  Improved multi-platform and multi-architecture support.
3a326bc9d4d8 more CONTRIBUTORS;
wenzelm
parents: 62205
diff changeset
   232
62060
b75764fc4c35 Added summability/Gamma/etc. to NEWS and CONTRIBUTORS
eberlm
parents: 62016
diff changeset
   233
* Winter 2015: Manuel Eberl, TUM
b75764fc4c35 Added summability/Gamma/etc. to NEWS and CONTRIBUTORS
eberlm
parents: 62016
diff changeset
   234
  The radius of convergence of power series and various summability tests.
62064
d9874039786e misc tuning for release;
wenzelm
parents: 62060
diff changeset
   235
  Harmonic numbers and the Euler-Mascheroni constant.
62060
b75764fc4c35 Added summability/Gamma/etc. to NEWS and CONTRIBUTORS
eberlm
parents: 62016
diff changeset
   236
  The Generalised Binomial Theorem.
62064
d9874039786e misc tuning for release;
wenzelm
parents: 62060
diff changeset
   237
  The complex and real Gamma/log-Gamma/Digamma/Polygamma functions and their
d9874039786e misc tuning for release;
wenzelm
parents: 62060
diff changeset
   238
  most important properties.
62138
d679e7d500ad crediting LCP in CONTRIBUTORS
paulson <lp15@cam.ac.uk>
parents: 62118
diff changeset
   239
62086
1c0246456ab9 Added formal power series updates to NEWS/CONTRIBUTORS
Manuel Eberl <eberlm@in.tum.de>
parents: 62084
diff changeset
   240
* Autumn 2015: Manuel Eberl, TUM
1c0246456ab9 Added formal power series updates to NEWS/CONTRIBUTORS
Manuel Eberl <eberlm@in.tum.de>
parents: 62084
diff changeset
   241
  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
   242
  Euclidean Ring and GCD instance for formal power series.
62060
b75764fc4c35 Added summability/Gamma/etc. to NEWS and CONTRIBUTORS
eberlm
parents: 62016
diff changeset
   243
61891
76189756ff65 documentation on last state of the art concerning interpretation
haftmann
parents: 61766
diff changeset
   244
* Autumn 2015: Florian Haftmann, TUM
62064
d9874039786e misc tuning for release;
wenzelm
parents: 62060
diff changeset
   245
  Rewrite definitions for global interpretations and sublocale declarations.
61891
76189756ff65 documentation on last state of the art concerning interpretation
haftmann
parents: 61766
diff changeset
   246
61766
507b39df1a57 add formalisation of Bourbaki-Witt fixpoint theorem
Andreas Lochbihler
parents: 61552
diff changeset
   247
* Autumn 2015: Andreas Lochbihler
62064
d9874039786e misc tuning for release;
wenzelm
parents: 62060
diff changeset
   248
  Bourbaki-Witt fixpoint theorem for increasing functions on chain-complete
d9874039786e misc tuning for release;
wenzelm
parents: 62060
diff changeset
   249
  partial orders.
61766
507b39df1a57 add formalisation of Bourbaki-Witt fixpoint theorem
Andreas Lochbihler
parents: 61552
diff changeset
   250
61552
980dd46a03fb Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
eberlm
parents: 60920
diff changeset
   251
* 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
   252
  A large number of additional binomial identities.
980dd46a03fb Added binomial identities to CONTRIBUTORS; small lemmas on of_int/pochhammer
eberlm
parents: 60920
diff changeset
   253
60632
e096d5aaa0f8 more CONTRIBUTORS;
wenzelm
parents: 60517
diff changeset
   254
* Summer 2015: Daniel Matichuk, NICTA and Makarius Wenzel
62064
d9874039786e misc tuning for release;
wenzelm
parents: 62060
diff changeset
   255
  Isar subgoal command for proof structure within unstructured proof scripts.
60632
e096d5aaa0f8 more CONTRIBUTORS;
wenzelm
parents: 60517
diff changeset
   256
60434
b050b557dbbe CONTRIBUTORS
haftmann
parents: 60301
diff changeset
   257
* Summer 2015: Florian Haftmann, TUM
60632
e096d5aaa0f8 more CONTRIBUTORS;
wenzelm
parents: 60517
diff changeset
   258
  Generic partial division in rings as inverse operation of multiplication.
60434
b050b557dbbe CONTRIBUTORS
haftmann
parents: 60301
diff changeset
   259
60517
f16e4fb20652 separate class for notions specific for integral (semi)domains, in contrast to fields where these are trivial
haftmann
parents: 60434
diff changeset
   260
* Summer 2015: Manuel Eberl and Florian Haftmann, TUM
62064
d9874039786e misc tuning for release;
wenzelm
parents: 62060
diff changeset
   261
  Type class hierarchy with common algebraic notions of integral (semi)domains
d9874039786e misc tuning for release;
wenzelm
parents: 62060
diff changeset
   262
  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
   263
60804
080a979a985b formal class for factorial (semi)rings
haftmann
parents: 60685
diff changeset
   264
* Summer 2015: Florian Haftmann, TUM
080a979a985b formal class for factorial (semi)rings
haftmann
parents: 60685
diff changeset
   265
  Fundamentals of abstract type class for factorial rings.
080a979a985b formal class for factorial (semi)rings
haftmann
parents: 60685
diff changeset
   266
60920
97c20589a0db NEWS, CONTRIBUTORS, documentation for lift_bnf
traytel
parents: 60804
diff changeset
   267
* Summer 2015: Julian Biendarra, TUM and Dmitriy Traytel, ETH Zurich
62064
d9874039786e misc tuning for release;
wenzelm
parents: 62060
diff changeset
   268
  Command to lift a BNF structure on the raw type to the abstract type for
d9874039786e misc tuning for release;
wenzelm
parents: 62060
diff changeset
   269
  typedefs.
60920
97c20589a0db NEWS, CONTRIBUTORS, documentation for lift_bnf
traytel
parents: 60804
diff changeset
   270
62236
3a326bc9d4d8 more CONTRIBUTORS;
wenzelm
parents: 62205
diff changeset
   271
* Summer 2014: Jeremy Avigad, Luke Serafin, CMU, and Johannes Hölzl, TUM
3a326bc9d4d8 more CONTRIBUTORS;
wenzelm
parents: 62205
diff changeset
   272
  Proof of the central limit theorem: includes weak convergence,
3a326bc9d4d8 more CONTRIBUTORS;
wenzelm
parents: 62205
diff changeset
   273
  characteristic functions, and Levy's uniqueness and continuity theorem.
3a326bc9d4d8 more CONTRIBUTORS;
wenzelm
parents: 62205
diff changeset
   274
60138
b11401808dac back to post-release mode -- after fork point;
wenzelm
parents: 60119
diff changeset
   275
60012
0c307c5c03f0 updated for release;
wenzelm
parents: 59980
diff changeset
   276
Contributions to Isabelle2015
0c307c5c03f0 updated for release;
wenzelm
parents: 59980
diff changeset
   277
-----------------------------
57695
987c9ceeaafd back to post-release mode -- after fork point;
wenzelm
parents: 57519
diff changeset
   278
60119
54bea620e54f added Eisbach, using version 3752768caa17 of its Bitbucket repository;
wenzelm
parents: 60012
diff changeset
   279
* 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
   280
  The Eisbach proof method language and "match" method.
54bea620e54f added Eisbach, using version 3752768caa17 of its Bitbucket repository;
wenzelm
parents: 60012
diff changeset
   281
60260
2795bd5e502e CONTRIBUTORS
kuncar
parents: 60119
diff changeset
   282
* Winter 2014 and Spring 2015: Ondrej Kuncar, TUM
60261
wenzelm
parents: 60260
diff changeset
   283
  Extension of lift_definition to execute lifted functions that have as a
wenzelm
parents: 60260
diff changeset
   284
  return type a datatype containing a subtype.
60260
2795bd5e502e CONTRIBUTORS
kuncar
parents: 60119
diff changeset
   285
59980
070f04c94b2e misc tuning for release;
wenzelm
parents: 59813
diff changeset
   286
* March 2015: Jasmin Blanchette, Inria & LORIA & MPII, Mathias Fleury, MPII,
070f04c94b2e misc tuning for release;
wenzelm
parents: 59813
diff changeset
   287
  and Dmitriy Traytel, TUM
59813
6320064f22bb more multiset theorems
blanchet
parents: 59092
diff changeset
   288
  More multiset theorems, syntax, and operations.
6320064f22bb more multiset theorems
blanchet
parents: 59092
diff changeset
   289
59980
070f04c94b2e misc tuning for release;
wenzelm
parents: 59813
diff changeset
   290
* December 2014: Johannes Hölzl, Manuel Eberl, Sudeep Kanav, TUM, and
070f04c94b2e misc tuning for release;
wenzelm
parents: 59813
diff changeset
   291
  Jeremy Avigad, Luke Serafin, CMU
070f04c94b2e misc tuning for release;
wenzelm
parents: 59813
diff changeset
   292
  Various integration theorems: mostly integration on intervals and
070f04c94b2e misc tuning for release;
wenzelm
parents: 59813
diff changeset
   293
  substitution.
59092
d469103c0737 add integral substitution theorems from Manuel Eberl, Jeremy Avigad, Luke Serafin, and Sudeep Kanav
hoelzl
parents: 58626
diff changeset
   294
58196
1b3fbfb85980 theory about lexicographic ordering on functions
haftmann
parents: 58023
diff changeset
   295
* September 2014: Florian Haftmann, TUM
1b3fbfb85980 theory about lexicographic ordering on functions
haftmann
parents: 58023
diff changeset
   296
  Lexicographic order on functions and
1b3fbfb85980 theory about lexicographic ordering on functions
haftmann
parents: 58023
diff changeset
   297
  sum/product over function bodies.
1b3fbfb85980 theory about lexicographic ordering on functions
haftmann
parents: 58023
diff changeset
   298
58626
6c473ed0ac70 move Code_Test to HOL/Library;
Andreas Lochbihler
parents: 58196
diff changeset
   299
* August 2014: Andreas Lochbihler, ETH Zurich
59980
070f04c94b2e misc tuning for release;
wenzelm
parents: 59813
diff changeset
   300
  Test infrastructure for executing generated code in target languages.
58626
6c473ed0ac70 move Code_Test to HOL/Library;
Andreas Lochbihler
parents: 58196
diff changeset
   301
58023
62826b36ac5e generic euclidean algorithm (due to Manuel Eberl)
haftmann
parents: 57882
diff changeset
   302
* August 2014: Manuel Eberl, TUM
59980
070f04c94b2e misc tuning for release;
wenzelm
parents: 59813
diff changeset
   303
  Generic euclidean algorithms for GCD et al.
58023
62826b36ac5e generic euclidean algorithm (due to Manuel Eberl)
haftmann
parents: 57882
diff changeset
   304
57695
987c9ceeaafd back to post-release mode -- after fork point;
wenzelm
parents: 57519
diff changeset
   305
57452
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   306
Contributions to Isabelle2014
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   307
-----------------------------
54055
5bf55a713232 back to post-release mode -- after fork point;
wenzelm
parents: 54051
diff changeset
   308
57513
55b2afc5ddfc added Tom's hyp_subst update
kleing
parents: 57474
diff changeset
   309
* July 2014: Thomas Sewell, NICTA
57516
wenzelm
parents: 57513
diff changeset
   310
  Preserve equality hypotheses in "clarify" and friends. New
wenzelm
parents: 57513
diff changeset
   311
  "hypsubst_thin" method configuration option.
57513
55b2afc5ddfc added Tom's hyp_subst update
kleing
parents: 57474
diff changeset
   312
57519
9e5f47e83629 CONTRIBUTORS
haftmann
parents: 57516
diff changeset
   313
* Summer 2014: Florian Haftmann, TUM
9e5f47e83629 CONTRIBUTORS
haftmann
parents: 57516
diff changeset
   314
  Consolidation and generalization of facts concerning (abelian)
9e5f47e83629 CONTRIBUTORS
haftmann
parents: 57516
diff changeset
   315
  semigroups and monoids, particularly products (resp. sums) on
9e5f47e83629 CONTRIBUTORS
haftmann
parents: 57516
diff changeset
   316
  finite sets.
57419
2b8b1a8587da CONTRIBUTORS
haftmann
parents: 57254
diff changeset
   317
57216
6cd8566e938e updated contributors to include students
blanchet
parents: 57030
diff changeset
   318
* Summer 2014: Mathias Fleury, ENS Rennes, and Albert Steckermeier, TUM
57452
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   319
  Work on exotic automatic theorem provers for Sledgehammer (LEO-II,
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   320
  veriT, Waldmeister, etc.).
57216
6cd8566e938e updated contributors to include students
blanchet
parents: 57030
diff changeset
   321
57875
wenzelm
parents: 57827
diff changeset
   322
* June 2014: Florian Haftmann, TUM
wenzelm
parents: 57827
diff changeset
   323
  Internal reorganisation of the local theory / named target stack.
wenzelm
parents: 57827
diff changeset
   324
57254
d3d91422f408 lemmas about the moments of the normal distribution
hoelzl
parents: 57252
diff changeset
   325
* June 2014: Sudeep Kanav, TUM, Jeremy Avigad, CMU, and Johannes Hölzl, TUM
57452
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   326
  Various properties of exponentially, Erlang, and normal distributed
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   327
  random variables.
57235
b0b9a10e4bf4 properties of Erlang and exponentially distributed random variables (by Sudeep Kanav)
hoelzl
parents: 57216
diff changeset
   328
57452
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   329
* May 2014: Cezary Kaliszyk, University of Innsbruck, and
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   330
  Jasmin Blanchette, TUM
57030
b592202a45cc CONTRIBUTORS
blanchet
parents: 56418
diff changeset
   331
  SML-based engines for MaSh.
b592202a45cc CONTRIBUTORS
blanchet
parents: 56418
diff changeset
   332
55913
c1409c103b77 proper UTF-8;
wenzelm
parents: 55895
diff changeset
   333
* March 2014: René Thiemann
55895
74a2758dcbae added contributor
nipkow
parents: 55316
diff changeset
   334
  Improved code generation for multisets.
74a2758dcbae added contributor
nipkow
parents: 55316
diff changeset
   335
56416
b9baecff0684 CONTRIBUTORS
haftmann
parents: 56118
diff changeset
   336
* February 2014: Florian Haftmann, TUM
57452
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   337
  Permanent interpretation inside theory, locale and class targets
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   338
  with mixin definitions.
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   339
57474
250decee4ac5 for new release
paulson <lp15@cam.ac.uk>
parents: 57452
diff changeset
   340
* Spring 2014: Lawrence C Paulson, Cambridge
250decee4ac5 for new release
paulson <lp15@cam.ac.uk>
parents: 57452
diff changeset
   341
  Theory Complex_Basic_Analysis. Tidying up Number_Theory vs Old_Number_Theory
250decee4ac5 for new release
paulson <lp15@cam.ac.uk>
parents: 57452
diff changeset
   342
57827
abc60f963842 CONTRIBUTORS;
wenzelm
parents: 57519
diff changeset
   343
* Winter 2013 and Spring 2014: Ondrej Kuncar, TUM
abc60f963842 CONTRIBUTORS;
wenzelm
parents: 57519
diff changeset
   344
  Various improvements to Lifting/Transfer, integration with the BNF package.
abc60f963842 CONTRIBUTORS;
wenzelm
parents: 57519
diff changeset
   345
57452
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   346
* Winter 2013 and Spring 2014: Makarius Wenzel, Université Paris-Sud / LRI
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   347
  Improvements of Isabelle/Scala and Isabelle/jEdit Prover IDE.
56416
b9baecff0684 CONTRIBUTORS
haftmann
parents: 56118
diff changeset
   348
57452
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   349
* Fall 2013 and Winter 2014: Martin Desharnais, Lorenz Panny,
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   350
  Dmitriy Traytel, and Jasmin Blanchette, TUM
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   351
  Various improvements to the BNF-based (co)datatype package,
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   352
  including a more polished "primcorec" command, optimizations, and
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   353
  integration in the "HOL" session.
56118
d3967fdc800a updated NEWS and CONTRIBUTORS (BNF, SMT2, Sledgehammer)
blanchet
parents: 55913
diff changeset
   354
57452
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   355
* Winter/Spring 2014: Sascha Boehme, QAware GmbH, and
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   356
  Jasmin Blanchette, TUM
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   357
  "SMT2" module and "smt2" proof method, based on SMT-LIB 2 and
ecad2a53755a misc updates for release;
wenzelm
parents: 57419
diff changeset
   358
  Z3 4.3.
56118
d3967fdc800a updated NEWS and CONTRIBUTORS (BNF, SMT2, Sledgehammer)
blanchet
parents: 55913
diff changeset
   359
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
   360
* 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
   361
  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
   362
  Isabelle/jEdit Prover IDE.
54055
5bf55a713232 back to post-release mode -- after fork point;
wenzelm
parents: 54051
diff changeset
   363
56416
b9baecff0684 CONTRIBUTORS
haftmann
parents: 56118
diff changeset
   364
* December 2013: Florian Haftmann, TUM
b9baecff0684 CONTRIBUTORS
haftmann
parents: 56118
diff changeset
   365
  Consolidation of abstract interpretations concerning min and max.
b9baecff0684 CONTRIBUTORS
haftmann
parents: 56118
diff changeset
   366
b9baecff0684 CONTRIBUTORS
haftmann
parents: 56118
diff changeset
   367
* November 2013: Florian Haftmann, TUM
56418
c267a0feb63a avoid romanism
haftmann
parents: 56416
diff changeset
   368
  Abolition of negative numeral literals in the logic.
56416
b9baecff0684 CONTRIBUTORS
haftmann
parents: 56118
diff changeset
   369
55913
c1409c103b77 proper UTF-8;
wenzelm
parents: 55895
diff changeset
   370
53984
b9139b14c1c5 updated for release;
wenzelm
parents: 53978
diff changeset
   371
Contributions to Isabelle2013-1
b9139b14c1c5 updated for release;
wenzelm
parents: 53978
diff changeset
   372
-------------------------------
50994
aafd4270b4d4 back to post-release mode -- after fork point;
wenzelm
parents: 50993
diff changeset
   373
54363
b0336bb8e638 CONTRIBUTORS
noschinl
parents: 54051
diff changeset
   374
* September 2013: Lars Noschinski, TUM
54364
wenzelm
parents: 54363
diff changeset
   375
  Conversion between function definitions as list of equations and
wenzelm
parents: 54363
diff changeset
   376
  case expressions in HOL.
wenzelm
parents: 54363
diff changeset
   377
  New library Simps_Case_Conv with commands case_of_simps,
wenzelm
parents: 54363
diff changeset
   378
  simps_of_case.
54363
b0336bb8e638 CONTRIBUTORS
noschinl
parents: 54051
diff changeset
   379
53396
5e446969033c more contributors;
wenzelm
parents: 53307
diff changeset
   380
* September 2013: Nik Sultana, University of Cambridge
5e446969033c more contributors;
wenzelm
parents: 53307
diff changeset
   381
  Improvements to HOL/TPTP parser and import facilities.
5e446969033c more contributors;
wenzelm
parents: 53307
diff changeset
   382
54029
4edfd0fd5536 NEWS and CONTRIBUTORS
traytel
parents: 54022
diff changeset
   383
* September 2013: Johannes Hölzl and Dmitriy Traytel, TUM
4edfd0fd5536 NEWS and CONTRIBUTORS
traytel
parents: 54022
diff changeset
   384
  New "coinduction" method (residing in HOL-BNF) to avoid boilerplate.
4edfd0fd5536 NEWS and CONTRIBUTORS
traytel
parents: 54022
diff changeset
   385
53984
b9139b14c1c5 updated for release;
wenzelm
parents: 53978
diff changeset
   386
* Summer 2013: Makarius Wenzel, Université Paris-Sud / LRI
b9139b14c1c5 updated for release;
wenzelm
parents: 53978
diff changeset
   387
  Improvements of Isabelle/Scala and Isabelle/jEdit Prover IDE.
b9139b14c1c5 updated for release;
wenzelm
parents: 53978
diff changeset
   388
53613
cdc780645a49 NEWS and CONTRIBUTORS
krauss
parents: 53396
diff changeset
   389
* Summer 2013: Manuel Eberl, TUM
cdc780645a49 NEWS and CONTRIBUTORS
krauss
parents: 53396
diff changeset
   390
  Generation of elimination rules in the function package.
cdc780645a49 NEWS and CONTRIBUTORS
krauss
parents: 53396
diff changeset
   391
  New command "fun_cases".
cdc780645a49 NEWS and CONTRIBUTORS
krauss
parents: 53396
diff changeset
   392
54051
wenzelm
parents: 54035
diff changeset
   393
* Summer 2013: Christian Sternagel, JAIST
wenzelm
parents: 54035
diff changeset
   394
  Improved support for ad hoc overloading of constants, including
wenzelm
parents: 54035
diff changeset
   395
  documentation and examples.
wenzelm
parents: 54035
diff changeset
   396
53396
5e446969033c more contributors;
wenzelm
parents: 53307
diff changeset
   397
* Spring and Summer 2013: Lorenz Panny, Dmitriy Traytel, and
5e446969033c more contributors;
wenzelm
parents: 53307
diff changeset
   398
  Jasmin Blanchette, TUM
56118
d3967fdc800a updated NEWS and CONTRIBUTORS (BNF, SMT2, Sledgehammer)
blanchet
parents: 55913
diff changeset
   399
  Various improvements to the BNF-based (co)datatype package, including
54010
5ac1495fed4e minor textual changes
blanchet
parents: 53984
diff changeset
   400
  "primrec_new" and "primcorec" commands and a compatibility layer.
53307
221ff2b39a35 updated news/contributors with BNF stuff
blanchet
parents: 53164
diff changeset
   401
54021
8089e82833b6 NEWS and CONTRIBUTORS
kuncar
parents: 54010
diff changeset
   402
* Spring and Summer 2013: Ondrej Kuncar, TUM
54035
wenzelm
parents: 54029
diff changeset
   403
  Various improvements of Lifting and Transfer packages.
54021
8089e82833b6 NEWS and CONTRIBUTORS
kuncar
parents: 54010
diff changeset
   404
8089e82833b6 NEWS and CONTRIBUTORS
kuncar
parents: 54010
diff changeset
   405
* Spring 2013: Brian Huffman, Galois Inc.
54035
wenzelm
parents: 54029
diff changeset
   406
  Improvements of the Transfer package.
54051
wenzelm
parents: 54035
diff changeset
   407
53728
2a25bcd8bf78 updated NEWS and CONTRIBUTORS
blanchet
parents: 53613
diff changeset
   408
* Summer 2013: Daniel Kühlwein, ICIS, Radboud University Nijmegen
2a25bcd8bf78 updated NEWS and CONTRIBUTORS
blanchet
parents: 53613
diff changeset
   409
  Jasmin Blanchette, TUM
2a25bcd8bf78 updated NEWS and CONTRIBUTORS
blanchet
parents: 53613
diff changeset
   410
  Various improvements to MaSh, including a server mode.
2a25bcd8bf78 updated NEWS and CONTRIBUTORS
blanchet
parents: 53613
diff changeset
   411
2a25bcd8bf78 updated NEWS and CONTRIBUTORS
blanchet
parents: 53613
diff changeset
   412
* First half of 2013: Steffen Smolka, TUM
2a25bcd8bf78 updated NEWS and CONTRIBUTORS
blanchet
parents: 53613
diff changeset
   413
  Further improvements to Sledgehammer's Isar proof generator.
2a25bcd8bf78 updated NEWS and CONTRIBUTORS
blanchet
parents: 53613
diff changeset
   414
52485
eed5cbe46f52 CONTRIBUTORS
haftmann
parents: 52266
diff changeset
   415
* May 2013: Florian Haftmann, TUM
eed5cbe46f52 CONTRIBUTORS
haftmann
parents: 52266
diff changeset
   416
  Ephemeral interpretation in local theories.
eed5cbe46f52 CONTRIBUTORS
haftmann
parents: 52266
diff changeset
   417
52266
86d6f57c2c1e NEWS about Spec_Check
bulwahn
parents: 51682
diff changeset
   418
* 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
   419
  Spec_Check: A Quickcheck tool for Isabelle/ML.
52266
86d6f57c2c1e NEWS about Spec_Check
bulwahn
parents: 51682
diff changeset
   420
51682
bdaa1582dc8b NEWS and CONTRIBUTORS
traytel
parents: 51489
diff changeset
   421
* April 2013: Stefan Berghofer, secunet Security Networks AG
bdaa1582dc8b NEWS and CONTRIBUTORS
traytel
parents: 51489
diff changeset
   422
  Dmitriy Traytel, TUM
bdaa1582dc8b NEWS and CONTRIBUTORS
traytel
parents: 51489
diff changeset
   423
  Makarius Wenzel, Université Paris-Sud / LRI
bdaa1582dc8b NEWS and CONTRIBUTORS
traytel
parents: 51489
diff changeset
   424
  Case translations as a separate check phase independent of the
bdaa1582dc8b NEWS and CONTRIBUTORS
traytel
parents: 51489
diff changeset
   425
  datatype package.
bdaa1582dc8b NEWS and CONTRIBUTORS
traytel
parents: 51489
diff changeset
   426
51487
f4bfdee99304 locales for abstract orders
haftmann
parents: 51173
diff changeset
   427
* March 2013: Florian Haftmann, TUM
51489
f738e6dbd844 fundamental revision of big operators on sets
haftmann
parents: 51487
diff changeset
   428
  Reform of "big operators" on sets.
f738e6dbd844 fundamental revision of big operators on sets
haftmann
parents: 51487
diff changeset
   429
f738e6dbd844 fundamental revision of big operators on sets
haftmann
parents: 51487
diff changeset
   430
* March 2013: Florian Haftmann, TUM
51487
f4bfdee99304 locales for abstract orders
haftmann
parents: 51173
diff changeset
   431
  Algebraic locale hierarchy for orderings and (semi)lattices.
f4bfdee99304 locales for abstract orders
haftmann
parents: 51173
diff changeset
   432
52503
wenzelm
parents: 52485
diff changeset
   433
* February 2013: Florian Haftmann, TUM
wenzelm
parents: 52485
diff changeset
   434
  Reworking and consolidation of code generation for target language
wenzelm
parents: 52485
diff changeset
   435
  numerals.
51167
55644f8caeb3 CONTRIBUTORS
haftmann
parents: 50994
diff changeset
   436
52503
wenzelm
parents: 52485
diff changeset
   437
* February 2013: Florian Haftmann, TUM
51173
3cbb4e95a565 Sieve of Eratosthenes
haftmann
parents: 51167
diff changeset
   438
  Sieve of Eratosthenes.
3cbb4e95a565 Sieve of Eratosthenes
haftmann
parents: 51167
diff changeset
   439
51167
55644f8caeb3 CONTRIBUTORS
haftmann
parents: 50994
diff changeset
   440
50993
2c3d0cb151c0 updated for release;
wenzelm
parents: 50991
diff changeset
   441
Contributions to Isabelle2013
2c3d0cb151c0 updated for release;
wenzelm
parents: 50991
diff changeset
   442
-----------------------------
47887
4e9c06c194d9 back to post-release mode -- after fork point;
wenzelm
parents: 47808
diff changeset
   443
49532
6f7cc8e42716 some PIDE NEWS from this summer;
wenzelm
parents: 49510
diff changeset
   444
* 2012: Makarius Wenzel, Université Paris-Sud / LRI
6f7cc8e42716 some PIDE NEWS from this summer;
wenzelm
parents: 49510
diff changeset
   445
  Improvements of Isabelle/Scala and Isabelle/jEdit Prover IDE.
6f7cc8e42716 some PIDE NEWS from this summer;
wenzelm
parents: 49510
diff changeset
   446
50648
3fa343c5bc0a updated for release;
wenzelm
parents: 50573
diff changeset
   447
* Fall 2012: Daniel Kühlwein, ICIS, Radboud University Nijmegen
50222
40e3c3be6bca added file headers
blanchet
parents: 50219
diff changeset
   448
  Jasmin Blanchette, TUM
40e3c3be6bca added file headers
blanchet
parents: 50219
diff changeset
   449
  Implemented Machine Learning for Sledgehammer (MaSh).
40e3c3be6bca added file headers
blanchet
parents: 50219
diff changeset
   450
50219
f6b95f0bba78 updated NEWS etc.
blanchet
parents: 50184
diff changeset
   451
* Fall 2012: Steffen Smolka, TUM
50648
3fa343c5bc0a updated for release;
wenzelm
parents: 50573
diff changeset
   452
  Various improvements to Sledgehammer's Isar proof generator,
3fa343c5bc0a updated for release;
wenzelm
parents: 50573
diff changeset
   453
  including a smart type annotation algorithm and proof shrinking.
50219
f6b95f0bba78 updated NEWS etc.
blanchet
parents: 50184
diff changeset
   454
50573
765c22baa1c9 new contributor
nipkow
parents: 50222
diff changeset
   455
* December 2012: Alessandro Coglio, Kestrel
50991
b3c6c9ef11b8 misc tuning for release;
wenzelm
parents: 50648
diff changeset
   456
  Contributions to HOL's Lattice library.
50573
765c22baa1c9 new contributor
nipkow
parents: 50222
diff changeset
   457
50142
bc82d25af543 CONTRIBUTION: add fabians work
hoelzl
parents: 49770
diff changeset
   458
* November 2012: Fabian Immler, TUM
50184
5a16f42a9b44 more NEWS/CONTRIBUTORS;
wenzelm
parents: 50142
diff changeset
   459
  "Symbols" dockable for Isabelle/jEdit.
5a16f42a9b44 more NEWS/CONTRIBUTORS;
wenzelm
parents: 50142
diff changeset
   460
5a16f42a9b44 more NEWS/CONTRIBUTORS;
wenzelm
parents: 50142
diff changeset
   461
* November 2012: Fabian Immler, TUM
5a16f42a9b44 more NEWS/CONTRIBUTORS;
wenzelm
parents: 50142
diff changeset
   462
  Proof of the Daniell-Kolmogorov theorem: the existence of the limit
5a16f42a9b44 more NEWS/CONTRIBUTORS;
wenzelm
parents: 50142
diff changeset
   463
  of projective families.
50142
bc82d25af543 CONTRIBUTION: add fabians work
hoelzl
parents: 49770
diff changeset
   464
49770
cf6a78acf445 efficient construction of red black trees from sorted associative lists
Andreas Lochbihler
parents: 49532
diff changeset
   465
* October 2012: Andreas Lochbihler, KIT
50184
5a16f42a9b44 more NEWS/CONTRIBUTORS;
wenzelm
parents: 50142
diff changeset
   466
  Efficient construction of red-black trees from sorted associative
5a16f42a9b44 more NEWS/CONTRIBUTORS;
wenzelm
parents: 50142
diff changeset
   467
  lists.
49770
cf6a78acf445 efficient construction of red black trees from sorted associative lists
Andreas Lochbihler
parents: 49532
diff changeset
   468
49190
e1e1d427747d lattice instances for option type
haftmann
parents: 49145
diff changeset
   469
* September 2012: Florian Haftmann, TUM
e1e1d427747d lattice instances for option type
haftmann
parents: 49145
diff changeset
   470
  Lattice instances for type option.
e1e1d427747d lattice instances for option type
haftmann
parents: 49145
diff changeset
   471
49145
0ee5983e3d59 NEWS; CONTRIBUTORS
Christian Sternagel
parents: 48977
diff changeset
   472
* September 2012: Christian Sternagel, JAIST
0ee5983e3d59 NEWS; CONTRIBUTORS
Christian Sternagel
parents: 48977
diff changeset
   473
  Consolidated HOL/Library (theories: Prefix_Order, Sublist, and
0ee5983e3d59 NEWS; CONTRIBUTORS
Christian Sternagel
parents: 48977
diff changeset
   474
  Sublist_Order) w.r.t. prefixes, suffixes, and embedding on lists.
0ee5983e3d59 NEWS; CONTRIBUTORS
Christian Sternagel
parents: 48977
diff changeset
   475
48977
ae12b92c145a updated NEWS and CONTRIBUTORS
blanchet
parents: 48585
diff changeset
   476
* 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
   477
  New BNF-based (co)datatype package.
48977
ae12b92c145a updated NEWS and CONTRIBUTORS
blanchet
parents: 48585
diff changeset
   478
ae12b92c145a updated NEWS and CONTRIBUTORS
blanchet
parents: 48585
diff changeset
   479
* August 2012: Andrei Popescu and Dmitriy Traytel, TUM
ae12b92c145a updated NEWS and CONTRIBUTORS
blanchet
parents: 48585
diff changeset
   480
  Theories of ordinals and cardinals.
ae12b92c145a updated NEWS and CONTRIBUTORS
blanchet
parents: 48585
diff changeset
   481
48585
a82910dd2270 announce advanced support for Isabelle sessions and build management;
wenzelm
parents: 48124
diff changeset
   482
* July 2012: Makarius Wenzel, Université Paris-Sud / LRI
a82910dd2270 announce advanced support for Isabelle sessions and build management;
wenzelm
parents: 48124
diff changeset
   483
  Advanced support for Isabelle sessions and build management, notably
a82910dd2270 announce advanced support for Isabelle sessions and build management;
wenzelm
parents: 48124
diff changeset
   484
  "isabelle build".
a82910dd2270 announce advanced support for Isabelle sessions and build management;
wenzelm
parents: 48124
diff changeset
   485
48111
33414f2e82ab NEWS and CONTRIBUTORS
bulwahn
parents: 47887
diff changeset
   486
* 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
   487
  Simproc for rewriting set comprehensions into pointfree expressions.
47887
4e9c06c194d9 back to post-release mode -- after fork point;
wenzelm
parents: 47808
diff changeset
   488
49481
818bf31759e7 NEWS and CONTRIBUTORS for a5377f6d9f14 and f0ecc1550998
Andreas Lochbihler
parents: 49190
diff changeset
   489
* May 2012: Andreas Lochbihler, KIT
818bf31759e7 NEWS and CONTRIBUTORS for a5377f6d9f14 and f0ecc1550998
Andreas Lochbihler
parents: 49190
diff changeset
   490
  Theory of almost everywhere constant functions.
48124
87c831e30f0a ignore morphism more explicitly;
wenzelm
parents: 48111
diff changeset
   491
50648
3fa343c5bc0a updated for release;
wenzelm
parents: 50573
diff changeset
   492
* 2010-2012: Markus Kaiser and Lukas Bulwahn, TUM
3fa343c5bc0a updated for release;
wenzelm
parents: 50573
diff changeset
   493
  Graphview in Scala/Swing.
3fa343c5bc0a updated for release;
wenzelm
parents: 50573
diff changeset
   494
3fa343c5bc0a updated for release;
wenzelm
parents: 50573
diff changeset
   495
47462
8f85051693d1 some updates for release;
wenzelm
parents: 47448
diff changeset
   496
Contributions to Isabelle2012
8f85051693d1 some updates for release;
wenzelm
parents: 47448
diff changeset
   497
-----------------------------
45109
20b3377b08d7 back to post-release mode;
wenzelm
parents: 44967
diff changeset
   498
47695
89a90da149a9 CONTRIBUTORS
hoelzl
parents: 47567
diff changeset
   499
* April 2012: Johannes Hölzl, TUM
47808
wenzelm
parents: 47700
diff changeset
   500
  Probability: Introduced type to represent measures instead of
wenzelm
parents: 47700
diff changeset
   501
  locales.
47695
89a90da149a9 CONTRIBUTORS
hoelzl
parents: 47567
diff changeset
   502
89a90da149a9 CONTRIBUTORS
hoelzl
parents: 47567
diff changeset
   503
* April 2012: Johannes Hölzl, Fabian Immler, TUM
89a90da149a9 CONTRIBUTORS
hoelzl
parents: 47567
diff changeset
   504
  Float: Moved to Dyadic rationals to represent floating point numers.
89a90da149a9 CONTRIBUTORS
hoelzl
parents: 47567
diff changeset
   505
47808
wenzelm
parents: 47700
diff changeset
   506
* April 2012: Thomas Sewell, NICTA and
wenzelm
parents: 47700
diff changeset
   507
  2010: Sascha Boehme, TUM
wenzelm
parents: 47700
diff changeset
   508
  Theory HOL/Word/WordBitwise: logic/circuit expansion of bitvector
wenzelm
parents: 47700
diff changeset
   509
  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
   510
47808
wenzelm
parents: 47700
diff changeset
   511
* March 2012: Christian Sternagel, JAIST
47448
bulwahn
parents: 47413
diff changeset
   512
  Consolidated theory of relation composition.
bulwahn
parents: 47413
diff changeset
   513
47413
a380515ed7e4 some coverage of HOL/TPTP;
wenzelm
parents: 47265
diff changeset
   514
* March 2012: Nik Sultana, University of Cambridge
a380515ed7e4 some coverage of HOL/TPTP;
wenzelm
parents: 47265
diff changeset
   515
  HOL/TPTP parser and import facilities.
a380515ed7e4 some coverage of HOL/TPTP;
wenzelm
parents: 47265
diff changeset
   516
47462
8f85051693d1 some updates for release;
wenzelm
parents: 47448
diff changeset
   517
* March 2012: Cezary Kaliszyk, University of Innsbruck and
8f85051693d1 some updates for release;
wenzelm
parents: 47448
diff changeset
   518
  Alexander Krauss, QAware GmbH
8f85051693d1 some updates for release;
wenzelm
parents: 47448
diff changeset
   519
  Faster and more scalable Import mechanism for HOL Light proofs.
8f85051693d1 some updates for release;
wenzelm
parents: 47448
diff changeset
   520
47563
01f687b84aff Sledgehammer NEWS and CONTRIBUTORS
blanchet
parents: 47485
diff changeset
   521
* January 2012: Florian Haftmann, TUM, et al.
46596
ef552075d0ef CONTRIBUTORS
haftmann
parents: 45109
diff changeset
   522
  (Re-)Introduction of the "set" type constructor.
ef552075d0ef CONTRIBUTORS
haftmann
parents: 45109
diff changeset
   523
47700
27a04da9c6e6 CONTRIBUTORS
kuncar
parents: 47695
diff changeset
   524
* 2012: Ondrej Kuncar, TUM
47808
wenzelm
parents: 47700
diff changeset
   525
  New package Lifting, various improvements and refinements to the
wenzelm
parents: 47700
diff changeset
   526
  Quotient package.
47700
27a04da9c6e6 CONTRIBUTORS
kuncar
parents: 47695
diff changeset
   527
47563
01f687b84aff Sledgehammer NEWS and CONTRIBUTORS
blanchet
parents: 47485
diff changeset
   528
* 2011/2012: Jasmin Blanchette, TUM
01f687b84aff Sledgehammer NEWS and CONTRIBUTORS
blanchet
parents: 47485
diff changeset
   529
  Various improvements to Sledgehammer, notably: tighter integration
47808
wenzelm
parents: 47700
diff changeset
   530
  with SPASS, support for more provers (Alt-Ergo, iProver,
wenzelm
parents: 47700
diff changeset
   531
  iProver-Eq).
47563
01f687b84aff Sledgehammer NEWS and CONTRIBUTORS
blanchet
parents: 47485
diff changeset
   532
47462
8f85051693d1 some updates for release;
wenzelm
parents: 47448
diff changeset
   533
* 2011/2012: Makarius Wenzel, Université Paris-Sud / LRI
47485
0b4698a31e9a more CONTRIBUTORS;
wenzelm
parents: 47462
diff changeset
   534
  Various refinements of local theory infrastructure.
47462
8f85051693d1 some updates for release;
wenzelm
parents: 47448
diff changeset
   535
  Improvements of Isabelle/Scala layer and Isabelle/jEdit Prover IDE.
47265
b8c98d476805 less modest NEWS; CONTRIBUTORS
krauss
parents: 46596
diff changeset
   536
45109
20b3377b08d7 back to post-release mode;
wenzelm
parents: 44967
diff changeset
   537
44801
a0459c50cfc9 some updates for release;
wenzelm
parents: 41651
diff changeset
   538
Contributions to Isabelle2011-1
a0459c50cfc9 some updates for release;
wenzelm
parents: 41651
diff changeset
   539
-------------------------------
41651
c78b786fe060 back to post-release mode;
wenzelm
parents: 41596
diff changeset
   540
44818
27ba81ad0890 theory of saturated naturals contributed by Peter Gammie
haftmann
parents: 41651
diff changeset
   541
* September 2011: Peter Gammie
44908
f05bff62f8a6 NEWS and CONTRIBUTORS
huffman
parents: 44901
diff changeset
   542
  Theory HOL/Library/Saturated: numbers with saturated arithmetic.
44818
27ba81ad0890 theory of saturated naturals contributed by Peter Gammie
haftmann
parents: 41651
diff changeset
   543
27ba81ad0890 theory of saturated naturals contributed by Peter Gammie
haftmann
parents: 41651
diff changeset
   544
* 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
   545
  Refined theory on complete lattices.
27ba81ad0890 theory of saturated naturals contributed by Peter Gammie
haftmann
parents: 41651
diff changeset
   546
44967
b94c1614e7d5 misc tuning for release;
wenzelm
parents: 44910
diff changeset
   547
* August 2011: Brian Huffman, Portland State University
b94c1614e7d5 misc tuning for release;
wenzelm
parents: 44910
diff changeset
   548
  Miscellaneous cleanup of Complex_Main and Multivariate_Analysis.
b94c1614e7d5 misc tuning for release;
wenzelm
parents: 44910
diff changeset
   549
b94c1614e7d5 misc tuning for release;
wenzelm
parents: 44910
diff changeset
   550
* June 2011: Brian Huffman, Portland State University
b94c1614e7d5 misc tuning for release;
wenzelm
parents: 44910
diff changeset
   551
  Proof method "countable_datatype" for theory Library/Countable.
b94c1614e7d5 misc tuning for release;
wenzelm
parents: 44910
diff changeset
   552
b94c1614e7d5 misc tuning for release;
wenzelm
parents: 44910
diff changeset
   553
* 2011: Jasmin Blanchette, TUM
b94c1614e7d5 misc tuning for release;
wenzelm
parents: 44910
diff changeset
   554
  Various improvements to Sledgehammer, notably: use of sound
b94c1614e7d5 misc tuning for release;
wenzelm
parents: 44910
diff changeset
   555
  translations, support for more provers (Waldmeister, LEO-II,
b94c1614e7d5 misc tuning for release;
wenzelm
parents: 44910
diff changeset
   556
  Satallax). Further development of Nitpick and 'try' command.
b94c1614e7d5 misc tuning for release;
wenzelm
parents: 44910
diff changeset
   557
b94c1614e7d5 misc tuning for release;
wenzelm
parents: 44910
diff changeset
   558
* 2011: Andreas Lochbihler, Karlsruhe Institute of Technology
b94c1614e7d5 misc tuning for release;
wenzelm
parents: 44910
diff changeset
   559
  Theory HOL/Library/Cset_Monad allows do notation for computable sets
b94c1614e7d5 misc tuning for release;
wenzelm
parents: 44910
diff changeset
   560
  (cset) via the generic monad ad-hoc overloading facility.
b94c1614e7d5 misc tuning for release;
wenzelm
parents: 44910
diff changeset
   561
b94c1614e7d5 misc tuning for release;
wenzelm
parents: 44910
diff changeset
   562
* 2011: Johannes Hölzl, Armin Heller, TUM and
b94c1614e7d5 misc tuning for release;
wenzelm
parents: 44910
diff changeset
   563
  Bogdan Grechuk, University of Edinburgh
b94c1614e7d5 misc tuning for release;
wenzelm
parents: 44910
diff changeset
   564
  Theory HOL/Library/Extended_Reals: real numbers extended with plus
b94c1614e7d5 misc tuning for release;
wenzelm
parents: 44910
diff changeset
   565
  and minus infinity.
b94c1614e7d5 misc tuning for release;
wenzelm
parents: 44910
diff changeset
   566
44882
3d853767e5f3 more CONTRIBUTORS;
wenzelm
parents: 44820
diff changeset
   567
* 2011: Makarius Wenzel, Université Paris-Sud / LRI
3d853767e5f3 more CONTRIBUTORS;
wenzelm
parents: 44820
diff changeset
   568
  Various building blocks for Isabelle/Scala layer and Isabelle/jEdit
3d853767e5f3 more CONTRIBUTORS;
wenzelm
parents: 44820
diff changeset
   569
  Prover IDE.
3d853767e5f3 more CONTRIBUTORS;
wenzelm
parents: 44820
diff changeset
   570
44908
f05bff62f8a6 NEWS and CONTRIBUTORS
huffman
parents: 44901
diff changeset
   571
41512
8445396e1e39 updated to Isabelle2011;
wenzelm
parents: 40379
diff changeset
   572
Contributions to Isabelle2011
8445396e1e39 updated to Isabelle2011;
wenzelm
parents: 40379
diff changeset
   573
-----------------------------
37383
22757d15cd86 back to non-release mode;
wenzelm
parents: 37303
diff changeset
   574
41567
72dd2eec64d8 Added entry for HOL-SPARK
berghofe
parents: 41531
diff changeset
   575
* January 2011: Stefan Berghofer, secunet Security Networks AG
72dd2eec64d8 Added entry for HOL-SPARK
berghofe
parents: 41531
diff changeset
   576
  HOL-SPARK: an interactive prover back-end for SPARK.
72dd2eec64d8 Added entry for HOL-SPARK
berghofe
parents: 41531
diff changeset
   577
40379
7ea01f842830 proper spelling;
wenzelm
parents: 40377
diff changeset
   578
* October 2010: Bogdan Grechuk, University of Edinburgh
7ea01f842830 proper spelling;
wenzelm
parents: 40377
diff changeset
   579
  Extended convex analysis in Multivariate Analysis.
7ea01f842830 proper spelling;
wenzelm
parents: 40377
diff changeset
   580
40287
4af3706bcd5d CONTRIBUTORS;
wenzelm
parents: 40120
diff changeset
   581
* October 2010: Dmitriy Traytel, TUM
4af3706bcd5d CONTRIBUTORS;
wenzelm
parents: 40120
diff changeset
   582
  Coercive subtyping via subtype constraints.
4af3706bcd5d CONTRIBUTORS;
wenzelm
parents: 40120
diff changeset
   583
41531
a392a18676e9 CONTRIBUTORS
krauss
parents: 41512
diff changeset
   584
* October 2010: Alexander Krauss, TUM
a392a18676e9 CONTRIBUTORS
krauss
parents: 41512
diff changeset
   585
  Command partial_function for function definitions based on complete
a392a18676e9 CONTRIBUTORS
krauss
parents: 41512
diff changeset
   586
  partial orders in HOL.
a392a18676e9 CONTRIBUTORS
krauss
parents: 41512
diff changeset
   587
39644
ad436fa9fc5b CONTRIBUTORS and NEWS
haftmann
parents: 38656
diff changeset
   588
* September 2010: Florian Haftmann, TUM
41596
e424bc65080d misc updates for release;
wenzelm
parents: 41567
diff changeset
   589
  Refined concepts for evaluation, i.e., normalization of terms using
41531
a392a18676e9 CONTRIBUTORS
krauss
parents: 41512
diff changeset
   590
  different techniques.
40120
c57fffa2727c CONTRIBUTORS
haftmann
parents: 39644
diff changeset
   591
c57fffa2727c CONTRIBUTORS
haftmann
parents: 39644
diff changeset
   592
* September 2010: Florian Haftmann, TUM
39644
ad436fa9fc5b CONTRIBUTORS and NEWS
haftmann
parents: 38656
diff changeset
   593
  Code generation for Scala.
ad436fa9fc5b CONTRIBUTORS and NEWS
haftmann
parents: 38656
diff changeset
   594
38656
d5d342611edb Rewrite the Probability theory.
hoelzl
parents: 38461
diff changeset
   595
* August 2010: Johannes Hoelzl, Armin Heller, and Robert Himmelmann, TUM
41596
e424bc65080d misc updates for release;
wenzelm
parents: 41567
diff changeset
   596
  Improved Probability theory in HOL.
38656
d5d342611edb Rewrite the Probability theory.
hoelzl
parents: 38461
diff changeset
   597
38461
75fc4087764e NEWS and CONTRIBUTORS
haftmann
parents: 37383
diff changeset
   598
* July 2010: Florian Haftmann, TUM
39644
ad436fa9fc5b CONTRIBUTORS and NEWS
haftmann
parents: 38656
diff changeset
   599
  Reworking and extension of the Imperative HOL framework.
38461
75fc4087764e NEWS and CONTRIBUTORS
haftmann
parents: 37383
diff changeset
   600
41596
e424bc65080d misc updates for release;
wenzelm
parents: 41567
diff changeset
   601
* July 2010: Alexander Krauss, TUM and Christian Sternagel, University
e424bc65080d misc updates for release;
wenzelm
parents: 41567
diff changeset
   602
    of Innsbruck
41531
a392a18676e9 CONTRIBUTORS
krauss
parents: 41512
diff changeset
   603
  Ad-hoc overloading. Generic do notation for monads.
a392a18676e9 CONTRIBUTORS
krauss
parents: 41512
diff changeset
   604
37383
22757d15cd86 back to non-release mode;
wenzelm
parents: 37303
diff changeset
   605
37144
fd6308b4df72 misc updates for release;
wenzelm
parents: 36416
diff changeset
   606
Contributions to Isabelle2009-2
41512
8445396e1e39 updated to Isabelle2011;
wenzelm
parents: 40379
diff changeset
   607
-------------------------------
33951
651028e34b5d back to after-release mode;
wenzelm
parents: 33897
diff changeset
   608
37303
0e4c721d4567 CONTRIBUTORS
krauss
parents: 37282
diff changeset
   609
* 2009/2010: Stefan Berghofer, Alexander Krauss, and Andreas Schropp, TUM,
0e4c721d4567 CONTRIBUTORS
krauss
parents: 37282
diff changeset
   610
  Makarius Wenzel, TUM / LRI
0e4c721d4567 CONTRIBUTORS
krauss
parents: 37282
diff changeset
   611
  Elimination of type classes from proof terms.
0e4c721d4567 CONTRIBUTORS
krauss
parents: 37282
diff changeset
   612
37144
fd6308b4df72 misc updates for release;
wenzelm
parents: 36416
diff changeset
   613
* April 2010: Florian Haftmann, TUM
36416
9459be72b89e NEWS and CONTRIBUTORS
haftmann
parents: 33951
diff changeset
   614
  Reorganization of abstract algebra type classes.
9459be72b89e NEWS and CONTRIBUTORS
haftmann
parents: 33951
diff changeset
   615
37144
fd6308b4df72 misc updates for release;
wenzelm
parents: 36416
diff changeset
   616
* April 2010: Florian Haftmann, TUM
36416
9459be72b89e NEWS and CONTRIBUTORS
haftmann
parents: 33951
diff changeset
   617
  Code generation for data representations involving invariants;
9459be72b89e NEWS and CONTRIBUTORS
haftmann
parents: 33951
diff changeset
   618
  various collections avaiable in theories Fset, Dlist, RBT,
9459be72b89e NEWS and CONTRIBUTORS
haftmann
parents: 33951
diff changeset
   619
  Mapping and AssocList.
9459be72b89e NEWS and CONTRIBUTORS
haftmann
parents: 33951
diff changeset
   620
37144
fd6308b4df72 misc updates for release;
wenzelm
parents: 36416
diff changeset
   621
* March 2010: Sascha Boehme, TUM
fd6308b4df72 misc updates for release;
wenzelm
parents: 36416
diff changeset
   622
  Efficient SHA1 library for Poly/ML.
fd6308b4df72 misc updates for release;
wenzelm
parents: 36416
diff changeset
   623
37282
935c75359742 more CONTRIBUTORS;
wenzelm
parents: 37144
diff changeset
   624
* February 2010: Cezary Kaliszyk and Christian Urban, TUM
935c75359742 more CONTRIBUTORS;
wenzelm
parents: 37144
diff changeset
   625
  Quotient type package for Isabelle/HOL.
935c75359742 more CONTRIBUTORS;
wenzelm
parents: 37144
diff changeset
   626
26874
b2daa27fc0a7 misc tuning;
wenzelm
parents: 26728
diff changeset
   627
33842
efa1b89c79e0 misc tuning and updates for official release;
wenzelm
parents: 33759
diff changeset
   628
Contributions to Isabelle2009-1
efa1b89c79e0 misc tuning and updates for official release;
wenzelm
parents: 33759
diff changeset
   629
-------------------------------
33649
854173fcd21c added a tabled implementation of the reflexive transitive closure
bulwahn
parents: 33627
diff changeset
   630
33862
fb95d9152fa9 CONTRIBUTORS
haftmann
parents: 33843
diff changeset
   631
* November 2009, Brian Huffman, PSU
fb95d9152fa9 CONTRIBUTORS
haftmann
parents: 33843
diff changeset
   632
  New definitional domain package for HOLCF.
fb95d9152fa9 CONTRIBUTORS
haftmann
parents: 33843
diff changeset
   633
33759
b369324fc244 Added the contributions of Robert Himmelmann to CONTRIBUTIONS and NEWS
hoelzl
parents: 33649
diff changeset
   634
* November 2009: Robert Himmelmann, TUM
33862
fb95d9152fa9 CONTRIBUTORS
haftmann
parents: 33843
diff changeset
   635
  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
   636
33842
efa1b89c79e0 misc tuning and updates for official release;
wenzelm
parents: 33759
diff changeset
   637
* November 2009: Stefan Berghofer and Lukas Bulwahn, TUM
efa1b89c79e0 misc tuning and updates for official release;
wenzelm
parents: 33759
diff changeset
   638
  A tabled implementation of the reflexive transitive closure.
33649
854173fcd21c added a tabled implementation of the reflexive transitive closure
bulwahn
parents: 33627
diff changeset
   639
33627
ffb4a811e34d announcing the predicate compiler in NEWS and CONTRIBUTORS
bulwahn
parents: 33419
diff changeset
   640
* November 2009: Lukas Bulwahn, TUM
33842
efa1b89c79e0 misc tuning and updates for official release;
wenzelm
parents: 33759
diff changeset
   641
  Predicate Compiler: a compiler for inductive predicates to
33843
23d09560d56d more NEWS, more tuning for release;
wenzelm
parents: 33842
diff changeset
   642
  equational specifications.
48977
ae12b92c145a updated NEWS and CONTRIBUTORS
blanchet
parents: 48585
diff changeset
   643
33897
6db9292f586a tuned affiliation;
wenzelm
parents: 33896
diff changeset
   644
* November 2009: Sascha Boehme, TUM and Burkhart Wolff, LRI Paris
33842
efa1b89c79e0 misc tuning and updates for official release;
wenzelm
parents: 33759
diff changeset
   645
  HOL-Boogie: an interactive prover back-end for Boogie and VCC.
33419
8ae45e87b992 added HOL-Boogie
boehmes
parents: 33203
diff changeset
   646
33192
08a39a957ed7 added Nitpick's theory and ML files to Isabelle/HOL;
blanchet
parents: 33010
diff changeset
   647
* October 2009: Jasmin Blanchette, TUM
33842
efa1b89c79e0 misc tuning and updates for official release;
wenzelm
parents: 33759
diff changeset
   648
  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
   649
33010
39f73a59e855 added proof reconstructon for Z3,
boehmes
parents: 33005
diff changeset
   650
* October 2009: Sascha Boehme, TUM
33182
45f6afe0a979 misc tuning and updates;
wenzelm
parents: 33010
diff changeset
   651
  Extension of SMT method: proof-reconstruction for the SMT solver Z3.
33010
39f73a59e855 added proof reconstructon for Z3,
boehmes
parents: 33005
diff changeset
   652
39f73a59e855 added proof reconstructon for Z3,
boehmes
parents: 33005
diff changeset
   653
* October 2009: Florian Haftmann, TUM
33182
45f6afe0a979 misc tuning and updates;
wenzelm
parents: 33010
diff changeset
   654
  Refinement of parts of the HOL datatype package.
33005
bd8e15958708 CONTRIBUTORS
haftmann
parents: 32762
diff changeset
   655
33010
39f73a59e855 added proof reconstructon for Z3,
boehmes
parents: 33005
diff changeset
   656
* October 2009: Florian Haftmann, TUM
33182
45f6afe0a979 misc tuning and updates;
wenzelm
parents: 33010
diff changeset
   657
  Generic term styles for term antiquotations.
33005
bd8e15958708 CONTRIBUTORS
haftmann
parents: 32762
diff changeset
   658
32762
5f485f98652f Thomas Sewell, NICTA: more efficient HOL/record implementation;
wenzelm
parents: 32618
diff changeset
   659
* September 2009: Thomas Sewell, NICTA
33182
45f6afe0a979 misc tuning and updates;
wenzelm
parents: 33010
diff changeset
   660
  More efficient HOL/record implementation.
32762
5f485f98652f Thomas Sewell, NICTA: more efficient HOL/record implementation;
wenzelm
parents: 32618
diff changeset
   661
32618
42865636d006 added new method "smt": an oracle-based connection to external SMT solvers
boehmes
parents: 32600
diff changeset
   662
* September 2009: Sascha Boehme, TUM
33182
45f6afe0a979 misc tuning and updates;
wenzelm
parents: 33010
diff changeset
   663
  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
   664
32600
1b3b0cc604ce tuned NEWS, added CONTRIBUTORS
haftmann
parents: 32268
diff changeset
   665
* September 2009: Florian Haftmann, TUM
33182
45f6afe0a979 misc tuning and updates;
wenzelm
parents: 33010
diff changeset
   666
  Refinement of sets and lattices.
32600
1b3b0cc604ce tuned NEWS, added CONTRIBUTORS
haftmann
parents: 32268
diff changeset
   667
1b3b0cc604ce tuned NEWS, added CONTRIBUTORS
haftmann
parents: 32268
diff changeset
   668
* July 2009: Jeremy Avigad and Amine Chaieb
33182
45f6afe0a979 misc tuning and updates;
wenzelm
parents: 33010
diff changeset
   669
  New number theory.
32600
1b3b0cc604ce tuned NEWS, added CONTRIBUTORS
haftmann
parents: 32268
diff changeset
   670
32268
d50f0cb67578 Functionality for sum of squares to call a remote csdp prover
Philipp Meyer
parents: 31997
diff changeset
   671
* July 2009: Philipp Meyer, TUM
33182
45f6afe0a979 misc tuning and updates;
wenzelm
parents: 33010
diff changeset
   672
  HOL/Library/Sum_Of_Squares: functionality to call a remote csdp
45f6afe0a979 misc tuning and updates;
wenzelm
parents: 33010
diff changeset
   673
  prover.
32268
d50f0cb67578 Functionality for sum of squares to call a remote csdp prover
Philipp Meyer
parents: 31997
diff changeset
   674
31997
de0d280c31a7 NEWS and CONTRIBUTORS
haftmann
parents: 31466
diff changeset
   675
* July 2009: Florian Haftmann, TUM
33182
45f6afe0a979 misc tuning and updates;
wenzelm
parents: 33010
diff changeset
   676
  New quickcheck implementation using new code generator.
31997
de0d280c31a7 NEWS and CONTRIBUTORS
haftmann
parents: 31466
diff changeset
   677
de0d280c31a7 NEWS and CONTRIBUTORS
haftmann
parents: 31466
diff changeset
   678
* July 2009: Florian Haftmann, TUM
39644
ad436fa9fc5b CONTRIBUTORS and NEWS
haftmann
parents: 38656
diff changeset
   679
  HOL/Library/Fset: an explicit type of sets; finite sets ready to use
33182
45f6afe0a979 misc tuning and updates;
wenzelm
parents: 33010
diff changeset
   680
  for code generation.
31466
48805704ecc6 CONTRIBUTORS
haftmann
parents: 30978
diff changeset
   681
48805704ecc6 CONTRIBUTORS
haftmann
parents: 30978
diff changeset
   682
* June 2009: Florian Haftmann, TUM
33843
23d09560d56d more NEWS, more tuning for release;
wenzelm
parents: 33842
diff changeset
   683
  HOL/Library/Tree: search trees implementing mappings, ready to use
33182
45f6afe0a979 misc tuning and updates;
wenzelm
parents: 33010
diff changeset
   684
  for code generation.
30978
b2da12097761 post Isabelle2009 version;
wenzelm
parents: 30886
diff changeset
   685
32268
d50f0cb67578 Functionality for sum of squares to call a remote csdp prover
Philipp Meyer
parents: 31997
diff changeset
   686
* March 2009: Philipp Meyer, TUM
33843
23d09560d56d more NEWS, more tuning for release;
wenzelm
parents: 33842
diff changeset
   687
  Minimization tool for results from Sledgehammer.
33182
45f6afe0a979 misc tuning and updates;
wenzelm
parents: 33010
diff changeset
   688
32268
d50f0cb67578 Functionality for sum of squares to call a remote csdp prover
Philipp Meyer
parents: 31997
diff changeset
   689
30978
b2da12097761 post Isabelle2009 version;
wenzelm
parents: 30886
diff changeset
   690
Contributions to Isabelle2009
b2da12097761 post Isabelle2009 version;
wenzelm
parents: 30886
diff changeset
   691
-----------------------------
b2da12097761 post Isabelle2009 version;
wenzelm
parents: 30886
diff changeset
   692
30383
ee2c7592e59f more contributors;
wenzelm
parents: 30179
diff changeset
   693
* March 2009: Robert Himmelmann, TUM and Amine Chaieb, University of
ee2c7592e59f more contributors;
wenzelm
parents: 30179
diff changeset
   694
  Cambridge
ee2c7592e59f more contributors;
wenzelm
parents: 30179
diff changeset
   695
  Elementary topology in Euclidean space.
ee2c7592e59f more contributors;
wenzelm
parents: 30179
diff changeset
   696
30886
dda08b76fa99 updated official title of contribution by Johannes Hoelzl;
wenzelm
parents: 30383
diff changeset
   697
* March 2009: Johannes Hoelzl, TUM
dda08b76fa99 updated official title of contribution by Johannes Hoelzl;
wenzelm
parents: 30383
diff changeset
   698
  Method "approximation", which proves real valued inequalities by
dda08b76fa99 updated official title of contribution by Johannes Hoelzl;
wenzelm
parents: 30383
diff changeset
   699
  computation.
dda08b76fa99 updated official title of contribution by Johannes Hoelzl;
wenzelm
parents: 30383
diff changeset
   700
30179
c703c9368c12 A Serbian theory, by Filip Maric.
wenzelm
parents: 30162
diff changeset
   701
* February 2009: Filip Maric, Univ. of Belgrade
c703c9368c12 A Serbian theory, by Filip Maric.
wenzelm
parents: 30162
diff changeset
   702
  A Serbian theory.
c703c9368c12 A Serbian theory, by Filip Maric.
wenzelm
parents: 30162
diff changeset
   703
30162
097673d2e50f more CONTRIBUTORS;
wenzelm
parents: 30154
diff changeset
   704
* February 2009: Jasmin Christian Blanchette, TUM
30154
9193a48d3f95 more CONTRIBUTORS;
wenzelm
parents: 29883
diff changeset
   705
  Misc cleanup of HOL/refute.
9193a48d3f95 more CONTRIBUTORS;
wenzelm
parents: 29883
diff changeset
   706
30162
097673d2e50f more CONTRIBUTORS;
wenzelm
parents: 30154
diff changeset
   707
* February 2009: Timothy Bourke, NICTA
29883
14841d4c808e added find_consts to NEWS and CONTRIBUTORS
kleing
parents: 29861
diff changeset
   708
  New find_consts command.
14841d4c808e added find_consts to NEWS and CONTRIBUTORS
kleing
parents: 29861
diff changeset
   709
30162
097673d2e50f more CONTRIBUTORS;
wenzelm
parents: 30154
diff changeset
   710
* February 2009: Timothy Bourke, NICTA
29861
3c348f5873f3 updated NEWS etc with "solves" criterion and auto_solves
kleing
parents: 29398
diff changeset
   711
  "solves" criterion for find_theorems and auto_solve option
3c348f5873f3 updated NEWS etc with "solves" criterion and auto_solves
kleing
parents: 29398
diff changeset
   712
29398
89813bbf0f3e NEWS and CONTRIBUTORS
haftmann
parents: 29182
diff changeset
   713
* December 2008: Clemens Ballarin, TUM
89813bbf0f3e NEWS and CONTRIBUTORS
haftmann
parents: 29182
diff changeset
   714
  New locale implementation.
89813bbf0f3e NEWS and CONTRIBUTORS
haftmann
parents: 29182
diff changeset
   715
29182
9304afad825e tuned NEWS; CONTRIBUTORS
krauss
parents: 29145
diff changeset
   716
* December 2008: Armin Heller, TUM and Alexander Krauss, TUM
9304afad825e tuned NEWS; CONTRIBUTORS
krauss
parents: 29145
diff changeset
   717
  Method "sizechange" for advanced termination proofs.
9304afad825e tuned NEWS; CONTRIBUTORS
krauss
parents: 29145
diff changeset
   718
28901
028a52be4078 added Tim's find_theorems performance patch
kleing
parents: 28604
diff changeset
   719
* November 2008: Timothy Bourke, NICTA
028a52be4078 added Tim's find_theorems performance patch
kleing
parents: 28604
diff changeset
   720
  Performance improvement (factor 50) for find_theorems.
028a52be4078 added Tim's find_theorems performance patch
kleing
parents: 28604
diff changeset
   721
29398
89813bbf0f3e NEWS and CONTRIBUTORS
haftmann
parents: 29182
diff changeset
   722
* 2008: Florian Haftmann, TUM
89813bbf0f3e NEWS and CONTRIBUTORS
haftmann
parents: 29182
diff changeset
   723
  Various extensions and restructurings in HOL, improvements
89813bbf0f3e NEWS and CONTRIBUTORS
haftmann
parents: 29182
diff changeset
   724
  in evaluation mechanisms, new module binding.ML for name bindings.
89813bbf0f3e NEWS and CONTRIBUTORS
haftmann
parents: 29182
diff changeset
   725
28604
f36496b73227 generic ATP manager based on threads (by Fabian Immler);
wenzelm
parents: 28474
diff changeset
   726
* October 2008: Fabian Immler, TUM
f36496b73227 generic ATP manager based on threads (by Fabian Immler);
wenzelm
parents: 28474
diff changeset
   727
  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
   728
  processes.  Additional ATP wrappers, including remote SystemOnTPTP
f36496b73227 generic ATP manager based on threads (by Fabian Immler);
wenzelm
parents: 28474
diff changeset
   729
  services.
f36496b73227 generic ATP manager based on threads (by Fabian Immler);
wenzelm
parents: 28474
diff changeset
   730
30162
097673d2e50f more CONTRIBUTORS;
wenzelm
parents: 30154
diff changeset
   731
* September 2008: Stefan Berghofer, TUM and Marc Bezem, Univ. Bergen
097673d2e50f more CONTRIBUTORS;
wenzelm
parents: 30154
diff changeset
   732
  Prover for coherent logic.
097673d2e50f more CONTRIBUTORS;
wenzelm
parents: 30154
diff changeset
   733
28474
d0b8b0a1fca5 Vampire wrapper script for remote SystemOnTPTP service (by Fabian Immler);
wenzelm
parents: 27009
diff changeset
   734
* August 2008: Fabian Immler, TUM
d0b8b0a1fca5 Vampire wrapper script for remote SystemOnTPTP service (by Fabian Immler);
wenzelm
parents: 27009
diff changeset
   735
  Vampire wrapper script for remote SystemOnTPTP service.
d0b8b0a1fca5 Vampire wrapper script for remote SystemOnTPTP service (by Fabian Immler);
wenzelm
parents: 27009
diff changeset
   736
d0b8b0a1fca5 Vampire wrapper script for remote SystemOnTPTP service (by Fabian Immler);
wenzelm
parents: 27009
diff changeset
   737
d0b8b0a1fca5 Vampire wrapper script for remote SystemOnTPTP service (by Fabian Immler);
wenzelm
parents: 27009
diff changeset
   738
Contributions to Isabelle2008
d0b8b0a1fca5 Vampire wrapper script for remote SystemOnTPTP service (by Fabian Immler);
wenzelm
parents: 27009
diff changeset
   739
-----------------------------
d0b8b0a1fca5 Vampire wrapper script for remote SystemOnTPTP service (by Fabian Immler);
wenzelm
parents: 27009
diff changeset
   740
27009
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   741
* 2007/2008:
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   742
  Alexander Krauss, TUM and Florian Haftmann, TUM and Stefan Berghofer, TUM
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   743
  HOL library improvements.
25468
d2c618390928 Peter Lammich: HOL-Lattice lemmas;
wenzelm
parents: 25454
diff changeset
   744
27009
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   745
* 2007/2008: Brian Huffman, PSU
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   746
  HOLCF library improvements.
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   747
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   748
* 2007/2008: Stefan Berghofer, TUM
30179
c703c9368c12 A Serbian theory, by Filip Maric.
wenzelm
parents: 30162
diff changeset
   749
  HOL-Nominal package improvements.
27009
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   750
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   751
* March 2008: Markus Reiter, TUM
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   752
  HOL/Library/RBT: red-black trees.
26728
1cfa52844c56 added entries
haftmann
parents: 26198
diff changeset
   753
26874
b2daa27fc0a7 misc tuning;
wenzelm
parents: 26728
diff changeset
   754
* February 2008: Alexander Krauss, TUM and Florian Haftmann, TUM and
b2daa27fc0a7 misc tuning;
wenzelm
parents: 26728
diff changeset
   755
  Lukas Bulwahn, TUM and John Matthews, Galois:
b2daa27fc0a7 misc tuning;
wenzelm
parents: 26728
diff changeset
   756
  HOL/Library/Imperative_HOL: Haskell-style imperative data structures
b2daa27fc0a7 misc tuning;
wenzelm
parents: 26728
diff changeset
   757
  for HOL.
26728
1cfa52844c56 added entries
haftmann
parents: 26198
diff changeset
   758
27009
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   759
* December 2007: Norbert Schirmer, Uni Saarbruecken
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   760
  Misc improvements of record package in HOL.
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   761
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   762
* December 2007: Florian Haftmann, TUM
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   763
  Overloading and class instantiation target.
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   764
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   765
* December 2007: Florian Haftmann, TUM
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   766
  New version of primrec package for local theories.
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   767
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   768
* December 2007: Alexander Krauss, TUM
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   769
  Method "induction_scheme" in HOL.
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   770
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   771
* November 2007: Peter Lammich, Uni Muenster
4f75f2c58123 more contribs;
wenzelm
parents: 26874
diff changeset
   772
  HOL-Lattice: some more lemmas.
26198
865bca530d4c HOL/Library/RBT.thy;
wenzelm
parents: 25468
diff changeset
   773
26874
b2daa27fc0a7 misc tuning;
wenzelm
parents: 26728
diff changeset
   774
25454
wenzelm
parents: 25449
diff changeset
   775
Contributions to Isabelle2007
wenzelm
parents: 25449
diff changeset
   776
-----------------------------
23252
67268bb40b21 Semiring normalization and Groebner Bases.
wenzelm
parents: 22449
diff changeset
   777
25409
b87196bb57da fixed typo;
schirmer
parents: 25398
diff changeset
   778
* October 2007: Norbert Schirmer, TUM / Uni Saarbruecken
25398
35f600d9bf06 HOL-Statespace;
wenzelm
parents: 25057
diff changeset
   779
  State Spaces: The Locale Way (in HOL).
35f600d9bf06 HOL-Statespace;
wenzelm
parents: 25057
diff changeset
   780
25057
021fcbe2aaa5 Mark A. Hillebrand, DFKI: Robust sub/superscripts in LaTeX document output.
wenzelm
parents: 24803
diff changeset
   781
* October 2007: Mark A. Hillebrand, DFKI
021fcbe2aaa5 Mark A. Hillebrand, DFKI: Robust sub/superscripts in LaTeX document output.
wenzelm
parents: 24803
diff changeset
   782
  Robust sub/superscripts in LaTeX document output.
021fcbe2aaa5 Mark A. Hillebrand, DFKI: Robust sub/superscripts in LaTeX document output.
wenzelm
parents: 24803
diff changeset
   783
24799
dff164b6f2a6 misc tuning and update;
wenzelm
parents: 24333
diff changeset
   784
* August 2007: Jeremy Dawson, NICTA and Paul Graunke, Galois and Brian
dff164b6f2a6 misc tuning and update;
wenzelm
parents: 24333
diff changeset
   785
    Huffman, PSU and Gerwin Klein, NICTA and John Matthews, Galois
24333
e77ea0ea7f2c * HOL-Word:
kleing
parents: 24332
diff changeset
   786
  HOL-Word: a library for fixed-size machine words in Isabelle.
e77ea0ea7f2c * HOL-Word:
kleing
parents: 24332
diff changeset
   787
24332
e3a2b75b1cf9 boolean algebras as locales and numbers as types by Brian Huffman
kleing
parents: 23449
diff changeset
   788
* August 2007: Brian Huffman, PSU
24799
dff164b6f2a6 misc tuning and update;
wenzelm
parents: 24333
diff changeset
   789
  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
   790
23252
67268bb40b21 Semiring normalization and Groebner Bases.
wenzelm
parents: 22449
diff changeset
   791
* June 2007: Amine Chaieb, TUM
24799
dff164b6f2a6 misc tuning and update;
wenzelm
parents: 24333
diff changeset
   792
  Semiring normalization and Groebner Bases.
25449
wenzelm
parents: 25409
diff changeset
   793
  Support for dense linear orders.
17866
wenzelm
parents: 17640
diff changeset
   794
23449
dd874e6a3282 integration of Metis prover
paulson
parents: 23382
diff changeset
   795
* June 2007: Joe Hurd, Oxford
24799
dff164b6f2a6 misc tuning and update;
wenzelm
parents: 24333
diff changeset
   796
  Metis theorem-prover.
dff164b6f2a6 misc tuning and update;
wenzelm
parents: 24333
diff changeset
   797
dff164b6f2a6 misc tuning and update;
wenzelm
parents: 24333
diff changeset
   798
* 2007: Kong W. Susanto, Cambridge
dff164b6f2a6 misc tuning and update;
wenzelm
parents: 24333
diff changeset
   799
  HOL: Metis prover integration.
23449
dd874e6a3282 integration of Metis prover
paulson
parents: 23382
diff changeset
   800
24799
dff164b6f2a6 misc tuning and update;
wenzelm
parents: 24333
diff changeset
   801
* 2007: Stefan Berghofer, TUM
25449
wenzelm
parents: 25409
diff changeset
   802
  HOL: inductive predicates and sets.
24799
dff164b6f2a6 misc tuning and update;
wenzelm
parents: 24333
diff changeset
   803
24803
38577b4b1fde Norbert Schirmer: record improvements;
wenzelm
parents: 24799
diff changeset
   804
* 2007: Norbert Schirmer, TUM
38577b4b1fde Norbert Schirmer: record improvements;
wenzelm
parents: 24799
diff changeset
   805
  HOL/record: misc improvements.
38577b4b1fde Norbert Schirmer: record improvements;
wenzelm
parents: 24799
diff changeset
   806
24799
dff164b6f2a6 misc tuning and update;
wenzelm
parents: 24333
diff changeset
   807
* 2006/2007: Alexander Krauss, TUM
dff164b6f2a6 misc tuning and update;
wenzelm
parents: 24333
diff changeset
   808
  HOL: function package and related theories on termination.
23449
dd874e6a3282 integration of Metis prover
paulson
parents: 23382
diff changeset
   809
22449
ece6952a8975 updated
haftmann
parents: 21242
diff changeset
   810
* 2006/2007: Florian Haftmann, TUM
ece6952a8975 updated
haftmann
parents: 21242
diff changeset
   811
  Pure: generic code generator framework.
ece6952a8975 updated
haftmann
parents: 21242
diff changeset
   812
  Pure: class package.
24799
dff164b6f2a6 misc tuning and update;
wenzelm
parents: 24333
diff changeset
   813
  HOL: theory reorganization, code generator setup.
dff164b6f2a6 misc tuning and update;
wenzelm
parents: 24333
diff changeset
   814
25449
wenzelm
parents: 25409
diff changeset
   815
* 2006/2007: Christian Urban, TUM and Stefan Berghofer, TUM and
wenzelm
parents: 25409
diff changeset
   816
    Julien Narboux, TUM
24799
dff164b6f2a6 misc tuning and update;
wenzelm
parents: 24333
diff changeset
   817
  HOL/Nominal package and related tools.
22449
ece6952a8975 updated
haftmann
parents: 21242
diff changeset
   818
21242
d73735bb33c1 * November 2006: Lukas Bulwahn, TUM -- HOL/function: method "lexicographic_order".
wenzelm
parents: 21169
diff changeset
   819
* November 2006: Lukas Bulwahn, TUM
24799
dff164b6f2a6 misc tuning and update;
wenzelm
parents: 24333
diff changeset
   820
  HOL: method "lexicographic_order" for function package.
21242
d73735bb33c1 * November 2006: Lukas Bulwahn, TUM -- HOL/function: method "lexicographic_order".
wenzelm
parents: 21169
diff changeset
   821
21169
b6a5c98c5e38 * October 2006: Stefan Hohe, TUM;
wenzelm
parents: 20340
diff changeset
   822
* October 2006: Stefan Hohe, TUM
b6a5c98c5e38 * October 2006: Stefan Hohe, TUM;
wenzelm
parents: 20340
diff changeset
   823
  HOL-Algebra: ideals and quotients over rings.
b6a5c98c5e38 * October 2006: Stefan Hohe, TUM;
wenzelm
parents: 20340
diff changeset
   824
20340
6afc1c133b86 Amine Chaieb: experimental generic reflection and reification in HOL;
wenzelm
parents: 20067
diff changeset
   825
* August 2006: Amine Chaieb, TUM
6afc1c133b86 Amine Chaieb: experimental generic reflection and reification in HOL;
wenzelm
parents: 20067
diff changeset
   826
  Experimental support for generic reflection and reification in HOL.
6afc1c133b86 Amine Chaieb: experimental generic reflection and reification in HOL;
wenzelm
parents: 20067
diff changeset
   827
20067
26bac504ef90 hex and binary numerals (contributed by Rafal Kolanski)
kleing
parents: 19896
diff changeset
   828
* July 2006: Rafal Kolanski, NICTA
26bac504ef90 hex and binary numerals (contributed by Rafal Kolanski)
kleing
parents: 19896
diff changeset
   829
  Hex (0xFF) and binary (0b1011) numerals.
26bac504ef90 hex and binary numerals (contributed by Rafal Kolanski)
kleing
parents: 19896
diff changeset
   830
19896
286d950883bc *** empty log message ***
nipkow
parents: 19650
diff changeset
   831
* May 2006: Klaus Aehlig, LMU
286d950883bc *** empty log message ***
nipkow
parents: 19650
diff changeset
   832
  Command 'normal_form': normalization by evaluation.
286d950883bc *** empty log message ***
nipkow
parents: 19650
diff changeset
   833
19650
33a94c5fc7bb Amine Chaieb: Ferrante and Rackoff Algorithm;
wenzelm
parents: 19470
diff changeset
   834
* May 2006: Amine Chaieb, TUM
33a94c5fc7bb Amine Chaieb: Ferrante and Rackoff Algorithm;
wenzelm
parents: 19470
diff changeset
   835
  HOL-Complex: Ferrante and Rackoff Algorithm for linear real
33a94c5fc7bb Amine Chaieb: Ferrante and Rackoff Algorithm;
wenzelm
parents: 19470
diff changeset
   836
  arithmetic.
19470
3572af78f114 added Ben Porter's stuff
kleing
parents: 17866
diff changeset
   837
3572af78f114 added Ben Porter's stuff
kleing
parents: 17866
diff changeset
   838
* February 2006: Benjamin Porter, NICTA
23382
0459ab90389a clarified who we consider to be a contributor
kleing
parents: 23252
diff changeset
   839
  HOL and HOL-Complex: generalised mean value theorem, continuum is
19470
3572af78f114 added Ben Porter's stuff
kleing
parents: 17866
diff changeset
   840
  not denumerable, harmonic and arithmetic series, and denumerability
3572af78f114 added Ben Porter's stuff
kleing
parents: 17866
diff changeset
   841
  of rationals.
17532
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   842
19650
33a94c5fc7bb Amine Chaieb: Ferrante and Rackoff Algorithm;
wenzelm
parents: 19470
diff changeset
   843
* October 2005: Martin Wildmoser, TUM
33a94c5fc7bb Amine Chaieb: Ferrante and Rackoff Algorithm;
wenzelm
parents: 19470
diff changeset
   844
  Sketch for Isar 'guess' element.
33a94c5fc7bb Amine Chaieb: Ferrante and Rackoff Algorithm;
wenzelm
parents: 19470
diff changeset
   845
33a94c5fc7bb Amine Chaieb: Ferrante and Rackoff Algorithm;
wenzelm
parents: 19470
diff changeset
   846
25454
wenzelm
parents: 25449
diff changeset
   847
Contributions to Isabelle2005
wenzelm
parents: 25449
diff changeset
   848
-----------------------------
17382
32a165db45ea Bernhard Haeupler: comm_ring;
wenzelm
parents: 16892
diff changeset
   849
17640
wenzelm
parents: 17572
diff changeset
   850
* September 2005: Lukas Bulwahn and Bernhard Haeupler, TUM
wenzelm
parents: 17572
diff changeset
   851
  HOL-Complex: Formalization of Taylor series.
wenzelm
parents: 17572
diff changeset
   852
wenzelm
parents: 17572
diff changeset
   853
* September 2005: Stephan Merz, Alwen Tiu, QSL Loria
wenzelm
parents: 17572
diff changeset
   854
  Components for SAT solver method using zChaff.
wenzelm
parents: 17572
diff changeset
   855
17534
56e8db202f66 HOL/ex/Chinese.thy;
wenzelm
parents: 17532
diff changeset
   856
* September 2005: Ning Zhang and Christian Urban, LMU Munich
56e8db202f66 HOL/ex/Chinese.thy;
wenzelm
parents: 17532
diff changeset
   857
  A Chinese theory.
56e8db202f66 HOL/ex/Chinese.thy;
wenzelm
parents: 17532
diff changeset
   858
17562
wenzelm
parents: 17543
diff changeset
   859
* September 2005: Bernhard Haeupler, TUM
17382
32a165db45ea Bernhard Haeupler: comm_ring;
wenzelm
parents: 16892
diff changeset
   860
  Method comm_ring for proving equalities in commutative rings.
16892
23887fee6071 more contribs;
wenzelm
parents: 16869
diff changeset
   861
17532
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   862
* July/August 2005: Jeremy Avigad, Carnegie Mellon University
16892
23887fee6071 more contribs;
wenzelm
parents: 16869
diff changeset
   863
  Various improvements of the HOL and HOL-Complex library.
16868
eaafda56b14c *** empty log message ***
wenzelm
parents: 16252
diff changeset
   864
16892
23887fee6071 more contribs;
wenzelm
parents: 16869
diff changeset
   865
* July 2005: Florian Zuleger, Johannes Hoelzl, and Simon Funke, TUM
23887fee6071 more contribs;
wenzelm
parents: 16869
diff changeset
   866
  Some structured proofs about completeness of real numbers.
23887fee6071 more contribs;
wenzelm
parents: 16869
diff changeset
   867
17532
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   868
* May 2005: Rafal Kolanski and Gerwin Klein, NICTA
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   869
  Improved retrieval of facts from theory/proof context.
15994
dd9023d84f44 proper Id line;
wenzelm
parents: 15993
diff changeset
   870
16252
8cddc62ed170 Lucas Dixon;
wenzelm
parents: 15994
diff changeset
   871
* February 2005: Lucas Dixon, University of Edinburgh
17532
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   872
  Improved subst method.
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   873
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   874
* 2005: Brian Huffman, OGI
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   875
  Various improvements of HOLCF.
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   876
  Some improvements of the HOL-Complex library.
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   877
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   878
* 2005: Claire Quigley and Jia Meng, University of Cambridge
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   879
  Some support for asynchronous communication with external provers
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   880
  (experimental).
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   881
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   882
* 2005: Florian Haftmann, TUM
17543
wenzelm
parents: 17534
diff changeset
   883
  Contributions to document 'sugar'.
17532
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   884
  Various ML combinators, notably linear functional transformations.
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   885
  Some cleanup of ML legacy.
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   886
  Additional antiquotations.
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   887
  Improved Isabelle web site.
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   888
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   889
* 2004/2005: David Aspinall, University of Edinburgh
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   890
  Various elements of XML and PGIP based communication with user
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   891
  interfaces (experimental).
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   892
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   893
* 2004/2005: Gerwin Klein, NICTA
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   894
  Contributions to document 'sugar'.
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   895
  Improved Isabelle web site.
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   896
  Improved HTML presentation of theories.
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   897
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   898
* 2004/2005: Clemens Ballarin, TUM
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   899
  Provers: tools for transitive relations and quasi orders.
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   900
  Improved version of locales, notably interpretation of locales.
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   901
  Improved version of HOL-Algebra.
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   902
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   903
* 2004/2005: Amine Chaieb, TUM
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   904
  Improved version of HOL presburger method.
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   905
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   906
* 2004/2005: Steven Obua, TUM
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   907
  Improved version of HOL/Import, support for HOL-Light.
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   908
  Improved version of HOL-Complex-Matrix.
17572
wenzelm
parents: 17562
diff changeset
   909
  Pure/defs: more sophisticated checks on well-formedness of overloading.
17543
wenzelm
parents: 17534
diff changeset
   910
  Pure/Tools: an experimental evaluator for lambda terms.
17532
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   911
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   912
* 2004/2005: Norbert Schirmer, TUM
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   913
  Contributions to document 'sugar'.
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   914
  Improved version of HOL/record.
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   915
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   916
* 2004/2005: Sebastian Skalberg, TUM
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   917
  Improved version of HOL/Import.
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   918
  Some internal ML reorganizations.
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   919
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   920
* 2004/2005: Tjark Weber, TUM
17640
wenzelm
parents: 17572
diff changeset
   921
  SAT solver method using zChaff.
17532
ab75f2b0cec6 more contributions;
wenzelm
parents: 17382
diff changeset
   922
  Improved version of HOL/refute.
62098
wenzelm
parents: 62086
diff changeset
   923
wenzelm
parents: 62086
diff changeset
   924
:maxLineLen=78: