Page MenuHomeIsabelle/Phabricator

No OneTemporary

This file is larger than 256 KB, so syntax highlighting was skipped.
diff --git a/admin/site/content/about.md b/admin/site/content/about.md
--- a/admin/site/content/about.md
+++ b/admin/site/content/about.md
@@ -1,54 +1,58 @@
---
title: "About"
-menu:
+menu:
main:
name: "About"
weight: 7
---
The Archive of Formal Proofs is a collection of proof libraries, examples, and larger scientific developments,
mechanically checked in the theorem prover Isabelle.
It is organized in the way of a scientific journal.
[Submissions](/submission) are refereed.
The archive repository is hosted on [Heptapod](https://foss.heptapod.net/isa-afp/) to provide easy free access to archive entries.
The entries are tested and maintained continuously against the current stable release of Isabelle.
Older versions of archive entries will remain available.
## Editors
The editors of the Archive of Formal Proofs are:
-* [Manuel Eberl](https://www.in.tum.de/~eberlm/), [Technische Universität München](https://www.tum.de/)
-* [Gerwin Klein](https://www.cse.unsw.edu.au/~kleing/), [Data61](https://www.data61.csiro.au)
-* [Tobias Nipkow](https://www.in.tum.de/~nipkow/), [Technische Universität München](https://www.tum.de/)
-* [Larry Paulson](https://www.cl.cam.ac.uk/users/lcp/), [University of Cambridge](https://www.cam.ac.uk/)
-* [René Thiemann](http://cl-informatik.uibk.ac.at/users/thiemann/), [University of Innsbruck](https://www.uibk.ac.at/)
+* [Manuel Eberl](http://pruvisto.org/), [University of Innsbruck](https://www.uibk.ac.at/)
+* [Gerwin Klein](https://www.cse.unsw.edu.au/~kleing/), [Proofcraft](https://proofcraft.systems) & [UNSW Sydney](https://www.unsw.edu.au/)
+* [Andreas Lochbihler](http://www.andreas-lochbihler.de),
+ [Digital Asset](https://www.digitalasset.com)
+* [Tobias Nipkow](https://www.in.tum.de/~nipkow/), [Technische Universität München](https://www.tum.de/)
+* [Larry Paulson](https://www.cl.cam.ac.uk/users/lcp/), [University of Cambridge](https://www.cam.ac.uk/)
+* [René Thiemann](http://cl-informatik.uibk.ac.at/users/thiemann/), [University of Innsbruck](https://www.uibk.ac.at/)
## Why
We aim to strengthen the community and to foster the development of formal proofs.
We hope that the Archive will provide:
-* a resource of knowledge, examples, and libraries for users,
-* a large and relevant test bed of theories for Isabelle developers, and
-* a central, citable place for authors to publish their theories
+* a resource of knowledge, examples, and libraries for users,
+* a large and relevant test bed of theories for Isabelle developers, and
+* a central, citable place for authors to publish their theories
We encourage authors of publications that contain Isabelle developments to make their theories available in the Archive of Formal Proofs and to refer to the archive entry in their publication. It makes it easier for referees to check the validity of theorems (all entries in the Archive are mechanically checked), it makes it easier for readers of the publication to understand details of your development, and it makes it easier to use and build on your work.
## License
All entries in the Archive of Formal Proofs are licensed under a [BSD-style License](LICENSE) or the [GNU LGPL](https://www.gnu.org/copyleft/lesser.html). This means they are free to download, free to use, free to change, and free to redistribute with minimal restrictions.
The authors retain their full copyright on their original work, including their right to make the development available under another, additional license in the future.
## Website
This website is the result of a project from the School of Informatics at the [University of Edinburgh](https://www.ed.ac.uk) by:
- * Carlin MacKenzie, [AIML](https://aiml.inf.ed.ac.uk)
- * James Vaughan, [AIAI](https://web.inf.ed.ac.uk/aiai/)
- * Jacques Fleuriot, [AIAI](https://web.inf.ed.ac.uk/aiai/)
+
+* Carlin MacKenzie, [AIML](https://aiml.inf.ed.ac.uk)
+* James Vaughan, [AIAI](https://web.inf.ed.ac.uk/aiai/)
+* Jacques Fleuriot, [AIAI](https://web.inf.ed.ac.uk/aiai/)
Integration and maintenance by:
- * [Fabian Huch](https://www21.in.tum.de/team/huch), [Technische Universität München](https://www.tum.de/)
+
+* [Fabian Huch](https://www21.in.tum.de/team/huch), [Technische Universität München](https://www.tum.de/)
diff --git a/admin/site/content/help.md b/admin/site/content/help.md
--- a/admin/site/content/help.md
+++ b/admin/site/content/help.md
@@ -1,62 +1,62 @@
---
title: Help
-menu:
+menu:
main:
name: "Help"
weight: 4
---
This section focuses on the Archive of Formal Proofs. For help with Isabelle, see the [Isabelle Wiki](https://isabelle.in.tum.de/community/Main_Page) and [Documentation](https://isabelle.in.tum.de/documentation.html)
## Referring to AFP Entries in Isabelle/JEdit
Once you have downloaded the AFP, you can include its articles and theories in your own developments. If you would like to make your work available to others _without_ having to include the AFP articles you depend on, here is how to do it.
-From Isabelle2021 on, the recommended method for making the whole AFP available to Isabelle is the `isabelle components -u` command.
+From Isabelle2021-1 on, the recommended method for making the whole AFP available to Isabelle is the `isabelle components -u` command.
#### Linux and Mac
Assuming you have downloaded and unzipped the afp to `/home/myself/afp`, run:
- isabelle components -u /home/myself/afp
+ isabelle components -u /home/myself/afp/thys
#### Windows
If the AFP is in `C:\afp`, run the following command in a Cygwin terminal:
- isabelle components -u /cygdrive/c/afp
+ isabelle components -u /cygdrive/c/afp/thys
#### Use
You can now refer to article `ABC` from the AFP in another theory via:
imports "ABC.Some_ABC_Theory"
This allows you to distribute your material separately from any AFP theories. Users of your distribution also need to install the AFP in the above manner.
## Citing Entries
The following gives an example of the preferred way for citing entries in the AFP:
> M. Jaskelioff and S. Merz, Proving the Correctness of Disk Paxos. _Archive of Formal Proofs_, June 2005, [https://isa-afp.org/entries/DiskPaxos.html](https://isa-afp.org/entries/DiskPaxos.html), Formal proof development.
-The bibtext entry for this would be:
+The bibtex entry for this would be:
```
@article{Jaskelioff-Merz-AFP05,
author = {Mauro Jaskelioff and Stephan Merz},
title = {Proving the Correctness of Disk Paxos},
journal = {Archive of Formal Proofs},
month = Jun,
year = 2005,
note = {\\url{https://isa-afp.org/entries/DiskPaxos.html}, Formal proof development},
ISSN = {2150-914x}
}
```
## Mailing Lists
* isabelle-users@cl.cam.ac.uk provides a forum for Isabelle users to discuss problems, exchange information, and make announcements. Users of official Isabelle releases should subscribe or see the archive.
-
+
* isabelle-dev@in.tum.de covers the Isabelle development process, including intermediate repository versions, and administrative issues concerning the website or testing infrastructure. Early adopters of development snapshots or repository versions should subscribe or see the archive (also available at mail-archive.com).
diff --git a/metadata/authors.toml b/metadata/authors.toml
--- a/metadata/authors.toml
+++ b/metadata/authors.toml
@@ -1,3486 +1,3495 @@
[lange]
name = "Christoph Lange"
[lange.emails]
lange_email = "math.semantic.web@gmail.com"
[lange.homepages]
[petrovic]
name = "Danijela Petrovic"
[petrovic.emails]
[petrovic.homepages]
petrovic_homepage = "http://www.matf.bg.ac.rs/~danijela"
[schimpf]
name = "Alexander Schimpf"
[schimpf.emails]
schimpf_email = "schimpfa@informatik.uni-freiburg.de"
[schimpf.homepages]
[murao]
name = "H. Murao"
[murao.emails]
[murao.homepages]
[bourke]
name = "Timothy Bourke"
[bourke.emails]
bourke_email = "tim@tbrk.org"
[bourke.homepages]
bourke_homepage = "http://www.tbrk.org"
[schaeffeler]
name = "Maximilian Schäffeler"
[schaeffeler.emails]
schaeffeler_email = "schaeffm@in.tum.de"
[schaeffeler.homepages]
[liut]
name = "Tao Liu"
[liut.emails]
[liut.homepages]
[sickert]
name = "Salomon Sickert"
[sickert.emails]
sickert_email = "s.sickert@tum.de"
[sickert.homepages]
sickert_homepage = "https://www7.in.tum.de/~sickert"
[lutz]
name = "Bianca Lutz"
[lutz.emails]
lutz_email = "sowilo@cs.tu-berlin.de"
[lutz.homepages]
[rizkallah]
name = "Christine Rizkallah"
[rizkallah.emails]
[rizkallah.homepages]
rizkallah_homepage = "https://www.mpi-inf.mpg.de/~crizkall/"
[pollak]
name = "Florian Pollak"
[pollak.emails]
pollak_email = "florian.pollak@gmail.com"
[pollak.homepages]
[sulejmani]
name = "Ujkan Sulejmani"
[sulejmani.emails]
[sulejmani.homepages]
[biendarra]
name = "Julian Biendarra"
[biendarra.emails]
[biendarra.homepages]
[saile]
name = "Christian Saile"
[saile.emails]
[saile.homepages]
saile_homepage = "http://dss.in.tum.de/staff/christian-saile.html"
[friedrich]
name = "Stefan Friedrich"
[friedrich.emails]
[friedrich.homepages]
[maximova]
name = "Alexandra Maximova"
[maximova.emails]
maximova_email = "amaximov@student.ethz.ch"
[maximova.homepages]
[stricker]
name = "Christian Stricker"
[stricker.emails]
[stricker.homepages]
stricker_homepage = "http://dss.in.tum.de/staff/christian-stricker.html"
[dyckhoff]
name = "Roy Dyckhoff"
[dyckhoff.emails]
[dyckhoff.homepages]
dyckhoff_homepage = "https://rd.host.cs.st-andrews.ac.uk"
[weidner]
name = "Arno Wilhelm-Weidner"
[weidner.emails]
weidner_email = "arno.wilhelm-weidner@tu-berlin.de"
[weidner.homepages]
[thomson]
name = "Fox Thomson"
[thomson.emails]
thomson_email = "foxthomson0@gmail.com"
[thomson.homepages]
[he]
name = "Yijun He"
[he.emails]
he_email = "yh403@cam.ac.uk"
[he.homepages]
[kammueller]
name = "Florian Kammüller"
[kammueller.emails]
kammueller_email = "flokam@cs.tu-berlin.de"
kammueller_email1 = "florian.kammuller@gmail.com"
[kammueller.homepages]
kammueller_homepage = "http://www.cs.mdx.ac.uk/people/florian-kammueller/"
[oostrom]
name = "Vincent van Oostrom"
[oostrom.emails]
[oostrom.homepages]
[klein]
name = "Gerwin Klein"
[klein.emails]
klein_email = "kleing@unsw.edu.au"
[klein.homepages]
klein_homepage = "http://www.cse.unsw.edu.au/~kleing/"
[simic]
name = "Danijela Simić"
[simic.emails]
simic_email = "danijela@matf.bg.ac.rs"
[simic.homepages]
simic_homepage = "http://poincare.matf.bg.ac.rs/~danijela"
[gao]
name = "Xin Gao"
[gao.emails]
[gao.homepages]
[guttmann]
name = "Walter Guttmann"
[guttmann.emails]
guttmann_email = "walter.guttmann@canterbury.ac.nz"
[guttmann.homepages]
guttmann_homepage = "https://www.cosc.canterbury.ac.nz/walter.guttmann/"
[mantel]
name = "Heiko Mantel"
[mantel.emails]
mantel_email = "mantel@mais.informatik.tu-darmstadt.de"
[mantel.homepages]
[schlichtkrull]
name = "Anders Schlichtkrull"
[schlichtkrull.emails]
schlichtkrull_email = "andschl@dtu.dk"
[schlichtkrull.homepages]
schlichtkrull_homepage = "https://people.compute.dtu.dk/andschl/"
[jaskolka]
name = "Jason Jaskolka"
[jaskolka.emails]
jaskolka_email = "jason.jaskolka@carleton.ca"
[jaskolka.homepages]
jaskolka_homepage = "https://carleton.ca/jaskolka/"
[rau]
name = "Martin Rau"
[rau.emails]
rau_email = "martin.rau@tum.de"
rau_email1 = "mrtnrau@googlemail.com"
[rau.homepages]
[bottesch]
name = "Ralph Bottesch"
[bottesch.emails]
bottesch_email = "ralph.bottesch@uibk.ac.at"
[bottesch.homepages]
bottesch_homepage = "http://cl-informatik.uibk.ac.at/users/bottesch/"
[bella]
name = "Giampaolo Bella"
[bella.emails]
bella_email = "giamp@dmi.unict.it"
[bella.homepages]
bella_homepage = "http://www.dmi.unict.it/~giamp/"
[dirix]
name = "Stefan Dirix"
[dirix.emails]
[dirix.homepages]
[nielsen]
name = "Finn Nielsen"
[nielsen.emails]
nielsen_email = "finn.nielsen@uni-muenster.de"
[nielsen.homepages]
[mansky]
name = "Susannah Mansky"
[mansky.emails]
mansky_email = "sjohnsn2@illinois.edu"
mansky_email1 = "susannahej@gmail.com"
[mansky.homepages]
[dunaev]
name = "Georgy Dunaev"
[dunaev.emails]
dunaev_email = "georgedunaev@gmail.com"
[dunaev.homepages]
[li]
name = "Wenda Li"
[li.emails]
li_email = "wl302@cam.ac.uk"
li_email1 = "liwenda1990@hotmail.com"
[li.homepages]
li_homepage = "https://www.cl.cam.ac.uk/~wl302/"
[stevens]
name = "Lukas Stevens"
[stevens.emails]
[stevens.homepages]
stevens_homepage = "https://www21.in.tum.de/team/stevensl"
[tourret]
name = "Sophie Tourret"
[tourret.emails]
tourret_email = "stourret@mpi-inf.mpg.de"
[tourret.homepages]
tourret_homepage = "https://www.mpi-inf.mpg.de/departments/automation-of-logic/people/sophie-tourret/"
[yu]
name = "Lei Yu"
[yu.emails]
yu_email = "ly271@cam.ac.uk"
[yu.homepages]
[grewe]
name = "Sylvia Grewe"
[grewe.emails]
grewe_email = "grewe@cs.tu-darmstadt.de"
[grewe.homepages]
[coghetto]
name = "Roland Coghetto"
[coghetto.emails]
coghetto_email = "roland_coghetto@hotmail.com"
[coghetto.homepages]
[schirmer]
name = "Norbert Schirmer"
[schirmer.emails]
schirmer_email = "norbert.schirmer@web.de"
[schirmer.homepages]
[immler]
name = "Fabian Immler"
[immler.emails]
immler_email = "immler@in.tum.de"
immler_email1 = "fimmler@cs.cmu.edu"
[immler.homepages]
immler_homepage = "https://home.in.tum.de/~immler/"
[tiu]
name = "Alwen Tiu"
[tiu.emails]
tiu_email = "ATiu@ntu.edu.sg"
[tiu.homepages]
tiu_homepage = "http://users.cecs.anu.edu.au/~tiu/"
[henrio]
name = "Ludovic Henrio"
[henrio.emails]
henrio_email = "Ludovic.Henrio@sophia.inria.fr"
[henrio.homepages]
[urban]
name = "Christian Urban"
[urban.emails]
urban_email = "christian.urban@kcl.ac.uk"
[urban.homepages]
urban_homepage = "https://nms.kcl.ac.uk/christian.urban/"
[michaelis]
name = "Julius Michaelis"
[michaelis.emails]
michaelis_email = "isabelleopenflow@liftm.de"
michaelis_email1 = "maintainafpppt@liftm.de"
michaelis_email2 = "bdd@liftm.de"
michaelis_email3 = "afp@liftm.de"
[michaelis.homepages]
michaelis_homepage = "http://liftm.de/"
[scott]
name = "Dana Scott"
[scott.emails]
[scott.homepages]
scott_homepage = "http://www.cs.cmu.edu/~scott/"
[wenzel]
name = "Makarius Wenzel"
[wenzel.emails]
wenzel_email = "Makarius.wenzel@lri.fr"
[wenzel.homepages]
[dardinier]
name = "Thibault Dardinier"
[dardinier.emails]
dardinier_email = "thibault.dardinier@inf.ethz.ch"
[dardinier.homepages]
dardinier_homepage = "https://dardinier.me/"
[lallemand]
name = "Joseph Lallemand"
[lallemand.emails]
lallemand_email = "joseph.lallemand@loria.fr"
[lallemand.homepages]
[schmoetten]
name = "Richard Schmoetten"
[schmoetten.emails]
schmoetten_email = "s1311325@sms.ed.ac.uk"
[schmoetten.homepages]
[cohen]
name = "Ernie Cohen"
[cohen.emails]
cohen_email = "ecohen@amazon.com"
[cohen.homepages]
[chapman]
name = "Peter Chapman"
[chapman.emails]
chapman_email = "pc@cs.st-andrews.ac.uk"
[chapman.homepages]
[rickmann]
name = "Christina Rickmann"
[rickmann.emails]
rickmann_email = "c.rickmann@tu-berlin.de"
[rickmann.homepages]
[raya]
name = "Rodrigo Raya"
[raya.emails]
[raya.homepages]
raya_homepage = "https://people.epfl.ch/rodrigo.raya"
[kadzioka]
name = "Jakub Kądziołka"
[kadzioka.emails]
kadzioka_email = "kuba@kadziolka.net"
[kadzioka.homepages]
[foster]
name = "Michael Foster"
[foster.emails]
foster_email = "m.foster@sheffield.ac.uk"
[foster.homepages]
[zhann]
name = "Naijun Zhan"
[zhann.emails]
[zhann.homepages]
[fuenmayor]
name = "David Fuenmayor"
[fuenmayor.emails]
fuenmayor_email = "davfuenmayor@gmail.com"
[fuenmayor.homepages]
[iwama]
name = "Fumiya Iwama"
[iwama.emails]
iwama_email = "d1623001@s.konan-u.ac.jp"
[iwama.homepages]
[feliachi]
name = "Abderrahmane Feliachi"
[feliachi.emails]
feliachi_email = "abderrahmane.feliachi@lri.fr"
[feliachi.homepages]
[sudbrock]
name = "Henning Sudbrock"
[sudbrock.emails]
sudbrock_email = "sudbrock@mais.informatik.tu-darmstadt.de"
[sudbrock.homepages]
[bauer]
name = "Gertrud Bauer"
[bauer.emails]
[bauer.homepages]
[lux]
name = "Alexander Lux"
[lux.emails]
lux_email = "lux@mais.informatik.tu-darmstadt.de"
[lux.homepages]
[seidler]
name = "Henning Seidler"
[seidler.emails]
seidler_email = "henning.seidler@mailbox.tu-berlin.de"
[seidler.homepages]
[desharnais]
name = "Martin Desharnais"
[desharnais.emails]
desharnais_email = "martin.desharnais@unibw.de"
[desharnais.homepages]
desharnais_homepage = "https://martin.desharnais.me"
[wasserrab]
name = "Daniel Wasserrab"
[wasserrab.emails]
[wasserrab.homepages]
wasserrab_homepage = "http://pp.info.uni-karlsruhe.de/personhp/daniel_wasserrab.php"
[fell]
name = "Julian Fell"
[fell.emails]
fell_email = "julian.fell@uq.net.au"
[fell.homepages]
[zhan]
name = "Bohua Zhan"
[zhan.emails]
zhan_email = "bzhan@ios.ac.cn"
[zhan.homepages]
zhan_homepage = "http://lcs.ios.ac.cn/~bzhan/"
[stephan]
name = "Werner Stephan"
[stephan.emails]
stephan_email = "stephan@dfki.de"
[stephan.homepages]
[david]
name = "Marco David"
[david.emails]
david_email = "marco.david@hotmail.de"
[david.homepages]
[olm]
name = "Markus Müller-Olm"
[olm.emails]
[olm.homepages]
olm_homepage = "http://cs.uni-muenster.de/u/mmo/"
[havle]
name = "Oto Havle"
[havle.emails]
havle_email = "oha@sysgo.com"
[havle.homepages]
[margetson]
name = "James Margetson"
[margetson.emails]
[margetson.homepages]
[scharager]
name = "Matias Scharager"
[scharager.emails]
scharager_email = "mscharag@cs.cmu.edu"
[scharager.homepages]
[haftmann]
name = "Florian Haftmann"
[haftmann.emails]
haftmann_email = "florian.haftmann@informatik.tu-muenchen.de"
[haftmann.homepages]
haftmann_homepage = "http://isabelle.in.tum.de/~haftmann"
[schoepe]
name = "Daniel Schoepe"
[schoepe.emails]
schoepe_email = "daniel@schoepe.org"
[schoepe.homepages]
[nagele]
name = "Julian Nagele"
[nagele.emails]
nagele_email = "julian.nagele@uibk.ac.at"
[nagele.homepages]
[hoefner]
name = "Peter Höfner"
[hoefner.emails]
hoefner_email = "peter@hoefner-online.de"
[hoefner.homepages]
hoefner_homepage = "http://www.hoefner-online.de/"
[derrick]
name = "John Derrick"
[derrick.emails]
derrick_email = "j.derrick@sheffield.ac.uk"
[derrick.homepages]
[beeren]
name = "Joel Beeren"
[beeren.emails]
[beeren.homepages]
[echenim]
name = "Mnacho Echenim"
[echenim.emails]
echenim_email = "mnacho.echenim@univ-grenoble-alpes.fr"
[echenim.homepages]
echenim_homepage = "https://lig-membres.imag.fr/mechenim/"
[vytiniotis]
name = "Dimitrios Vytiniotis"
[vytiniotis.emails]
[vytiniotis.homepages]
vytiniotis_homepage = "http://research.microsoft.com/en-us/people/dimitris/"
[beringer]
name = "Lennart Beringer"
[beringer.emails]
beringer_email = "lennart.beringer@ifi.lmu.de"
[beringer.homepages]
[wickerson]
name = "John Wickerson"
[wickerson.emails]
[wickerson.homepages]
wickerson_homepage = "http://www.doc.ic.ac.uk/~jpw48"
[eberl]
name = "Manuel Eberl"
[eberl.emails]
eberl_email = "manuel@pruvisto.org"
eberl_email1 = "manuel.eberl@tum.de"
[eberl.homepages]
eberl_homepage = "https://pruvisto.org/"
eberl_homepage2 = "https://www.in.tum.de/~eberlm"
[noce]
name = "Pasquale Noce"
[noce.emails]
noce_email = "pasquale.noce.lavoro@gmail.com"
[noce.homepages]
[gunther]
name = "Emmanuel Gunther"
[gunther.emails]
gunther_email = "gunther@famaf.unc.edu.ar"
[gunther.homepages]
[nemouchi]
name = "Yakoub Nemouchi"
[nemouchi.emails]
nemouchi_email = "nemouchi@lri.fr"
nemouchi_email1 = "yakoub.nemouchi@york.ac.uk"
[nemouchi.homepages]
[stueber]
name = "Anke Stüber"
[stueber.emails]
stueber_email = "anke.stueber@campus.tu-berlin.de"
[stueber.homepages]
[sternagel]
name = "Christian Sternagel"
[sternagel.emails]
sternagel_email = "c.sternagel@gmail.com"
sternagel_email1 = "christian.sternagel@uibk.ac.at"
[sternagel.homepages]
sternagel_homepage = "http://cl-informatik.uibk.ac.at/users/griff/"
[sachtleben]
name = "Robert Sachtleben"
[sachtleben.emails]
sachtleben_email = "rob_sac@uni-bremen.de"
[sachtleben.homepages]
[kastermans]
name = "Bart Kastermans"
[kastermans.emails]
[kastermans.homepages]
kastermans_homepage = "http://kasterma.net"
[pal]
name = "Abhik Pal"
[pal.emails]
[pal.homepages]
[thiemann]
name = "René Thiemann"
[thiemann.emails]
thiemann_email = "rene.thiemann@uibk.ac.at"
[thiemann.homepages]
thiemann_homepage = "http://cl-informatik.uibk.ac.at/users/thiemann/"
[campo]
name = "Alejandro del Campo"
[campo.emails]
campo_email = "alejandro.del-campo@alum.unirioja.es"
[campo.homepages]
[raska]
name = "Martin Raška"
[raska.emails]
[raska.homepages]
[stannett]
name = "Mike Stannett"
[stannett.emails]
stannett_email = "m.stannett@sheffield.ac.uk"
[stannett.homepages]
[back]
name = "Ralph-Johan Back"
[back.emails]
[back.homepages]
back_homepage = "http://users.abo.fi/Ralph-Johan.Back/"
[bruegger]
name = "Lukas Brügger"
[bruegger.emails]
bruegger_email = "lukas.a.bruegger@gmail.com"
[bruegger.homepages]
[kuncak]
name = "Viktor Kuncak"
[kuncak.emails]
[kuncak.homepages]
kuncak_homepage = "http://lara.epfl.ch/~kuncak/"
[gaudel]
name = "Marie-Claude Gaudel"
[gaudel.emails]
gaudel_email = "mcg@lri.fr"
[gaudel.homepages]
[sison]
name = "Robert Sison"
[sison.emails]
[sison.homepages]
[benzmueller]
name = "Christoph Benzmüller"
[benzmueller.emails]
benzmueller_email = "c.benzmueller@gmail.com"
benzmueller_email1 = "c.benzmueller@fu-berlin.de"
[benzmueller.homepages]
benzmueller_homepage = "http://christoph-benzmueller.de"
benzmueller_homepage1 = "http://page.mi.fu-berlin.de/cbenzmueller/"
[from]
name = "Asta Halkjær From"
[from.emails]
from_email = "ahfrom@dtu.dk"
[from.homepages]
from_homepage = "https://people.compute.dtu.dk/ahfrom/"
[tuongj]
name = "Joseph Tuong"
[tuongj.emails]
[tuongj.homepages]
[zeller]
name = "Peter Zeller"
[zeller.emails]
zeller_email = "p_zeller@cs.uni-kl.de"
[zeller.homepages]
[schmidinger]
name = "Lukas Schmidinger"
[schmidinger.emails]
[schmidinger.homepages]
[ravindran]
name = "Binoy Ravindran"
[ravindran.emails]
[ravindran.homepages]
[rizaldi]
name = "Albert Rizaldi"
[rizaldi.emails]
rizaldi_email = "albert.rizaldi@ntu.edu.sg"
[rizaldi.homepages]
[sabouret]
name = "Nicolas Sabouret"
[sabouret.emails]
[sabouret.homepages]
[butler]
name = "David Butler"
[butler.emails]
butler_email = "dbutler@turing.ac.uk"
[butler.homepages]
butler_homepage = "https://www.turing.ac.uk/people/doctoral-students/david-butler"
[sprenger]
name = "Christoph Sprenger"
[sprenger.emails]
sprenger_email = "sprenger@inf.ethz.ch"
[sprenger.homepages]
[bordg]
name = "Anthony Bordg"
[bordg.emails]
bordg_email = "apdb3@cam.ac.uk"
[bordg.homepages]
bordg_homepage = "https://sites.google.com/site/anthonybordg/"
[bhatt]
name = "Bhargav Bhatt"
[bhatt.emails]
bhatt_email = "bhargav.bhatt@inf.ethz.ch"
[bhatt.homepages]
[gonzalez]
name = "Edgar Gonzàlez"
[gonzalez.emails]
gonzalez_email = "edgargip@google.com"
[gonzalez.homepages]
[adelsberger]
name = "Stephan Adelsberger"
[adelsberger.emails]
adelsberger_email = "stvienna@gmail.com"
[adelsberger.homepages]
adelsberger_homepage = "http://nm.wu.ac.at/nm/sadelsbe"
[schleicher]
name = "Dierk Schleicher"
[schleicher.emails]
[schleicher.homepages]
[ying]
name = "Shenggang Ying"
[ying.emails]
[ying.homepages]
[brien]
name = "Nicolas Robinson-O'Brien"
[brien.emails]
[brien.homepages]
[kobayashi]
name = "Hidetsune Kobayashi"
[kobayashi.emails]
[kobayashi.homepages]
[krauss]
name = "Alexander Krauss"
[krauss.emails]
krauss_email = "krauss@in.tum.de"
[krauss.homepages]
krauss_homepage = "http://www.in.tum.de/~krauss"
[somaini]
name = "Ivano Somaini"
[somaini.emails]
[somaini.homepages]
[seidl]
name = "Benedikt Seidl"
[seidl.emails]
seidl_email = "benedikt.seidl@tum.de"
[seidl.homepages]
[edmonds]
name = "Chelsea Edmonds"
[edmonds.emails]
edmonds_email = "cle47@cam.ac.uk"
[edmonds.homepages]
edmonds_homepage = "https://www.cst.cam.ac.uk/people/cle47"
[debrat]
name = "Henri Debrat"
[debrat.emails]
debrat_email = "henri.debrat@loria.fr"
[debrat.homepages]
[holub]
name = "Štěpán Holub"
[holub.emails]
holub_email = "holub@karlin.mff.cuni.cz"
[holub.homepages]
holub_homepage = "https://www2.karlin.mff.cuni.cz/~holub/"
[beresford]
name = "Alastair R. Beresford"
[beresford.emails]
beresford_email = "arb33@cam.ac.uk"
[beresford.homepages]
[terraf]
name = "Pedro Sánchez Terraf"
[terraf.emails]
terraf_email = "psterraf@unc.edu.ar"
[terraf.homepages]
terraf_homepage = "https://cs.famaf.unc.edu.ar/~pedro/home_en.html"
[raumer]
name = "Jakob von Raumer"
[raumer.emails]
raumer_email = "psxjv4@nottingham.ac.uk"
[raumer.homepages]
[pagano]
name = "Miguel Pagano"
[pagano.emails]
pagano_email = "miguel.pagano@unc.edu.ar"
[pagano.homepages]
pagano_homepage = "https://cs.famaf.unc.edu.ar/~mpagano/"
[coglio]
name = "Alessandro Coglio"
[coglio.emails]
coglio_email = "coglio@kestrel.edu"
[coglio.homepages]
coglio_homepage = "http://www.kestrel.edu/~coglio"
[caballero]
name = "José Manuel Rodríguez Caballero"
[caballero.emails]
caballero_email = "jose.manuel.rodriguez.caballero@ut.ee"
[caballero.homepages]
caballero_homepage = "https://josephcmac.github.io/"
[grechuk]
name = "Bogdan Grechuk"
[grechuk.emails]
grechuk_email = "grechukbogdan@yandex.ru"
[grechuk.homepages]
[sewell]
name = "Thomas Sewell"
[sewell.emails]
[sewell.homepages]
[leustean]
name = "Laurentiu Leustean"
[leustean.emails]
[leustean.homepages]
[rosskopf]
name = "Simon Roßkopf"
[rosskopf.emails]
rosskopf_email = "rosskops@in.tum.de"
[rosskopf.homepages]
rosskopf_homepage = "http://www21.in.tum.de/~rosskops"
[aspinall]
name = "David Aspinall"
[aspinall.emails]
[aspinall.homepages]
aspinall_homepage = "http://homepages.inf.ed.ac.uk/da/"
[ausaf]
name = "Fahad Ausaf"
[ausaf.emails]
[ausaf.homepages]
ausaf_homepage = "http://kcl.academia.edu/FahadAusaf"
[diekmann]
name = "Cornelius Diekmann"
[diekmann.emails]
diekmann_email = "diekmann@net.in.tum.de"
[diekmann.homepages]
diekmann_homepage = "http://net.in.tum.de/~diekmann"
[fouillard]
name = "Valentin Fouillard"
[fouillard.emails]
fouillard_email = "valentin.fouillard@limsi.fr"
[fouillard.homepages]
[willenbrink]
name = "Sebastian Willenbrink"
[willenbrink.emails]
willenbrink_email = "sebastian.willenbrink@tum.de"
[willenbrink.homepages]
[xu]
name = "Jian Xu"
[xu.emails]
[xu.homepages]
[wang]
name = "Shuling Wang"
[wang.emails]
[wang.homepages]
[ridge]
name = "Tom Ridge"
[ridge.emails]
[ridge.homepages]
[kleppmann]
name = "Martin Kleppmann"
[kleppmann.emails]
kleppmann_email = "martin.kleppmann@cl.cam.ac.uk"
[kleppmann.homepages]
[kreuzer]
name = "Katharina Kreuzer"
[kreuzer.emails]
kreuzer_email = "kreuzerk@in.tum.de"
[kreuzer.homepages]
kreuzer_homepage = "https://www21.in.tum.de/team/kreuzer/"
[traut]
name = "Christoph Traut"
[traut.emails]
[traut.homepages]
[blanchette]
name = "Jasmin Christian Blanchette"
[blanchette.emails]
blanchette_email = "jasmin.blanchette@gmail.com"
blanchette_email1 = "j.c.blanchette@vu.nl"
[blanchette.homepages]
blanchette_homepage = "http://www21.in.tum.de/~blanchet"
blanchette_homepage1 = "https://www.cs.vu.nl/~jbe248/"
[van]
name = "Hai Nguyen Van"
[van.emails]
van_email = "hai.nguyenvan.phie@gmail.com"
[van.homepages]
[brunner]
name = "Julian Brunner"
[brunner.emails]
brunner_email = "brunnerj@in.tum.de"
[brunner.homepages]
brunner_homepage = "http://www21.in.tum.de/~brunnerj/"
[reiche]
name = "Sebastian Reiche"
[reiche.emails]
[reiche.homepages]
reiche_homepage = "https://www.linkedin.com/in/sebastian-reiche-0b2093178"
[eriksson]
name = "Lars-Henrik Eriksson"
[eriksson.emails]
eriksson_email = "lhe@it.uu.se"
[eriksson.homepages]
[nipkow]
name = "Tobias Nipkow"
[nipkow.emails]
nipkow_email = "nipkow@in.tum.de"
[nipkow.homepages]
nipkow_homepage = "https://www.in.tum.de/~nipkow/"
[divason]
name = "Jose Divasón"
[divason.emails]
divason_email = "jose.divason@unirioja.es"
[divason.homepages]
divason_homepage = "https://www.unirioja.es/cu/jodivaso/"
[barsotti]
name = "Damián Barsotti"
[barsotti.emails]
[barsotti.homepages]
barsotti_homepage = "http://www.cs.famaf.unc.edu.ar/~damian/"
[nagashima]
name = "Yutaka Nagashima"
[nagashima.emails]
nagashima_email = "Yutaka.Nagashima@data61.csiro.au"
[nagashima.homepages]
[avigad]
name = "Jeremy Avigad"
[avigad.emails]
avigad_email = "avigad@cmu.edu"
[avigad.homepages]
avigad_homepage = "http://www.andrew.cmu.edu/user/avigad/"
[abdulaziz]
name = "Mohammad Abdulaziz"
[abdulaziz.emails]
abdulaziz_email = "mohammad.abdulaziz@in.tum.de"
abdulaziz_email1 = "mohammad.abdulaziz8@gmail.com"
[abdulaziz.homepages]
abdulaziz_homepage = "http://home.in.tum.de/~mansour/"
[kuncar]
name = "Ondřej Kunčar"
[kuncar.emails]
[kuncar.homepages]
kuncar_homepage = "http://www21.in.tum.de/~kuncar/"
[borgstroem]
name = "Johannes Borgström"
[borgstroem.emails]
borgstroem_email = "johannes.borgstrom@it.uu.se"
[borgstroem.homepages]
[kurz]
name = "Friedrich Kurz"
[kurz.emails]
kurz_email = "friedrich.kurz@tum.de"
[kurz.homepages]
[noschinski]
name = "Lars Noschinski"
[noschinski.emails]
noschinski_email = "noschinl@gmail.com"
[noschinski.homepages]
noschinski_homepage = "http://www21.in.tum.de/~noschinl/"
[liy]
name = "Yangjia Li"
[liy.emails]
[liy.homepages]
[wimmer]
name = "Simon Wimmer"
[wimmer.emails]
wimmer_email = "simon.wimmer@tum.de"
[wimmer.homepages]
wimmer_homepage = "http://home.in.tum.de/~wimmers/"
[gammie]
name = "Peter Gammie"
[gammie.emails]
gammie_email = "peteg42@gmail.com"
[gammie.homepages]
gammie_homepage = "http://peteg.org"
[snelting]
name = "Gregor Snelting"
[snelting.emails]
[snelting.homepages]
snelting_homepage = "http://pp.info.uni-karlsruhe.de/personhp/gregor_snelting.php"
[stark]
name = "Eugene W. Stark"
[stark.emails]
stark_email = "stark@cs.stonybrook.edu"
[stark.homepages]
[engelhardt]
name = "Kai Engelhardt"
[engelhardt.emails]
[engelhardt.homepages]
[fleury]
name = "Mathias Fleury"
[fleury.emails]
fleury_email = "fleury@mpi-inf.mpg.de"
fleury_email1 = "mathias.fleury@jku.at"
[fleury.homepages]
fleury_homepage = "http://fmv.jku.at/fleury"
[griebel]
name = "Simon Griebel"
[griebel.emails]
griebel_email = "s.griebel@tum.de"
[griebel.homepages]
[zhang]
name = "Yu Zhang"
[zhang.emails]
[zhang.homepages]
[spichkova]
name = "Maria Spichkova"
[spichkova.emails]
spichkova_email = "maria.spichkova@rmit.edu.au"
[spichkova.homepages]
[andronick]
name = "June Andronick"
[andronick.emails]
[andronick.homepages]
[lammich]
name = "Peter Lammich"
[lammich.emails]
lammich_email = "lammich@in.tum.de"
lammich_email1 = "peter.lammich@uni-muenster.de"
[lammich.homepages]
lammich_homepage = "http://www21.in.tum.de/~lammich"
[maricf]
name = "Filip Marić"
[maricf.emails]
maricf_email = "filip@matf.bg.ac.rs"
[maricf.homepages]
maricf_homepage = "http://www.matf.bg.ac.rs/~filip"
[popescu]
name = "Andrei Popescu"
[popescu.emails]
popescu_email = "a.popescu@sheffield.ac.uk"
popescu_email1 = "uuomul@yahoo.com"
popescu_email2 = "a.popescu@mdx.ac.uk"
[popescu.homepages]
popescu_homepage = "https://www.andreipopescu.uk"
[chen]
name = "L. Chen"
[chen.emails]
[chen.homepages]
[helke]
name = "Steffen Helke"
[helke.emails]
helke_email = "helke@cs.tu-berlin.de"
[helke.homepages]
[pohjola]
name = "Johannes Åman Pohjola"
[pohjola.emails]
[pohjola.homepages]
[yingm]
name = "Mingsheng Ying"
[yingm.emails]
[yingm.homepages]
[fosterj]
name = "J. Nathan Foster"
[fosterj.emails]
[fosterj.homepages]
fosterj_homepage = "http://www.cs.cornell.edu/~jnfoster/"
[verbeek]
name = "Freek Verbeek"
[verbeek.emails]
verbeek_email = "Freek.Verbeek@ou.nl"
verbeek_email1 = "freek@vt.edu"
[verbeek.homepages]
[struth]
name = "Georg Struth"
[struth.emails]
struth_email = "g.struth@sheffield.ac.uk"
[struth.homepages]
struth_homepage = "http://staffwww.dcs.shef.ac.uk/people/G.Struth/"
[mitsch]
name = "Stefan Mitsch"
[mitsch.emails]
mitsch_email = "smitsch@cs.cmu.edu"
[mitsch.homepages]
[nordhoff]
name = "Benedikt Nordhoff"
[nordhoff.emails]
nordhoff_email = "b.n@wwu.de"
nordhoff_email1 = "b_nord01@uni-muenster.de"
[nordhoff.homepages]
[kirchner]
name = "Daniel Kirchner"
[kirchner.emails]
kirchner_email = "daniel@ekpyron.org"
[kirchner.homepages]
[merz]
name = "Stephan Merz"
[merz.emails]
merz_email = "Stephan.Merz@loria.fr"
[merz.homepages]
merz_homepage = "http://www.loria.fr/~merz"
[fernandez]
name = "Matthew Fernandez"
[fernandez.emails]
[fernandez.homepages]
[kolanski]
name = "Rafal Kolanski"
[kolanski.emails]
kolanski_email = "rafal.kolanski@nicta.com.au"
[kolanski.homepages]
[strnisa]
name = "Rok Strniša"
[strnisa.emails]
strnisa_email = "rok@strnisa.com"
[strnisa.homepages]
strnisa_homepage = "http://rok.strnisa.com/lj/"
[liuy]
name = "Yang Liu"
[liuy.emails]
liuy_email = "yangliu@ntu.edu.sg"
[liuy.homepages]
[jacobsen]
name = "Frederik Krogsdal Jacobsen"
[jacobsen.emails]
jacobsen_email = "fkjac@dtu.dk"
[jacobsen.homepages]
jacobsen_homepage = "http://people.compute.dtu.dk/fkjac/"
[crighton]
name = "Aaron Crighton"
[crighton.emails]
crighton_email = "crightoa@mcmaster.ca"
[crighton.homepages]
[matiyasevich]
name = "Yuri Matiyasevich"
[matiyasevich.emails]
[matiyasevich.homepages]
[kaliszyk]
name = "Cezary Kaliszyk"
[kaliszyk.emails]
kaliszyk_email = "cezary.kaliszyk@uibk.ac.at"
[kaliszyk.homepages]
kaliszyk_homepage = "http://cl-informatik.uibk.ac.at/users/cek/"
[voisin]
name = "Frederic Voisin"
[voisin.emails]
[voisin.homepages]
[kaufmann]
name = "Daniela Kaufmann"
[kaufmann.emails]
[kaufmann.homepages]
kaufmann_homepage = "http://fmv.jku.at/kaufmann"
[milehins]
name = "Mihails Milehins"
[milehins.emails]
milehins_email = "mihailsmilehins@gmail.com"
[milehins.homepages]
[cordwell]
name = "Katherine Cordwell"
[cordwell.emails]
cordwell_email = "kcordwel@cs.cmu.edu"
[cordwell.homepages]
cordwell_homepage = "https://www.cs.cmu.edu/~kcordwel/"
[smaus]
name = "Jan-Georg Smaus"
[smaus.emails]
[smaus.homepages]
smaus_homepage = "http://www.irit.fr/~Jan-Georg.Smaus"
[sefidgar]
name = "S. Reza Sefidgar"
[sefidgar.emails]
sefidgar_email = "reza.sefidgar@inf.ethz.ch"
[sefidgar.homepages]
[steinberg]
name = "Matías Steinberg"
[steinberg.emails]
steinberg_email = "matias.steinberg@mi.unc.edu.ar"
[steinberg.homepages]
[furusawa]
name = "Hitoshi Furusawa"
[furusawa.emails]
[furusawa.homepages]
furusawa_homepage = "http://www.sci.kagoshima-u.ac.jp/~furusawa/"
[unruh]
name = "Dominique Unruh"
[unruh.emails]
unruh_email = "unruh@ut.ee"
[unruh.homepages]
unruh_homepage = "https://www.ut.ee/~unruh/"
[yamada]
name = "Akihisa Yamada"
[yamada.emails]
yamada_email = "akihisa.yamada@uibk.ac.at"
yamada_email1 = "ayamada@trs.cm.is.nagoya-u.ac.jp"
yamada_email2 = "akihisa.yamada@aist.go.jp"
yamada_email3 = "akihisayamada@nii.ac.jp"
[yamada.homepages]
yamada_homepage = "http://group-mmm.org/~ayamada/"
[smola]
name = "Filip Smola"
[smola.emails]
smola_email = "f.smola@sms.ed.ac.uk"
[smola.homepages]
[pusch]
name = "Cornelia Pusch"
[pusch.emails]
[pusch.homepages]
[ogawa]
name = "Mizuhito Ogawa"
[ogawa.emails]
[ogawa.homepages]
[bulwahn]
name = "Lukas Bulwahn"
[bulwahn.emails]
bulwahn_email = "lukas.bulwahn@gmail.com"
[bulwahn.homepages]
[obua]
name = "Steven Obua"
[obua.emails]
obua_email = "steven@recursivemind.com"
[obua.homepages]
[bayer]
name = "Jonas Bayer"
[bayer.emails]
bayer_email = "jonas.bayer999@gmail.com"
[bayer.homepages]
[brun]
name = "Matthias Brun"
[brun.emails]
brun_email = "matthias.brun@inf.ethz.ch"
[brun.homepages]
[aransay]
name = "Jesús Aransay"
[aransay.emails]
aransay_email = "jesus-maria.aransay@unirioja.es"
[aransay.homepages]
aransay_homepage = "https://www.unirioja.es/cu/jearansa"
[gioiosa]
name = "Gianpaolo Gioiosa"
[gioiosa.emails]
[gioiosa.homepages]
[karayel]
name = "Emin Karayel"
[karayel.emails]
karayel_email = "me@eminkarayel.de"
[karayel.homepages]
karayel_homepage = "https://orcid.org/0000-0003-3290-5034"
[koller]
name = "Lukas Koller"
[koller.emails]
koller_email = "lukas.koller@tum.de"
[koller.homepages]
[starosta]
name = "Štěpán Starosta"
[starosta.emails]
starosta_email = "stepan.starosta@fit.cvut.cz"
[starosta.homepages]
starosta_homepage = "https://users.fit.cvut.cz/~staroste/"
[zhangx]
name = "Xingyuan Zhang"
[zhangx.emails]
[zhangx.homepages]
[katovsky]
name = "Alexander Katovsky"
[katovsky.emails]
katovsky_email = "apk32@cam.ac.uk"
katovsky_email1 = "alexander.katovsky@cantab.net"
[katovsky.homepages]
[roessle]
name = "Ian Roessle"
[roessle.emails]
[roessle.homepages]
[schoepf]
name = "Jonas Schöpf"
[schoepf.emails]
schoepf_email = "jonas.schoepf@uibk.ac.at"
[schoepf.homepages]
[gheri]
name = "Lorenzo Gheri"
[gheri.emails]
gheri_email = "lor.gheri@gmail.com"
[gheri.homepages]
[oosterhuis]
name = "Roelof Oosterhuis"
[oosterhuis.emails]
oosterhuis_email = "roelofoosterhuis@gmail.com"
[oosterhuis.homepages]
[robillard]
name = "Simon Robillard"
[robillard.emails]
[robillard.homepages]
robillard_homepage = "https://simon-robillard.net/"
[rauch]
name = "Nicole Rauch"
[rauch.emails]
rauch_email = "rauch@informatik.uni-kl.de"
[rauch.homepages]
[wolff]
name = "Burkhart Wolff"
[wolff.emails]
wolff_email = "burkhart.wolff@lri.fr"
[wolff.homepages]
wolff_homepage = "https://www.lri.fr/~wolff/"
[lattuada]
name = "Andrea Lattuada"
[lattuada.emails]
[lattuada.homepages]
lattuada_homepage = "https://andrea.lattuada.me"
[pierzchalski]
name = "Edward Pierzchalski"
[pierzchalski.emails]
[pierzchalski.homepages]
[chaieb]
name = "Amine Chaieb"
[chaieb.emails]
[chaieb.homepages]
[raszyk]
name = "Martin Raszyk"
[raszyk.emails]
raszyk_email = "martin.raszyk@inf.ethz.ch"
raszyk_email1 = "m.raszyk@gmail.com"
[raszyk.homepages]
[zee]
name = "Karen Zee"
[zee.emails]
zee_email = "kkz@mit.edu"
[zee.homepages]
zee_homepage = "http://www.mit.edu/~kkz/"
[jensen]
name = "Alexander Birch Jensen"
[jensen.emails]
jensen_email = "aleje@dtu.dk"
[jensen.homepages]
jensen_homepage = "https://people.compute.dtu.dk/aleje/"
[murray]
name = "Toby Murray"
[murray.emails]
murray_email = "toby.murray@unimelb.edu.au"
[murray.homepages]
murray_homepage = "https://people.eng.unimelb.edu.au/tobym/"
[hupel]
name = "Lars Hupel"
[hupel.emails]
hupel_email = "hupel@in.tum.de"
hupel_email1 = "lars@hupel.info"
[hupel.homepages]
hupel_homepage = "https://www21.in.tum.de/~hupel/"
hupel_homepage1 = "https://lars.hupel.info/"
[rowat]
name = "Colin Rowat"
[rowat.emails]
rowat_email = "c.rowat@bham.ac.uk"
[rowat.homepages]
[schneider]
name = "Joshua Schneider"
[schneider.emails]
schneider_email = "joshua.schneider@inf.ethz.ch"
[schneider.homepages]
[cousin]
name = "Marie Cousin"
[cousin.emails]
cousin_email = "marie.cousin@grenoble-inp.org"
[cousin.homepages]
[parsert]
name = "Julian Parsert"
[parsert.emails]
parsert_email = "julian.parsert@gmail.com"
parsert_email1 = "julian.parsert@uibk.ac.at"
[parsert.homepages]
parsert_homepage = "http://www.parsert.com/"
[aehlig]
name = "Klaus Aehlig"
[aehlig.emails]
[aehlig.homepages]
aehlig_homepage = "http://www.linta.de/~aehlig/"
[argyraki]
name = "Angeliki Koutsoukou-Argyraki"
[argyraki.emails]
argyraki_email = "ak2110@cam.ac.uk"
[argyraki.homepages]
argyraki_homepage = "https://www.cl.cam.ac.uk/~ak2110/"
argyraki_homepage2 = "https://www.cst.cam.ac.uk/people/ak2110"
[ye]
name = "Lina Ye"
[ye.emails]
ye_email = "lina.ye@lri.fr"
[ye.homepages]
[moeller]
name = "Bernhard Möller"
[moeller.emails]
[moeller.homepages]
moeller_homepage = "https://www.informatik.uni-augsburg.de/en/chairs/dbis/pmi/staff/moeller/"
[zankl]
name = "Harald Zankl"
[zankl.emails]
zankl_email = "Harald.Zankl@uibk.ac.at"
[zankl.homepages]
zankl_homepage = "http://cl-informatik.uibk.ac.at/users/hzankl"
[langenstein]
name = "Bruno Langenstein"
[langenstein.emails]
langenstein_email = "langenstein@dfki.de"
[langenstein.homepages]
[breitner]
name = "Joachim Breitner"
[breitner.emails]
breitner_email = "mail@joachim-breitner.de"
breitner_email1 = "joachim@cis.upenn.edu"
[breitner.homepages]
breitner_homepage = "http://pp.ipd.kit.edu/~breitner"
[thommes]
name = "Joseph Thommes"
[thommes.emails]
thommes_email = "joseph-thommes@gmx.de"
[thommes.homepages]
[loibl]
name = "Matthias Loibl"
[loibl.emails]
[loibl.homepages]
[cock]
name = "David Cock"
[cock.emails]
cock_email = "david.cock@nicta.com.au"
[cock.homepages]
[stuewe]
name = "Daniel Stüwe"
[stuewe.emails]
[stuewe.homepages]
[decova]
name = "Sára Decova"
[decova.emails]
[decova.homepages]
[nikiforov]
name = "Denis Nikiforov"
[nikiforov.emails]
nikiforov_email = "denis.nikif@gmail.com"
[nikiforov.homepages]
[traytel]
name = "Dmitriy Traytel"
[traytel.emails]
traytel_email = "traytel@in.tum.de"
traytel_email1 = "traytel@inf.ethz.ch"
traytel_email2 = "traytel@di.ku.dk"
[traytel.homepages]
traytel_homepage = "https://traytel.bitbucket.io/"
[tverdyshev]
name = "Sergey Tverdyshev"
[tverdyshev.emails]
tverdyshev_email = "stv@sysgo.com"
[tverdyshev.homepages]
[wassell]
name = "Mark Wassell"
[wassell.emails]
wassell_email = "mpwassell@gmail.com"
[wassell.homepages]
[ijbema]
name = "Mark Ijbema"
[ijbema.emails]
ijbema_email = "ijbema@fmf.nl"
[ijbema.homepages]
[wirt]
name = "Kai Wirt"
[wirt.emails]
[wirt.homepages]
[matache]
name = "Cristina Matache"
[matache.emails]
matache_email = "cris.matache@gmail.com"
[matache.homepages]
[ito]
name = "Yosuke Ito"
[ito.emails]
ito_email = "glacier345@gmail.com"
[ito.homepages]
[maric]
name = "Ognjen Marić"
[maric.emails]
maric_email = "ogi.afp@mynosefroze.com"
[maric.homepages]
[heimes]
name = "Lukas Heimes"
[heimes.emails]
heimes_email = "heimesl@student.ethz.ch"
[heimes.homepages]
[parrow]
name = "Joachim Parrow"
[parrow.emails]
parrow_email = "joachim.parrow@it.uu.se"
[parrow.homepages]
[naraschewski]
name = "Wolfgang Naraschewski"
[naraschewski.emails]
[naraschewski.homepages]
[amani]
name = "Sidney Amani"
[amani.emails]
amani_email = "sidney.amani@data61.csiro.au"
[amani.homepages]
[palmer]
name = "Jake Palmer"
[palmer.emails]
palmer_email = "jake.palmer@ed.ac.uk"
[palmer.homepages]
[bockenek]
name = "Joshua Bockenek"
[bockenek.emails]
[bockenek.homepages]
[lachnitt]
name = "Hanna Lachnitt"
[lachnitt.emails]
lachnitt_email = "lachnitt@stanford.edu"
[lachnitt.homepages]
[rabe]
name = "Markus N. Rabe"
[rabe.emails]
[rabe.homepages]
rabe_homepage = "http://www.react.uni-saarland.de/people/rabe.html"
[munive]
name = "Jonathan Julian Huerta y Munive"
[munive.emails]
munive_email = "jjhuertaymunive1@sheffield.ac.uk"
munive_email1 = "jonjulian23@gmail.com"
[munive.homepages]
[gouezel]
name = "Sebastien Gouezel"
[gouezel.emails]
gouezel_email = "sebastien.gouezel@univ-rennes1.fr"
[gouezel.homepages]
gouezel_homepage = "http://www.math.sciences.univ-nantes.fr/~gouezel/"
[brucker]
name = "Achim D. Brucker"
[brucker.emails]
brucker_email = "a.brucker@exeter.ac.uk"
brucker_email1 = "brucker@spamfence.net"
brucker_email2 = "adbrucker@0x5f.org"
[brucker.homepages]
brucker_homepage = "https://www.brucker.ch/"
[sato]
name = "Tetsuya Sato"
[sato.emails]
sato_email = "tsato@c.titech.ac.jp"
[sato.homepages]
sato_homepage = "https://sites.google.com/view/tetsuyasato/"
[huffman]
name = "Brian Huffman"
[huffman.emails]
huffman_email = "huffman@in.tum.de"
huffman_email1 = "brianh@cs.pdx.edu"
[huffman.homepages]
huffman_homepage = "http://cs.pdx.edu/~brianh/"
[fleuriot]
name = "Jacques D. Fleuriot"
[fleuriot.emails]
fleuriot_email = "Jacques.Fleuriot@ed.ac.uk"
fleuriot_email1 = "jdf@ed.ac.uk"
[fleuriot.homepages]
fleuriot_homepage = "https://www.inf.ed.ac.uk/people/staff/Jacques_Fleuriot.html"
[hess]
name = "Andreas V. Hess"
[hess.emails]
hess_email = "avhe@dtu.dk"
hess_email1 = "andreasvhess@gmail.com"
[hess.homepages]
[marmsoler]
name = "Diego Marmsoler"
[marmsoler.emails]
marmsoler_email = "diego.marmsoler@tum.de"
[marmsoler.homepages]
marmsoler_homepage = "http://marmsoler.com"
[hibon]
name = "Quentin Hibon"
[hibon.emails]
hibon_email = "qh225@cl.cam.ac.uk"
[hibon.homepages]
[tasch]
name = "Markus Tasch"
[tasch.emails]
tasch_email = "tasch@mais.informatik.tu-darmstadt.de"
[tasch.homepages]
[doty]
name = "Matthew Wampler-Doty"
[doty.emails]
[doty.homepages]
[berghofer]
name = "Stefan Berghofer"
[berghofer.emails]
berghofer_email = "berghofe@in.tum.de"
[berghofer.homepages]
berghofer_homepage = "http://www.in.tum.de/~berghofe"
[hirata]
name = "Michikazu Hirata"
[hirata.emails]
hirata_email = "hirata.m.ac@m.titech.ac.jp"
[hirata.homepages]
[sylvestre]
name = "Jeremy Sylvestre"
[sylvestre.emails]
sylvestre_email = "jeremy.sylvestre@ualberta.ca"
sylvestre_email1 = "jsylvest@ualberta.ca"
[sylvestre.homepages]
sylvestre_homepage = "http://ualberta.ca/~jsylvest/"
[lindenberg]
name = "Christina Lindenberg"
[lindenberg.emails]
[lindenberg.homepages]
[joosten]
name = "Sebastiaan J. C. Joosten"
[joosten.emails]
joosten_email = "sebastiaan.joosten@uibk.ac.at"
joosten_email1 = "sjcjoosten@gmail.com"
joosten_email2 = "s.j.c.joosten@utwente.nl"
[joosten.homepages]
joosten_homepage = "https://sjcjoosten.nl/"
[blumson]
name = "Ben Blumson"
[blumson.emails]
blumson_email = "benblumson@gmail.com"
[blumson.homepages]
blumson_homepage = "https://philpeople.org/profiles/ben-blumson"
[hosking]
name = "Tony Hosking"
[hosking.emails]
[hosking.homepages]
hosking_homepage = "https://www.cs.purdue.edu/homes/hosking/"
[preoteasa]
name = "Viorel Preoteasa"
[preoteasa.emails]
preoteasa_email = "viorel.preoteasa@aalto.fi"
[preoteasa.homepages]
preoteasa_homepage = "http://users.abo.fi/vpreotea/"
[gutkovas]
name = "Ramunas Gutkovas"
[gutkovas.emails]
gutkovas_email = "ramunas.gutkovas@it.uu.se"
[gutkovas.homepages]
[minamide]
name = "Yasuhiko Minamide"
[minamide.emails]
minamide_email = "minamide@is.titech.ac.jp"
[minamide.homepages]
minamide_homepage = "https://sv.c.titech.ac.jp/minamide/index.en.html"
[waldmann]
name = "Uwe Waldmann"
[waldmann.emails]
waldmann_email = "waldmann@mpi-inf.mpg.de"
[waldmann.homepages]
[lewis]
name = "Corey Lewis"
[lewis.emails]
lewis_email = "corey.lewis@data61.csiro.au"
[lewis.homepages]
[peters]
name = "Kirstin Peters"
[peters.emails]
peters_email = "kirstin.peters@tu-berlin.de"
[peters.homepages]
[ortner]
name = "Veronika Ortner"
[ortner.emails]
[ortner.homepages]
[fiedler]
name = "Ben Fiedler"
[fiedler.emails]
fiedler_email = "ben.fiedler@inf.ethz.ch"
[fiedler.homepages]
[becker]
name = "Heiko Becker"
[becker.emails]
becker_email = "hbecker@mpi-sws.org"
[becker.homepages]
[bracevac]
name = "Oliver Bračevac"
[bracevac.emails]
bracevac_email = "bracevac@st.informatik.tu-darmstadt.de"
[bracevac.homepages]
[bohrer]
name = "Rose Bohrer"
[bohrer.emails]
bohrer_email = "rose.bohrer.cs@gmail.com"
[bohrer.homepages]
[londono]
name = "Alejandro Gómez-Londoño"
[londono.emails]
londono_email = "alejandro.gomez@chalmers.se"
[londono.homepages]
[armstrong]
name = "Alasdair Armstrong"
[armstrong.emails]
[armstrong.homepages]
[glabbeek]
name = "Rob van Glabbeek"
[glabbeek.emails]
[glabbeek.homepages]
glabbeek_homepage = "http://theory.stanford.edu/~rvg/"
[jiangd]
name = "Dongchen Jiang"
[jiangd.emails]
jiangd_email = "dongchenjiang@googlemail.com"
[jiangd.homepages]
[meis]
name = "Rene Meis"
[meis.emails]
meis_email = "rene.meis@uni-muenster.de"
meis_email1 = "rene.meis@uni-due.de"
[meis.homepages]
[hofmann]
name = "Martin Hofmann"
[hofmann.emails]
[hofmann.homepages]
hofmann_homepage = "http://www.tcs.informatik.uni-muenchen.de/~mhofmann"
[kerber]
name = "Manfred Kerber"
[kerber.emails]
kerber_email = "mnfrd.krbr@gmail.com"
[kerber.homepages]
kerber_homepage = "http://www.cs.bham.ac.uk/~mmk"
[linker]
name = "Sven Linker"
[linker.emails]
linker_email = "s.linker@liverpool.ac.uk"
[linker.homepages]
[balbach]
name = "Frank J. Balbach"
[balbach.emails]
balbach_email = "frank-balbach@gmx.de"
[balbach.homepages]
[weber]
name = "Tjark Weber"
[weber.emails]
weber_email = "tjark.weber@it.uu.se"
[weber.homepages]
weber_homepage = "http://user.it.uu.se/~tjawe125/"
[hellauer]
name = "Fabian Hellauer"
[hellauer.emails]
hellauer_email = "hellauer@in.tum.de"
[hellauer.homepages]
[reiter]
name = "Markus Reiter"
[reiter.emails]
[reiter.homepages]
[herzberg]
name = "Michael Herzberg"
[herzberg.emails]
herzberg_email = "mail@michael-herzberg.de"
[herzberg.homepages]
herzberg_homepage = "http://www.dcs.shef.ac.uk/cgi-bin/makeperson?M.Herzberg"
[overbeek]
name = "Roy Overbeek"
[overbeek.emails]
overbeek_email = "Roy.Overbeek@cwi.nl"
[overbeek.homepages]
[koerner]
name = "Stefan Körner"
[koerner.emails]
koerner_email = "s_koer03@uni-muenster.de"
[koerner.homepages]
[tan]
name = "Yong Kiam Tan"
[tan.emails]
tan_email = "yongkiat@cs.cmu.edu"
[tan.homepages]
tan_homepage = "https://www.cs.cmu.edu/~yongkiat/"
[esparza]
name = "Javier Esparza"
[esparza.emails]
[esparza.homepages]
esparza_homepage = "https://www7.in.tum.de/~esparza/"
[platzer]
name = "André Platzer"
[platzer.emails]
platzer_email = "aplatzer@cs.cmu.edu"
[platzer.homepages]
platzer_homepage = "https://www.cs.cmu.edu/~aplatzer/"
[matichuk]
name = "Daniel Matichuk"
[matichuk.emails]
[matichuk.homepages]
[rawson]
name = "Michael Rawson"
[rawson.emails]
rawson_email = "michaelrawson76@gmail.com"
rawson_email1 = "mr644@cam.ac.uk"
[rawson.homepages]
[bisping]
name = "Benjamin Bisping"
[bisping.emails]
bisping_email = "benjamin.bisping@campus.tu-berlin.de"
[bisping.homepages]
[sanan]
name = "David Sanan"
[sanan.emails]
sanan_email = "sanan@ntu.edu.sg"
[sanan.homepages]
[jungnickel]
name = "Tim Jungnickel"
[jungnickel.emails]
jungnickel_email = "tim.jungnickel@tu-berlin.de"
[jungnickel.homepages]
[ammer]
name = "Thomas Ammer"
[ammer.emails]
[ammer.homepages]
[mulligan]
name = "Dominic P. Mulligan"
[mulligan.emails]
mulligan_email = "dominic.p.mulligan@googlemail.com"
mulligan_email1 = "Dominic.Mulligan@arm.com"
[mulligan.homepages]
[georgescu]
name = "George Georgescu"
[georgescu.emails]
[georgescu.homepages]
[aissat]
name = "Romain Aissat"
[aissat.emails]
[aissat.homepages]
[gore]
name = "Rajeev Gore"
[gore.emails]
gore_email = "rajeev.gore@anu.edu.au"
[gore.homepages]
[gomes]
name = "Victor B. F. Gomes"
[gomes.emails]
gomes_email = "victor.gomes@cl.cam.ac.uk"
gomes_email2 = "victorborgesfg@gmail.com"
gomes_email4 = "vborgesferreiragomes1@sheffield.ac.uk"
[gomes.homepages]
gomes_homepage = "http://www.dcs.shef.ac.uk/~victor"
[trachtenherz]
name = "David Trachtenherz"
[trachtenherz.emails]
[trachtenherz.homepages]
[lohner]
name = "Denis Lohner"
[lohner.emails]
lohner_email = "denis.lohner@kit.edu"
[lohner.homepages]
lohner_homepage = "http://pp.ipd.kit.edu/person.php?id=88"
[richter]
name = "Stefan Richter"
[richter.emails]
richter_email = "richter@informatik.rwth-aachen.de"
[richter.homepages]
richter_homepage = "http://www-lti.informatik.rwth-aachen.de/~richter/"
[nemeti]
name = "István Németi"
[nemeti.emails]
[nemeti.homepages]
nemeti_homepage = "http://www.renyi.hu/~nemeti/"
[bentkamp]
name = "Alexander Bentkamp"
[bentkamp.emails]
bentkamp_email = "bentkamp@gmail.com"
bentkamp_email1 = "a.bentkamp@vu.nl"
[bentkamp.homepages]
bentkamp_homepage = "https://www.cs.vu.nl/~abp290/"
[zeyda]
name = "Frank Zeyda"
[zeyda.emails]
zeyda_email = "frank.zeyda@york.ac.uk"
[zeyda.homepages]
[tuerk]
name = "Thomas Tuerk"
[tuerk.emails]
[tuerk.homepages]
[ribeiro]
name = "Pedro Ribeiro"
[ribeiro.emails]
[ribeiro.homepages]
[raedle]
name = "Jonas Rädle"
[raedle.emails]
raedle_email = "jonas.raedle@gmail.com"
raedle_email1 = "jonas.raedle@tum.de"
[raedle.homepages]
[peltier]
name = "Nicolas Peltier"
[peltier.emails]
peltier_email = "Nicolas.Peltier@imag.fr"
[peltier.homepages]
peltier_homepage = "http://membres-lig.imag.fr/peltier/"
[kappelmann]
name = "Kevin Kappelmann"
[kappelmann.emails]
kappelmann_email = "kevin.kappelmann@tum.de"
[kappelmann.homepages]
kappelmann_homepage = "https://www21.in.tum.de/team/kappelmk/"
[hoelzl]
name = "Johannes Hölzl"
[hoelzl.emails]
hoelzl_email = "hoelzl@in.tum.de"
[hoelzl.homepages]
hoelzl_homepage = "http://home.in.tum.de/~hoelzl"
[ballarin]
name = "Clemens Ballarin"
[ballarin.emails]
ballarin_email = "ballarin@in.tum.de"
[ballarin.homepages]
ballarin_homepage = "http://www21.in.tum.de/~ballarin/"
[wu]
name = "Chunhan Wu"
[wu.emails]
[wu.homepages]
[paulson]
name = "Lawrence C. Paulson"
[paulson.emails]
paulson_email = "lp15@cam.ac.uk"
[paulson.homepages]
paulson_homepage = "https://www.cl.cam.ac.uk/~lp15/"
[paleo]
name = "Bruno Woltzenlogel Paleo"
[paleo.emails]
[paleo.homepages]
paleo_homepage = "http://www.logic.at/staff/bruno/"
[wagner]
name = "Max Wagner"
[wagner.emails]
wagner_email = "max@trollbu.de"
[wagner.homepages]
[lochbihler]
name = "Andreas Lochbihler"
[lochbihler.emails]
lochbihler_email = "andreas.lochbihler@digitalasset.com"
lochbihler_email1 = "mail@andreas-lochbihler.de"
[lochbihler.homepages]
lochbihler_homepage = "http://www.andreas-lochbihler.de/"
[porter]
name = "Benjamin Porter"
[porter.emails]
[porter.homepages]
[boehme]
name = "Sascha Böhme"
[boehme.emails]
boehme_email = "boehmes@in.tum.de"
[boehme.homepages]
boehme_homepage = "http://www21.in.tum.de/~boehmes/"
[hou]
name = "Zhe Hou"
[hou.emails]
hou_email = "zhe.hou@ntu.edu.sg"
[hou.homepages]
[mitchell]
name = "Neil Mitchell"
[mitchell.emails]
[mitchell.homepages]
[gay]
name = "Richard Gay"
[gay.emails]
gay_email = "gay@mais.informatik.tu-darmstadt.de"
[gay.homepages]
[oldenburg]
name = "Lennart Oldenburg"
[oldenburg.emails]
[oldenburg.homepages]
[lochmann]
name = "Alexander Lochmann"
[lochmann.emails]
lochmann_email = "alexander.lochmann@uibk.ac.at"
[lochmann.homepages]
[lim]
name = "Japheth Lim"
[lim.emails]
[lim.homepages]
[keinholz]
name = "Jonas Keinholz"
[keinholz.emails]
[keinholz.homepages]
[taylor]
name = "Ramsay G. Taylor"
[taylor.emails]
taylor_email = "r.g.taylor@sheffield.ac.uk"
[taylor.homepages]
[bauereiss]
name = "Thomas Bauereiss"
[bauereiss.emails]
bauereiss_email = "thomas@bauereiss.name"
[bauereiss.homepages]
[lee]
name = "Holden Lee"
[lee.emails]
lee_email = "holdenl@princeton.edu"
[lee.homepages]
[weerwag]
name = "Timmy Weerwag"
[weerwag.emails]
[weerwag.homepages]
[sudhof]
name = "Henry Sudhof"
[sudhof.emails]
sudhof_email = "hsudhof@cs.tu-berlin.de"
[sudhof.homepages]
[nedzelsky]
name = "Michael Nedzelsky"
[nedzelsky.emails]
nedzelsky_email = "MichaelNedzelsky@yandex.ru"
[nedzelsky.homepages]
[romanos]
name = "Ralph Romanos"
[romanos.emails]
romanos_email = "ralph.romanos@student.ecp.fr"
[romanos.homepages]
[doczkal]
name = "Christian Doczkal"
[doczkal.emails]
doczkal_email = "doczkal@ps.uni-saarland.de"
[doczkal.homepages]
[buyse]
name = "Maxime Buyse"
[buyse.emails]
buyse_email = "maxime.buyse@polytechnique.edu"
[buyse.homepages]
[guiol]
name = "Hervé Guiol"
[guiol.emails]
guiol_email = "herve.guiol@univ-grenoble-alpes.fr"
[guiol.homepages]
[brodmann]
name = "Paul-David Brodmann"
[brodmann.emails]
brodmann_email = "p.brodmann@tu-berlin.de"
[brodmann.homepages]
[moedersheim]
name = "Sebastian Mödersheim"
[moedersheim.emails]
moedersheim_email = "samo@dtu.dk"
[moedersheim.homepages]
moedersheim_homepage = "https://people.compute.dtu.dk/samo/"
[hu]
name = "Shuwei Hu"
[hu.emails]
hu_email = "shuwei.hu@tum.de"
[hu.homepages]
[wand]
name = "Daniel Wand"
[wand.emails]
wand_email = "dwand@mpi-inf.mpg.de"
[wand.homepages]
[velykis]
name = "Andrius Velykis"
[velykis.emails]
[velykis.homepages]
velykis_homepage = "http://andrius.velykis.lt"
[felgenhauer]
name = "Bertram Felgenhauer"
[felgenhauer.emails]
felgenhauer_email = "bertram.felgenhauer@uibk.ac.at"
felgenhauer_email1 = "int-e@gmx.de"
[felgenhauer.homepages]
[sauer]
name = "Jens Sauer"
[sauer.emails]
sauer_email = "sauer@mais.informatik.tu-darmstadt.de"
[sauer.homepages]
[dittmann]
name = "Christoph Dittmann"
[dittmann.emails]
dittmann_email = "isabelle@christoph-d.de"
[dittmann.homepages]
dittmann_homepage = "http://logic.las.tu-berlin.de/Members/Dittmann/"
[muendler]
name = "Niels Mündler"
[muendler.emails]
muendler_email = "n.muendler@tum.de"
[muendler.homepages]
[somogyi]
name = "Dániel Somogyi"
[somogyi.emails]
[somogyi.homepages]
[makarios]
name = "T. J. M. Makarios"
[makarios.emails]
makarios_email = "tjm1983@gmail.com"
[makarios.homepages]
[nishihara]
name = "Toshiaki Nishihara"
[nishihara.emails]
[nishihara.homepages]
[losa]
name = "Giuliano Losa"
[losa.emails]
losa_email = "giuliano.losa@epfl.ch"
losa_email1 = "giuliano@galois.com"
losa_email2 = "giuliano@losa.fr"
[losa.homepages]
[grov]
name = "Gudmund Grov"
[grov.emails]
grov_email = "ggrov@inf.ed.ac.uk"
[grov.homepages]
grov_homepage = "http://homepages.inf.ed.ac.uk/ggrov"
[bharadwaj]
name = "Abhijith Bharadwaj"
[bharadwaj.emails]
[bharadwaj.homepages]
[clouston]
name = "Ranald Clouston"
[clouston.emails]
clouston_email = "ranald.clouston@cs.au.dk"
[clouston.homepages]
[jaskelioff]
name = "Mauro Jaskelioff"
[jaskelioff.emails]
[jaskelioff.homepages]
jaskelioff_homepage = "http://www.fceia.unr.edu.ar/~mauro/"
[caminati]
name = "Marco B. Caminati"
[caminati.emails]
[caminati.homepages]
[bengtson]
name = "Jesper Bengtson"
[bengtson.emails]
[bengtson.homepages]
bengtson_homepage = "http://www.itu.dk/people/jebe"
[boutry]
name = "Pierre Boutry"
[boutry.emails]
boutry_email = "boutry@unistra.fr"
[boutry.homepages]
[sternagelt]
name = "Thomas Sternagel"
[sternagelt.emails]
[sternagelt.homepages]
[guerraoui]
name = "Rachid Guerraoui"
[guerraoui.emails]
guerraoui_email = "rachid.guerraoui@epfl.ch"
[guerraoui.homepages]
[dongol]
name = "Brijesh Dongol"
[dongol.emails]
dongol_email = "brijesh.dongol@brunel.ac.uk"
[dongol.homepages]
[tuong]
name = "Frédéric Tuong"
[tuong.emails]
tuong_email = "tuong@users.gforge.inria.fr"
tuong_email1 = "ftuong@lri.fr"
[tuong.homepages]
tuong_homepage = "https://www.lri.fr/~ftuong/"
[ullrich]
name = "Sebastian Ullrich"
[ullrich.emails]
ullrich_email = "sebasti@nullri.ch"
[ullrich.homepages]
[essmann]
name = "Robin Eßmann"
[essmann.emails]
essmann_email = "robin.essmann@tum.de"
[essmann.homepages]
[liu]
name = "Junyi Liu"
[liu.emails]
[liu.homepages]
[villadsen]
name = "Jørgen Villadsen"
[villadsen.emails]
villadsen_email = "jovi@dtu.dk"
[villadsen.homepages]
villadsen_homepage = "https://people.compute.dtu.dk/jovi/"
[fosters]
name = "Simon Foster"
[fosters.emails]
fosters_email = "simon.foster@york.ac.uk"
[fosters.homepages]
fosters_homepage = "https://www-users.cs.york.ac.uk/~simonf/"
[dubut]
name = "Jérémy Dubut"
[dubut.emails]
dubut_email = "dubut@nii.ac.jp"
[dubut.homepages]
dubut_homepage = "http://group-mmm.org/~dubut/"
[jiang]
name = "Nan Jiang"
[jiang.emails]
jiang_email = "nanjiang@whu.edu.cn"
[jiang.homepages]
[hetzl]
name = "Stefan Hetzl"
[hetzl.emails]
hetzl_email = "hetzl@logic.at"
[hetzl.homepages]
hetzl_homepage = "http://www.logic.at/people/hetzl/"
[parkinson]
name = "Matthew Parkinson"
[parkinson.emails]
[parkinson.homepages]
parkinson_homepage = "http://research.microsoft.com/people/mattpark/"
[maletzky]
name = "Alexander Maletzky"
[maletzky.emails]
maletzky_email = "alexander.maletzky@risc.jku.at"
maletzky_email1 = "alexander.maletzky@risc-software.at"
[maletzky.homepages]
maletzky_homepage = "https://risc.jku.at/m/alexander-maletzky/"
[keefe]
name = "Greg O'Keefe"
[keefe.emails]
[keefe.homepages]
keefe_homepage = "http://users.rsise.anu.edu.au/~okeefe/"
[brandt]
name = "Felix Brandt"
[brandt.emails]
[brandt.homepages]
brandt_homepage = "http://dss.in.tum.de/staff/brandt.html"
[blasum]
name = "Holger Blasum"
[blasum.emails]
blasum_email = "holger.blasum@sysgo.com"
[blasum.homepages]
[messner]
name = "Florian Messner"
[messner.emails]
messner_email = "florian.g.messner@uibk.ac.at"
[messner.homepages]
[diaz]
name = "Javier Díaz"
[diaz.emails]
diaz_email = "javier.diaz.manzi@gmail.com"
[diaz.homepages]
[prathamesh]
name = "T.V.H. Prathamesh"
[prathamesh.emails]
prathamesh_email = "prathamesh@imsc.res.in"
[prathamesh.homepages]
[nestmann]
name = "Uwe Nestmann"
[nestmann.emails]
[nestmann.homepages]
nestmann_homepage = "https://www.mtv.tu-berlin.de/nestmann/"
[siek]
name = "Jeremy Siek"
[siek.emails]
siek_email = "jsiek@indiana.edu"
[siek.homepages]
siek_homepage = "http://homes.soic.indiana.edu/jsiek/"
[stock]
name = "Benedikt Stock"
[stock.emails]
stock_email = "benedikt1999@freenet.de"
[stock.homepages]
[boyton]
name = "Andrew Boyton"
[boyton.emails]
boyton_email = "andrew.boyton@nicta.com.au"
[boyton.homepages]
[taha]
name = "Safouan Taha"
[taha.emails]
taha_email = "safouan.taha@lri.fr"
[taha.homepages]
[ghourabi]
name = "Fadoua Ghourabi"
[ghourabi.emails]
ghourabi_email = "fadouaghourabi@gmail.com"
[ghourabi.homepages]
[brinkop]
name = "Hauke Brinkop"
[brinkop.emails]
brinkop_email = "hauke.brinkop@googlemail.com"
[brinkop.homepages]
[neumann]
name = "René Neumann"
[neumann.emails]
neumann_email = "rene.neumann@in.tum.de"
[neumann.homepages]
[schmaltz]
name = "Julien Schmaltz"
[schmaltz.emails]
schmaltz_email = "Julien.Schmaltz@ou.nl"
[schmaltz.homepages]
[haslbeck]
name = "Max W. Haslbeck"
[haslbeck.emails]
haslbeck_email = "maximilian.haslbeck@uibk.ac.at"
haslbeck_email1 = "haslbecm@in.tum.de"
haslbeck_email2 = "max.haslbeck@gmx.de"
[haslbeck.homepages]
haslbeck_homepage = "http://cl-informatik.uibk.ac.at/users/mhaslbeck/"
[reynaud]
name = "Alban Reynaud"
[reynaud.emails]
[reynaud.homepages]
[boulanger]
name = "Frédéric Boulanger"
[boulanger.emails]
boulanger_email = "frederic.boulanger@centralesupelec.fr"
[boulanger.homepages]
[spasic]
name = "Mirko Spasić"
[spasic.emails]
spasic_email = "mirko@matf.bg.ac.rs"
[spasic.homepages]
[heller]
name = "Armin Heller"
[heller.emails]
[heller.homepages]
[watt]
name = "Conrad Watt"
[watt.emails]
watt_email = "caw77@cam.ac.uk"
[watt.homepages]
watt_homepage = "http://www.cl.cam.ac.uk/~caw77/"
[hayes]
name = "Ian J. Hayes"
[hayes.emails]
hayes_email = "ian.hayes@itee.uq.edu.au"
[hayes.homepages]
[haslbeckm]
name = "Maximilian P. L. Haslbeck"
[haslbeckm.emails]
haslbeckm_email = "haslbema@in.tum.de"
[haslbeckm.homepages]
haslbeckm_homepage = "http://in.tum.de/~haslbema/"
[bortin]
name = "Maksym Bortin"
[bortin.emails]
bortin_email = "maksym.bortin@nicta.com.au"
[bortin.homepages]
+
+[klenze]
+name = "Tobias Klenze"
+
+[klenze.emails]
+klenze_email = "tobias.klenze@inf.ethz.ch"
+
+[klenze.homepages]
+
diff --git a/metadata/entries/IsaNet.toml b/metadata/entries/IsaNet.toml
new file mode 100644
--- /dev/null
+++ b/metadata/entries/IsaNet.toml
@@ -0,0 +1,60 @@
+title = "IsaNet: Formalization of a Verification Framework for Secure Data Plane Protocols"
+date = 2022-06-08
+topics = [
+ "Computer science/Security",
+ "Computer science/Networks",
+]
+abstract = """
+Today's Internet is built on decades-old networking protocols
+that lack scalability, reliability and security. In response, the
+networking community has developed <em>path-aware</em> Internet
+architectures that solve these issues while simultaneously empowering
+end hosts. In these architectures, autonomous systems authorize
+forwarding paths in accordance with their routing policies, and
+protect paths using cryptographic authenticators. For each packet, the
+sending end host selects an authorized path and embeds it and its
+authenticators in the packet header. This allows routers to
+efficiently determine how to forward the packet. The central security
+property of the data plane, i.e., of forwarding, is that packets can
+only travel along authorized paths. This property, which we call
+<em>path authorization</em>, protects the routing policies of autonomous
+systems from malicious senders. The fundamental role of packet
+forwarding in the Internet's ecosystem and the complexity of the
+authentication mechanisms employed call for a formal analysis. We
+develop IsaNet, a parameterized verification framework for data plane
+protocols in Isabelle/HOL. We first formulate an abstract model
+without an attacker for which we prove path authorization. We then
+refine this model by introducing a Dolev--Yao attacker and by
+protecting authorized paths using (generic) cryptographic validation
+fields. This model is parametrized by the path authorization mechanism
+and assumes five simple verification conditions. We propose novel
+attacker models and different sets of assumptions on the underlying
+routing protocol. We validate our framework by instantiating it with
+nine concrete protocols variants and prove that they each satisfy the
+verification conditions (and hence path authorization). The invariants
+needed for the security proof are proven in the parametrized model
+instead of the instance models. Our framework thus supports low-effort
+security proofs for data plane protocols. In contrast to what could be
+achieved with state-of-the-art automated protocol verifiers, our
+results hold for arbitrary network topologies and sets of authorized
+paths."""
+license = "bsd"
+note = ""
+
+[authors]
+
+[authors.klenze]
+email = "klenze_email"
+
+[authors.sprenger]
+email = "sprenger_email"
+
+[contributors]
+
+[notify]
+klenze = "klenze_email"
+sprenger = "sprenger_email"
+
+[history]
+
+[extra]
diff --git a/metadata/releases.toml b/metadata/releases.toml
--- a/metadata/releases.toml
+++ b/metadata/releases.toml
@@ -1,5676 +1,7078 @@
[ADS_Functor]
-2020 = 2020-04-27
-2021 = 2021-12-14
+2020-04-27 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[AI_Planning_Languages_Semantics]
-2020 = 2020-10-30
-2021 = 2021-12-14
+2020-10-30 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[AODV]
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2014-11-01 = "2014"
+2014-11-03 = "2014"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[AVL-Trees]
-2003 = 2004-03-19
-2004 = 2004-05-21
-2005 = 2005-10-14
-2007 = 2007-11-27
-2008 = 2008-06-10
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2004-03-19 = "2003"
+2004-04-20 = "2004"
+2004-05-21 = "2004"
+2005-10-14 = "2005"
+2007-11-27 = "2007"
+2008-06-10 = "2008"
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[AWN]
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2014-03-15 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Abortable_Linearizable_Modules]
-2011-1 = 2012-03-02
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2012-03-02 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Abs_Int_ITP2012]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Abstract-Hoare-Logics]
-2007 = 2007-11-27
-2008 = 2008-06-10
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2007-11-27 = "2007"
+2008-06-10 = "2008"
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Abstract-Rewriting]
-2009-1 = 2010-06-17
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2010-06-17 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Abstract_Completeness]
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2014-04-16 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Abstract_Soundness]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
-
-[Ackermanns_not_PR]
-2021 = 2021-12-14
-
-[Actuarial_Mathematics]
-2021 = 2021-12-14
+2017-02-13 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Adaptive_State_Counting]
-2019 = 2019-08-19
-2020 = 2020-04-18
-2021 = 2021-12-14
+2019-08-19 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Affine_Arithmetic]
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Aggregation_Algebras]
-2018 = 2018-09-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2018-09-16 = "2018"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Akra_Bazzi]
-2015 = 2015-07-24
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2015-07-15 = "2015"
+2015-07-24 = "2015"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Algebraic_Numbers]
-2015 = 2015-12-22
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2015-12-22 = "2015"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Algebraic_VCs]
-2016 = 2016-06-18
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-06-18 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Allen_Calculus]
-2016 = 2016-10-05
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-28
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-09-29 = "2016"
+2016-10-05 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2019-06-28 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Amicable_Numbers]
-2020 = 2020-08-15
-2021 = 2021-12-14
+2020-08-15 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Amortized_Complexity]
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2015 = 2015-05-28
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2014-08-28 = "2013-2"
+2015-05-19 = "2014"
+2015-05-27 = "2014"
+2015-05-28 = "2015"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[AnselmGod]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-09-08 = "2016-1"
+2017-09-11 = "2016-1"
+2017-09-18 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Applicative_Lifting]
-2015 = 2015-12-22
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2015-12-22 = "2015"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Approximation_Algorithms]
-2019 = 2020-01-16
-2020 = 2020-04-18
-2021 = 2021-12-14
+2020-01-16 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Architectural_Design_Patterns]
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2018-03-01 = "2017"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Aristotles_Assertoric_Syllogistic]
-2019 = 2019-10-17
-2020 = 2020-04-18
-2021 = 2021-12-14
+2019-10-17 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Arith_Prog_Rel_Primes]
-2019 = 2020-02-10
-2020 = 2020-04-18
-2021 = 2021-12-14
+2020-02-10 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[ArrowImpossibilityGS]
-2009 = 2009-09-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-03-02
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2009-04-29 = "2009"
+2009-09-29 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-03-02 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Attack_Trees]
-2021 = 2021-12-14
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Auto2_HOL]
-2018 = 2018-11-29
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2018-11-29 = "2018"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Auto2_Imperative_HOL]
-2018 = 2019-01-22
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2019-01-22 = "2018"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[AutoFocus-Stream]
-2011 = 2011-02-24
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-03-08
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2011-02-24 = "2011"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-03-08 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Automated_Stateful_Protocol_Verification]
-2020 = 2020-05-20
-2021 = 2021-12-14
+2020-05-20 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Automatic_Refinement]
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[AxiomaticCategoryTheory]
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2018-05-23 = "2017"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[BDD]
-2007 = 2008-03-07
-2008 = 2008-06-10
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2008-03-07 = "2007"
+2008-06-10 = "2008"
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[BD_Security_Compositional]
-2021 = 2021-12-14
+2021-12-14 = "2021"
[BNF_CC]
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2018-04-25 = "2017"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[BNF_Operations]
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[BTree]
-2021 = 2021-12-14
+2021-02-26 = "2021"
+2021-12-14 = "2021"
[Banach_Steinhaus]
-2020 = 2020-05-11
-2021 = 2021-12-14
+2020-05-06 = "2020"
+2020-05-11 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Belief_Revision]
-2021 = 2021-12-14
+2021-10-22 = "2021"
+2021-12-14 = "2021"
[Bell_Numbers_Spivey]
-2016 = 2016-05-04
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-05-04 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[BenOr_Kozen_Reif]
-2021 = 2021-12-14
+2021-04-25 = "2021"
+2021-12-14 = "2021"
[Berlekamp_Zassenhaus]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2018 = 2018-09-07
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2018-09-07 = "2018"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Bernoulli]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-01-24 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Bertrands_Postulate]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-01-18 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Bicategory]
-2019 = 2020-01-09
-2020 = 2020-04-18
-2021 = 2021-12-14
+2020-01-09 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[BinarySearchTree]
-2004 = 2004-09-21
-2005 = 2005-10-14
-2007 = 2007-11-27
-2008 = 2008-06-10
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2004-04-20 = "2004"
+2004-04-21 = "2004"
+2004-09-21 = "2004"
+2005-10-14 = "2005"
+2007-11-27 = "2007"
+2008-06-10 = "2008"
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Binding_Syntax_Theory]
-2018 = 2019-04-08
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2019-04-08 = "2018"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Binomial-Heaps]
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-03-02
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2010-10-28 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-03-02 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Binomial-Queues]
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[BirdKMP]
-2020 = 2020-09-02
-2021 = 2021-12-14
+2020-09-02 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Blue_Eyes]
-2020 = 2021-02-01
-2021 = 2021-12-14
+2021-02-01 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Bondy]
-2012 = 2012-10-27
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2012-10-27 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Boolean_Expression_Checkers]
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2014-06-08 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Bounded_Deducibility_Security]
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2014-04-24 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Buchi_Complementation]
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-10-27 = "2017"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Budan_Fourier]
-2018 = 2018-09-04
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2018-09-04 = "2018"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Buffons_Needle]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-06-06 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Buildings]
-2016 = 2016-07-01
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-07-01 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[BytecodeLogicJmlTypes]
-2008 = 2008-12-22
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2008-12-22 = "2008"
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[C2KA_DistributedSystems]
-2019 = 2019-08-06
-2020 = 2020-04-18
-2021 = 2021-12-14
+2019-08-06 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[CAVA_Automata]
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2014-05-29 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[CAVA_LTL_Modelchecker]
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2014-05-29 = "2013-2"
+2014-05-30 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[CCS]
-2012 = 2012-06-14
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2012-06-14 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[CISC-Kernel]
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2014-07-18 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[CRDT]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-07-07 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[CSP_RefTK]
-2020 = 2021-01-12
-2021 = 2021-12-14
+2021-01-12 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[CYK]
-2016 = 2016-04-27
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-04-27 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[CZH_Elementary_Categories]
-2021 = 2021-12-14
+2021-09-14 = "2021"
+2021-10-05 = "2021"
+2021-12-14 = "2021"
[CZH_Foundations]
-2021 = 2021-12-14
+2021-09-14 = "2021"
+2021-10-05 = "2021"
+2021-12-14 = "2021"
[CZH_Universal_Constructions]
-2021 = 2021-12-14
+2021-09-14 = "2021"
+2021-10-05 = "2021"
+2021-12-14 = "2021"
[CakeML]
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[CakeML_Codegen]
-2019 = 2019-07-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2019-07-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Call_Arity]
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2015-02-20 = "2014"
+2015-02-21 = "2014"
+2015-05-11 = "2014"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Card_Equiv_Relations]
-2016 = 2016-05-24
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-05-24 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Card_Multisets]
-2016 = 2016-06-26
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-06-26 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Card_Number_Partitions]
-2015 = 2016-01-14
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-01-14 = "2015"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Card_Partitions]
-2015 = 2015-12-13
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2015-12-13 = "2015"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Cartan_FP]
-2016 = 2016-03-09
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-03-09 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Case_Labeling]
-2015 = 2015-08-17
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2015-07-24 = "2015"
+2015-07-27 = "2015"
+2015-08-17 = "2015"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Catalan_Numbers]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Category]
-2004 = 2005-05-01
-2005 = 2005-10-14
-2007 = 2007-11-27
-2008 = 2008-06-10
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-03-02
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2005-04-21 = "2004"
+2005-05-01 = "2004"
+2005-10-14 = "2005"
+2007-11-27 = "2007"
+2008-06-10 = "2008"
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-03-02 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Category2]
-2009-1 = 2010-06-21
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-03-02
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2010-06-21 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-03-02 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Category3]
-2016 = 2016-06-26
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-06-26 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Cauchy]
-2005 = 2006-03-14
-2007 = 2007-11-27
-2008 = 2008-06-10
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2006-03-14 = "2005"
+2007-11-27 = "2007"
+2008-06-10 = "2008"
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Cayley_Hamilton]
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2014-09-16 = "2014"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Certification_Monads]
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2014-10-08 = "2014"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Chandy_Lamport]
-2020 = 2020-08-04
-2021 = 2021-12-14
+2020-08-04 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Chord_Segments]
-2016 = 2016-10-11
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-10-11 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Circus]
-2012 = 2012-05-29
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2012-05-29 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Clean]
-2019 = 2019-10-16
-2020 = 2020-04-18
-2021 = 2021-12-14
-
-[Clique_and_Monotone_Circuits]
-2021 = 2021-12-14
+2019-10-16 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[ClockSynchInst]
-2005 = 2006-03-15
-2007 = 2007-11-27
-2008 = 2008-06-10
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-03-02
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2006-03-15 = "2005"
+2007-11-27 = "2007"
+2008-06-10 = "2008"
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-03-02 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Closest_Pair_Points]
-2019 = 2020-01-14
-2020 = 2020-04-18
-2021 = 2021-12-14
+2020-01-14 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[CoCon]
-2021 = 2021-12-14
+2021-12-14 = "2021"
[CoSMeDis]
-2021 = 2021-12-14
+2021-12-14 = "2021"
[CoSMed]
-2021 = 2021-12-14
+2021-12-14 = "2021"
[CofGroups]
-2009 = 2009-09-05
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-03-02
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2009-08-09 = "2009"
+2009-09-05 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-03-02 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Coinductive]
-2009-1 = 2010-02-15
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-03-02
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2010-02-14 = "2009-1"
+2010-02-15 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-03-02 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Coinductive_Languages]
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Collections]
-2009 = 2009-11-29
-2009-1 = 2009-12-13
-2009-2 = 2011-02-11
-2011-1 = 2011-10-12
-2012 = 2012-05-24
-2013 = 2013-03-02
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
-
-[Combinable_Wands]
-2021 = 2021-12-14
+2009-11-29 = "2009"
+2009-12-12 = "2009-1"
+2009-12-13 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2011-10-12 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-03-02 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Combinatorics_Words]
-2021 = 2021-12-14
+2021-05-26 = "2021"
+2021-12-14 = "2021"
[Combinatorics_Words_Graph_Lemma]
-2021 = 2021-12-14
+2021-05-26 = "2021"
+2021-12-14 = "2021"
[Combinatorics_Words_Lyndon]
-2021 = 2021-12-14
+2021-05-26 = "2021"
+2021-12-14 = "2021"
[Comparison_Sort_Lower_Bound]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-03-16 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Compiling-Exceptions-Correctly]
-2004 = 2004-07-09
-2005 = 2005-10-14
-2007 = 2007-11-27
-2008 = 2008-06-10
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2004-07-09 = "2004"
+2005-10-14 = "2005"
+2007-11-27 = "2007"
+2008-06-10 = "2008"
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Complete_Non_Orders]
-2019 = 2019-06-28
-2020 = 2020-04-18
-2021 = 2021-12-14
+2019-06-28 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Completeness]
-2004 = 2005-07-22
-2005 = 2005-10-14
-2007 = 2007-11-27
-2008 = 2008-06-10
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-03-02
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2004-09-20 = "2004"
+2004-09-21 = "2004"
+2005-07-22 = "2004"
+2005-10-14 = "2005"
+2007-11-27 = "2007"
+2008-06-10 = "2008"
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-03-02 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Complex_Bounded_Operators]
-2021 = 2021-12-14
+2021-09-20 = "2021"
+2021-12-14 = "2021"
[Complex_Geometry]
-2019 = 2020-01-17
-2020 = 2020-04-18
-2021 = 2021-12-14
+2020-01-17 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Complx]
-2016 = 2016-11-29
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-11-29 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[ComponentDependencies]
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2014-04-29 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[ConcurrentGC]
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2015-04-15 = "2014"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[ConcurrentIMP]
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2015-04-15 = "2014"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Concurrent_Ref_Alg]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-01-04 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Concurrent_Revisions]
-2018 = 2019-01-03
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2019-01-03 = "2018"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Conditional_Simplification]
-2021 = 2021-12-14
+2021-09-14 = "2021"
+2021-10-05 = "2021"
+2021-12-14 = "2021"
[Conditional_Transfer_Rule]
-2021 = 2021-12-14
+2021-09-14 = "2021"
+2021-10-13 = "2021"
+2021-12-14 = "2021"
[Consensus_Refined]
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2015-03-19 = "2014"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Constructive_Cryptography]
-2018 = 2018-12-20
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2018-12-19 = "2018"
+2018-12-20 = "2018"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Constructive_Cryptography_CM]
-2021 = 2021-12-14
+2021-03-18 = "2021"
+2021-12-14 = "2021"
[Constructor_Funs]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-04-20 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Containers]
-2013 = 2013-04-23
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2013-04-23 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
["CoreC++"]
-2005 = 2006-05-16
-2007 = 2007-11-27
-2008 = 2008-06-10
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-03-02
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2006-05-16 = "2005"
+2007-11-27 = "2007"
+2008-06-10 = "2008"
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-03-02 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Core_DOM]
-2018 = 2019-01-07
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2019-01-07 = "2018"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Core_SC_DOM]
-2020 = 2020-11-26
-2021 = 2021-12-14
+2020-11-26 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Correctness_Algebras]
-2021 = 2021-12-14
-
-[Cotangent_PFD_Formula]
-2021 = 2021-12-14
+2021-10-20 = "2021"
+2021-12-14 = "2021"
[Count_Complex_Roots]
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-10-18 = "2017"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[CryptHOL]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-05-11 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[CryptoBasedCompositionalProperties]
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2014-01-11 = "2013-2"
+2014-01-14 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Cubic_Quartic_Equations]
-2021 = 2021-12-14
+2021-09-03 = "2021"
+2021-12-14 = "2021"
[DFS_Framework]
-2016 = 2016-07-05
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2020-01-14
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-07-05 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-01-14 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[DOM_Components]
-2021 = 2021-12-14
-
-[DPRM_Theorem]
-2021 = 2021-12-14
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[DPT-SAT-Solver]
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2015 = 2015-07-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2015-07-27 = "2015"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[DataRefinementIBP]
-2009-1 = 2010-05-28
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2010-05-28 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Datatype_Order_Generator]
-2012 = 2012-08-07
-2013 = 2013-03-02
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2012-08-07 = "2012"
+2013-02-16 = "2013"
+2013-03-02 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Decl_Sem_Fun_PL]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-07-24 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Decreasing-Diagrams]
-2013-1 = 2013-12-02
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2013-11-18 = "2013-1"
+2013-12-02 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Decreasing-Diagrams-II]
-2015 = 2015-08-21
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
-
-[Dedekind_Real]
-2021 = 2021-12-14
+2015-08-21 = "2015"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Deep_Learning]
-2016 = 2016-11-10
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-11-10 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Delta_System_Lemma]
-2020 = 2020-12-28
-2021 = 2021-12-14
+2020-12-28 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Density_Compiler]
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2014-10-09 = "2014"
+2014-12-22 = "2014"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Dependent_SIFUM_Refinement]
-2016 = 2016-06-28
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-06-28 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Dependent_SIFUM_Type_Systems]
-2016 = 2016-06-25
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-06-25 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Depth-First-Search]
-2004 = 2004-06-24
-2005 = 2005-10-14
-2007 = 2007-11-27
-2008 = 2008-06-10
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2004-06-24 = "2004"
+2005-10-14 = "2005"
+2007-11-27 = "2007"
+2008-06-10 = "2008"
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Derangements]
-2015 = 2015-11-20
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2015-06-28 = "2015"
+2015-11-20 = "2015"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Deriving]
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Descartes_Sign_Rule]
-2015 = 2016-01-05
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-01-05 = "2015"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Design_Theory]
-2021 = 2021-12-14
+2021-09-02 = "2021"
+2021-12-14 = "2021"
[Dict_Construction]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Differential_Dynamic_Logic]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-02-14 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Differential_Game_Logic]
-2019 = 2019-06-24
-2020 = 2020-04-18
-2021 = 2021-12-14
-
-[Digit_Expansions]
-2021 = 2021-12-14
+2019-06-24 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Dijkstra_Shortest_Path]
-2011-1 = 2012-03-15
-2012 = 2012-05-24
-2013 = 2013-03-08
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2012-02-10 = "2011-1"
+2012-03-15 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-03-08 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Diophantine_Eqns_Lin_Hom]
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-10-15 = "2017"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Dirichlet_L]
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Dirichlet_Series]
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-10-16 = "2017"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[DiscretePricing]
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2018-07-18 = "2017"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Discrete_Summation]
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2014-04-13 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[DiskPaxos]
-2004 = 2005-06-22
-2005 = 2005-10-14
-2007 = 2007-11-27
-2008 = 2008-06-10
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2005-06-22 = "2004"
+2005-10-14 = "2005"
+2007-11-27 = "2007"
+2008-06-10 = "2008"
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Dominance_CHK]
-2021 = 2021-12-14
+2021-09-07 = "2021"
+2021-12-14 = "2021"
[DynamicArchitectures]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-07-31 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Dynamic_Tables]
-2015 = 2015-06-08
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2015-06-07 = "2015"
+2015-06-08 = "2015"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[E_Transcendental]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-01-13 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Echelon_Form]
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2015-02-12 = "2014"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[EdmondsKarp_Maxflow]
-2016 = 2016-08-12
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-08-12 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Efficient-Mergesort]
-2011-1 = 2011-11-10
-2012 = 2012-05-24
-2013 = 2013-03-02
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2011-11-10 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-03-02 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Elliptic_Curves_Group_Law]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-03-01 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Encodability_Process_Calculi]
-2015 = 2015-08-11
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2015-08-11 = "2015"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Epistemic_Logic]
-2018 = 2018-10-29
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
-
-[Equivalence_Relation_Enumeration]
-2021 = 2021-12-14
+2018-10-29 = "2018"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Ergodic_Theory]
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Error_Function]
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2018-02-07 = "2017"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Euler_MacLaurin]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-03-14 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Euler_Partition]
-2015 = 2015-11-20
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
-
-[Eval_FO]
-2021 = 2021-12-14
-
-[Example-Submission]
-2021 = 2021-12-14
+2015-11-20 = "2015"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Extended_Finite_State_Machine_Inference]
-2020 = 2020-09-19
-2021 = 2021-12-14
+2020-09-19 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Extended_Finite_State_Machines]
-2020 = 2020-09-19
-2021 = 2021-12-14
+2020-09-19 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[FFT]
-2005 = 2005-10-14
-2007 = 2007-11-27
-2008 = 2008-06-10
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2005-10-14 = "2005"
+2007-11-27 = "2007"
+2008-06-10 = "2008"
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[FLP]
-2016 = 2016-05-18
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-05-18 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[FOL-Fitting]
-2007 = 2007-11-27
-2008 = 2008-06-10
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-03-02
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2007-11-27 = "2007"
+2008-06-10 = "2008"
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-03-02 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[FOL_Axiomatic]
-2021 = 2021-12-14
+2021-10-05 = "2021"
+2021-12-14 = "2021"
[FOL_Harrison]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-01-04 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[FOL_Seq_Calc1]
-2019 = 2019-07-18
-2020 = 2020-04-18
-2021 = 2021-12-14
-
-[FOL_Seq_Calc2]
-2021 = 2021-12-14
-
-[FOL_Seq_Calc3]
-2021 = 2021-12-14
-
-[FO_Theory_Rewriting]
-2021 = 2021-12-14
+2019-07-18 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Factor_Algebraic_Polynomial]
-2021 = 2021-12-14
+2021-11-14 = "2021"
+2021-12-14 = "2021"
[Factored_Transition_System_Bounding]
-2018 = 2018-10-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2018-10-16 = "2018"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Falling_Factorial_Sum]
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-12-30 = "2017"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Farkas]
-2018 = 2019-01-21
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2019-01-21 = "2018"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[FeatherweightJava]
-2005 = 2006-04-06
-2007 = 2007-11-27
-2008 = 2008-06-10
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2006-04-05 = "2005"
+2006-04-06 = "2005"
+2007-11-27 = "2007"
+2008-06-10 = "2008"
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Featherweight_OCL]
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2014-01-16 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Fermat3_4]
-2007 = 2007-11-27
-2008 = 2008-06-10
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2007-11-27 = "2007"
+2008-06-10 = "2008"
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[FileRefinement]
-2004 = 2004-12-15
-2005 = 2005-10-14
-2007 = 2007-11-27
-2008 = 2008-06-10
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2004-12-15 = "2004"
+2005-10-14 = "2005"
+2007-11-27 = "2007"
+2008-06-10 = "2008"
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[FinFun]
-2009 = 2009-05-25
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-03-02
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2009-05-25 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-03-02 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Finger-Trees]
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-03-02
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2010-10-28 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-03-02 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Finite-Map-Extras]
-2020 = 2020-12-02
-2021 = 2021-12-14
+2020-12-02 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Finite_Automata_HF]
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
-
-[Finite_Fields]
-2021 = 2021-12-14
+2015-02-05 = "2014"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Finitely_Generated_Abelian_Groups]
-2021 = 2021-12-14
+2021-07-13 = "2021"
+2021-12-14 = "2021"
[First_Order_Terms]
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2018-02-06 = "2017"
+2018-02-07 = "2017"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[First_Welfare_Theorem]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-09-04 = "2016-1"
+2017-09-05 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Fishburn_Impossibility]
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2018-03-23 = "2017"
+2018-06-10 = "2017"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Fisher_Yates]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
-
-[Fishers_Inequality]
-2021 = 2021-12-14
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Flow_Networks]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2020-01-14
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-06-02 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-01-14 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Floyd_Warshall]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-05-09 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Flyspeck-Tame]
-2007 = 2008-01-04
-2008 = 2008-06-10
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-25
-2013 = 2013-03-02
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2018 = 2018-08-17
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2007-11-27 = "2007"
+2008-01-04 = "2007"
+2008-06-10 = "2008"
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-25 = "2012"
+2013-02-16 = "2013"
+2013-03-02 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-17 = "2018"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[FocusStreamsCaseStudies]
-2013-1 = 2013-11-18
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2013-11-18 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Forcing]
-2020 = 2020-05-07
-2021 = 2021-12-14
+2020-05-06 = "2020"
+2020-05-07 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Formal_Puiseux_Series]
-2021 = 2021-12-14
+2021-02-24 = "2021"
+2021-12-14 = "2021"
[Formal_SSA]
-2015 = 2016-02-08
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2016-02-08 = "2015"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Formula_Derivatives]
-2015 = 2015-05-28
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2015-05-28 = "2015"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Foundation_of_geometry]
-2021 = 2021-12-14
+2021-12-13 = "2021"
+2021-12-14 = "2021"
[Fourier]
-2019 = 2019-09-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2019-09-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Free-Boolean-Algebra]
-2009-1 = 2010-03-29
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-03-02
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2010-03-29 = "2009-1"
+2010-06-30 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-03-02 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Free-Groups]
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
-
-[Frequency_Moments]
-2021 = 2021-12-14
+2010-07-01 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Fresh_Identifiers]
-2021 = 2021-12-14
+2021-08-18 = "2021"
+2021-12-14 = "2021"
[FunWithFunctions]
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-07-01 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[FunWithTilings]
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-02-16
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-07-01 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Functional-Automata]
-2003 = 2004-03-30
-2004 = 2004-05-21
-2005 = 2005-10-14
-2007 = 2007-11-27
-2008 = 2008-06-10
-2009 = 2009-04-29
-2009-1 = 2009-12-12
-2009-2 = 2011-02-11
-2011-1 = 2011-10-11
-2012 = 2012-05-24
-2013 = 2013-03-02
-2013-1 = 2013-11-17
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2004-03-30 = "2003"
+2004-04-20 = "2004"
+2004-05-21 = "2004"
+2005-10-14 = "2005"
+2007-11-27 = "2007"
+2008-06-10 = "2008"
+2009-04-29 = "2009"
+2009-12-12 = "2009-1"
+2010-07-01 = "2009-2"
+2011-02-11 = "2009-2"
+2011-10-11 = "2011-1"
+2012-05-24 = "2012"
+2013-02-16 = "2013"
+2013-03-02 = "2013"
+2013-11-17 = "2013-1"
+2013-12-11 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Functional_Ordered_Resolution_Prover]
-2018 = 2018-11-29
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2018-11-29 = "2018"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Furstenberg_Topology]
-2019 = 2020-03-27
-2020 = 2020-04-18
-2021 = 2021-12-14
+2020-03-27 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[GPU_Kernel_PL]
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2014-04-06 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[Gabow_SCC]
-2013-2 = 2014-08-28
-2014 = 2015-05-27
-2016 = 2016-02-22
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2014-05-29 = "2013-2"
+2014-08-28 = "2013-2"
+2015-05-27 = "2014"
+2016-02-22 = "2016"
+2016-12-17 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"
+2019-06-11 = "2019"
+2020-04-18 = "2020"
+2021-02-23 = "2021"
+2021-12-14 = "2021"
[GaleStewart_Games]
-2021 = 2021-12-14
-
-[Gale_Shapley]
-2021 = 2021-12-14
+2021-04-28 = "2021"
+2021-12-14 = "2021"
[Game_Based_Crypto]
-2016-1 = 2017-10-10
-2017 = 2018-08-16
-2019 = 2019-06-11
-2020 = 2020-04-18
-2021 = 2021-12-14
+2017-05-11 = "2016-1"
+2017-10-10 = "2016-1"
+2018-08-16 = "2017"