-
Notifications
You must be signed in to change notification settings - Fork 0
/
H10.v
25 lines (20 loc) · 1.03 KB
/
H10.v
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
(**************************************************************)
(* Copyright Dominique Larchey-Wendling [*] *)
(* *)
(* [*] Affiliation LORIA -- CNRS *)
(**************************************************************)
(* This file is distributed under the terms of the *)
(* CeCILL v2 FREE SOFTWARE LICENSE AGREEMENT *)
(**************************************************************)
From Undecidability.Shared.Libs.DLW Require Import pos vec.
From Undecidability.H10.Dio Require Import dio_single.
Set Implicit Arguments.
(* Hilbert's Tenth problem: given a diophantine equation with n
variable and no parameters, does it have a solution *)
Definition H10_PROBLEM := { n : nat & dio_polynomial (pos n) (pos 0)
* dio_polynomial (pos n) (pos 0) }%type.
Definition H10 : H10_PROBLEM -> Prop.
Proof.
intros (n & p & q).
apply (dio_single_pred (p,q)), (fun _ => 0).
Defined.