Library hydras.Ackermann.PAconsistent

PAconsistent.v
Original file by Russel O' Connor

From Coq Require Import Arith.
From hydras.Ackermann Require Import folProof folProp PA model.

Definition natModel : Model LNT :=
  model LNT nat
    (fun f : Functions LNT
     match f return (naryFunc nat (arityF LNT f)) with
     | Languages.Plus_fun x y : naty + x
     | Languages.Times_fun x y : naty × x
     | Languages.Succ_S
     | Languages.Zero_ ⇒ 0
     end)
    (fun r : Relations LNTmatch r with end).

Theorem PAconsistent : Consistent LNT PA.