Skip to content

Commit

Permalink
chore(number_theory/dioph): fix docs (#12011)
Browse files Browse the repository at this point in the history
  • Loading branch information
ericrbg committed Feb 13, 2022
1 parent af1355c commit b08dc17
Showing 1 changed file with 3 additions and 1 deletion.
4 changes: 3 additions & 1 deletion src/number_theory/dioph.lean
Expand Up @@ -23,7 +23,9 @@ there exists `t : ℕ^β` with `p (v, t) = 0`.
* `is_poly`: a predicate stating that a function is a multivariate integer polynomial.
* `poly`: the type of multivariate integer polynomial functions.
* `dioph`: a predicate stating that a set `S ⊆ ℕ^α` is Diophantine, i.e. that
* `dioph`: a predicate stating that a set is Diophantine, i.e. a set `S ⊆ ℕ^α` is
Diophantine if there exists a polynomial on `α ⊕ β` such that `v ∈ S` iff there
exists `t : ℕ^β` with `p (v, t) = 0`.
* `dioph_fn`: a predicate on a function stating that it is Diophantine in the sense that its graph
is Diophantine as a set.
Expand Down

0 comments on commit b08dc17

Please sign in to comment.