Skip to content

Commit

Permalink
doc(citation.md): Add a citation.md file (#17202)
Browse files Browse the repository at this point in the history
Creating a PR as suggested [here](https://leanprover.zulipchat.com/#narrow/stream/113488-general/topic/Citing.20lean.20.2B.20mathlib/near/306109993). Feel free to suggest or directly commit changes to the wording.
  • Loading branch information
BoltonBailey committed Nov 6, 2022
1 parent 8efef27 commit e8ecfea
Show file tree
Hide file tree
Showing 2 changed files with 75 additions and 1 deletion.
43 changes: 43 additions & 0 deletions CITATION.md
@@ -0,0 +1,43 @@

# Citing Mathlib

You can cite `mathlib` using the following BibTeX entry:

```bib
@InProceedings{ mathlib2020,
author = {The mathlib Community},
title = {The Lean Mathematical Library},
year = {2020},
isbn = {9781450370974},
publisher = {Association for Computing Machinery},
address = {New York, NY, USA},
url = {https://doi.org/10.1145/3372885.3373824},
doi = {10.1145/3372885.3373824},
booktitle = {Proceedings of the 9th ACM SIGPLAN International
Conference on Certified Programs and Proofs},
pages = {367-381},
numpages = {15},
keywords = {formal proof, formal library, Lean, mathlib},
location = {New Orleans, LA, USA},
series = {CPP 2020}
}
```

The `mathlib` project is actively maintained and updated. In the interest of reproducibility, you may want to manage your code's dependency on `mathlib` using the [`leanproject`](https://leanprover-community.github.io/leanproject.html) command-line tool. This will help ensure others can retrieve the right version of `mathlib` for your project.

Lean was introduced in the paper ["The Lean Theorem Prover"](https://www.semanticscholar.org/paper/The-Lean-Theorem-Prover-(System-Description)-Moura-Kong/2a441a46e228ed0ea2251a4e61be6c7025b45766), by de Moura et al., which you can cite using:

```bib
@InProceedings{ demoura2015lean,
author = {de Moura, Leonardo and Kong, Soonho and Avigad, Jeremy and
van Doorn, Floris and von Raumer, Jakob},
editor = {Felty, Amy P. and Middeldorp, Aart},
title = {The Lean Theorem Prover (System Description)},
booktitle = {Automated Deduction - CADE-25},
year = {2015},
publisher = {Springer International Publishing},
address = {Cham},
pages = {378--388},
isbn = {978-3-319-21401-6}
}
```
33 changes: 32 additions & 1 deletion docs/references.bib
Expand Up @@ -574,6 +574,19 @@ @InProceedings{ deligne_formulaire
mrreviewer = {Jacques Velu}
}

@InProceedings{ demoura2015lean,
author = {de Moura, Leonardo and Kong, Soonho and Avigad, Jeremy and
van Doorn, Floris and von Raumer, Jakob},
editor = {Felty, Amy P. and Middeldorp, Aart},
title = {The Lean Theorem Prover (System Description)},
booktitle = {Automated Deduction - CADE-25},
year = {2015},
publisher = {Springer International Publishing},
address = {Cham},
pages = {378--388},
isbn = {978-3-319-21401-6}
}

@Article{ dold1958,
author = {Dold, Albrecht},
title = {Homology of symmetric products and other functors of
Expand Down Expand Up @@ -1379,7 +1392,25 @@ @Article{ markowsky1976
author = {Markowsky, George},
year = {1976},
month = {Dec},
pages = {53–68}
pages = {53-68}
}

@InProceedings{ mathlib2020,
author = {The mathlib Community},
title = {The Lean Mathematical Library},
year = {2020},
isbn = {9781450370974},
publisher = {Association for Computing Machinery},
address = {New York, NY, USA},
url = {https://doi.org/10.1145/3372885.3373824},
doi = {10.1145/3372885.3373824},
booktitle = {Proceedings of the 9th ACM SIGPLAN International
Conference on Certified Programs and Proofs},
pages = {367-381},
numpages = {15},
keywords = {formal proof, formal library, Lean, mathlib},
location = {New Orleans, LA, USA},
series = {CPP 2020}
}

@InProceedings{ mcbride1996,
Expand Down

0 comments on commit e8ecfea

Please sign in to comment.