Skip to content

Commit b967df4

Browse files
update to Coq 8.20
1 parent f2ff92e commit b967df4

File tree

10 files changed

+26
-15
lines changed

10 files changed

+26
-15
lines changed

.github/workflows/build.yml

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -12,7 +12,7 @@ jobs:
1212
strategy:
1313
matrix:
1414
coq_version:
15-
- '8.18'
15+
- '8.20'
1616
ocaml_version:
1717
- '4.14-flambda'
1818
fail-fast: true

opam

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -1,5 +1,5 @@
11
opam-version: "2.0"
2-
version: "1.0+8.18"
2+
version: "1.0+8.20"
33
maintainer: "[email protected]"
44
homepage: "https://github.com/uds-psl/coq-library-fol/"
55
dev-repo: "git+https://github.com/uds-psl/coq-library-fol/"
@@ -25,11 +25,11 @@ install: [
2525
[make "install"]
2626
]
2727
depends: [
28-
"coq" {>= "8.18" & < "8.19~"}
29-
"coq-library-undecidability" {= "1.1.1+8.18"}
28+
"coq" {>= "8.20" & < "9.0~"}
29+
"coq-library-undecidability" {= "1.1.2+8.20"}
3030
]
3131
synopsis: "A Coq Library for First-Order Logic"
3232
url {
33-
git: "https://github.com/uds-psl/coq-library-fol.git#v1.0+8.18"
33+
git: "https://github.com/uds-psl/coq-library-fol.git#v1.0+8.20"
3434
}
3535

theories/Completeness/HeytingMacNeille.v

Lines changed: 5 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -7,8 +7,11 @@ Require Export Coq.Program.Basics.
77
From FOL Require Import FullSyntax.
88
From FOL Require Import Heyting.Heyting.
99

10-
11-
Structure HeytingMorphism (HA1 HA2 : HeytingAlgebra) (F : HA1 -> HA2) : Type :=
10+
(* Morally this is in [Type]. But since all fields are in [Prop], putting this into
11+
[Prop] is fine due to subsingleton elimination, and because it is not computationally
12+
relevant anyways. *)
13+
(* Changing it back to [Type] makes Coq warn that this could just as well be in [Prop]. *)
14+
Structure HeytingMorphism (HA1 HA2 : HeytingAlgebra) (F : HA1 -> HA2) : Prop :=
1215
{
1316
F_inj : forall u v, F u = F v -> u = v ;
1417
F_mono : forall u v, u <= v -> F u <= F v ;

theories/Completeness/KripkeCompleteness.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -239,7 +239,7 @@ Section KripkeCompleteness.
239239

240240
Notation "A <<=C B" := (ctx_incl A B) (at level 20).
241241
Notation "A ⊢SC phi" := ((proj1_sig A) ⊢SE phi) (at level 20).
242-
Notation "A ;; psi ⊢sC phi" := ((proj1_sig A) ;; psi ⊢sE phi) (at level 20).
242+
Notation "A ;; psi ⊢sC phi" := ((proj1_sig A) ;; psi ⊢sE phi) (at level 70).
243243

244244
Ltac dest_con_ctx :=
245245
match goal with

theories/Incompleteness/bin_qdec.v

Lines changed: 2 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -10,6 +10,8 @@ Open Scope string_scope.
1010

1111
Require Import Setoid.
1212

13+
(* TODO FIXME the conflicting notation is not actually enabled (it is only Reserved), it should be refactored in coq-library-undecidability. *)
14+
#[warnings="notation-incompatible-prefix"]
1315
Require Import Undecidability.Shared.Libs.DLW.Vec.vec.
1416

1517
Require Import String.

theories/Incompleteness/ctq.v

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -7,7 +7,6 @@ From FOL.Proofmode Require Import Theories ProofMode.
77
From FOL.Incompleteness Require Import Axiomatisations utils fol_utils qdec bin_qdec sigma1 epf epf_mu.
88

99
Require Import Lia String List Cantor.
10-
Import ListNotations.
1110

1211
(** ** Church's Thesis for Q *)
1312
Section ctq.

theories/Incompleteness/epf_mu.v

Lines changed: 4 additions & 4 deletions
Original file line numberDiff line numberDiff line change
@@ -12,8 +12,8 @@ Require Import Undecidability.Synthetic.EnumerabilityFacts.
1212
From Coq.Logic Require Import ConstructiveEpsilon.
1313
From FOL.Incompleteness Require Import utils epf fol_utils qdec sigma1.
1414

15-
Import ListNotations.
16-
15+
(* Coq's ListNotation clashes with notations from MuRec *)
16+
Local Notation "[ e ]" := (cons e nil) (at level 70).
1717

1818
Derive Signature for Vector.t.
1919

@@ -46,7 +46,7 @@ End recalg_enum.
4646

4747

4848
Lemma erase_ra_rel alg x y :
49-
(exists k, evalfun k (erase alg) [x] = Some y) <->
49+
(exists k, evalfun k (erase alg) ([x]) = Some y) <->
5050
ra_rel alg (Vector.cons _ x _ (Vector.nil _)) y.
5151
Proof.
5252
split.
@@ -63,7 +63,7 @@ Qed.
6363
Definition mu_step : recalg 1 -> nat -\ nat.
6464
Proof.
6565
intros c x. unshelve eexists.
66-
{ intros k. exact (evalfun k (erase c) [x]). }
66+
{ intros k. exact (evalfun k (erase c) ([x])). }
6767
unfold core_valid.
6868
intros y1 y2 k1 k2 H1 H2. unfold evalfun in *.
6969
eapply ra_rel_fun.

theories/Incompleteness/fol_incompleteness.v

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -9,7 +9,6 @@ From FOL.Incompleteness Require Import Axiomatisations utils fol_utils qdec bin_
99
From FOL.Proofmode Require Import Theories ProofMode.
1010

1111
Require Import Lia String List.
12-
Import ListNotations.
1312

1413
(* * Incompleteness of first-order logic *)
1514

theories/Proofmode/Hoas.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -58,7 +58,7 @@ Notation "¬ A" := ((A → ⊥)%hoas) (at level 42) : hoas_scope.
5858
Notation "A '↔' B" := ((A → B)%hoas ∧ (B → A)%hoas) (at level 43) : hoas_scope.
5959

6060
Definition convert `{funcs_signature, preds_signature, operators} f := (@conv _ _ _ 0 f).
61-
Arguments convert {_ _ _} f%hoas.
61+
Arguments convert {_ _ _} f%_hoas.
6262

6363
Notation "<< f" := (ltac:(let y := eval cbn -[subst_form] in (convert f) in exact y)) (at level 200, only parsing).
6464

theories/_CoqProject

Lines changed: 8 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -5,6 +5,14 @@ COQDOCFLAGS = "--charset utf-8 -s --with-header ../website/resources/header.html
55

66
-Q . FOL
77

8+
9+
# Warning seems incorrect, see https://github.com/coq/coq/issues/19631
10+
# Disabled for now to reduce spam.
11+
-arg -w -arg -notation-incompatible-prefix
12+
# Disable warnings about vectors being hard to use. We know how to work with them.
13+
-arg -w -arg -warn-library-file-stdlib-vector
14+
15+
816
FullSyntax.v
917
FragmentSyntax.v
1018
Arithmetics.v

0 commit comments

Comments
 (0)