File tree Expand file tree Collapse file tree 10 files changed +26
-15
lines changed
Expand file tree Collapse file tree 10 files changed +26
-15
lines changed Original file line number Diff line number Diff line change 1212 strategy :
1313 matrix :
1414 coq_version :
15- - ' 8.18 '
15+ - ' 8.20 '
1616 ocaml_version :
1717 - ' 4.14-flambda'
1818 fail-fast : true
Original file line number Diff line number Diff line change 11opam-version: "2.0"
2- version: "1.0+8.18 "
2+ version: "1.0+8.20 "
3344homepage: "https://github.com/uds-psl/coq-library-fol/"
55dev-repo: "git+https://github.com/uds-psl/coq-library-fol/"
@@ -25,11 +25,11 @@ install: [
2525 [make "install"]
2626]
2727depends: [
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]
3131synopsis: "A Coq Library for First-Order Logic"
3232url {
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
Original file line number Diff line number Diff line change @@ -7,8 +7,11 @@ Require Export Coq.Program.Basics.
77From FOL Require Import FullSyntax.
88From 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 ;
Original file line number Diff line number Diff 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
Original file line number Diff line number Diff line change @@ -10,6 +10,8 @@ Open Scope string_scope.
1010
1111Require 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"]
1315Require Import Undecidability.Shared.Libs.DLW.Vec.vec.
1416
1517Require Import String.
Original file line number Diff line number Diff line change @@ -7,7 +7,6 @@ From FOL.Proofmode Require Import Theories ProofMode.
77From FOL.Incompleteness Require Import Axiomatisations utils fol_utils qdec bin_qdec sigma1 epf epf_mu.
88
99Require Import Lia String List Cantor.
10- Import ListNotations.
1110
1211(** ** Church's Thesis for Q *)
1312Section ctq.
Original file line number Diff line number Diff line change @@ -12,8 +12,8 @@ Require Import Undecidability.Synthetic.EnumerabilityFacts.
1212From Coq.Logic Require Import ConstructiveEpsilon.
1313From 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
1818Derive Signature for Vector.t.
1919
@@ -46,7 +46,7 @@ End recalg_enum.
4646
4747
4848Lemma 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.
5151Proof .
5252 split.
6363Definition mu_step : recalg 1 -> nat -\ nat.
6464Proof .
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.
Original file line number Diff line number Diff line change @@ -9,7 +9,6 @@ From FOL.Incompleteness Require Import Axiomatisations utils fol_utils qdec bin_
99From FOL.Proofmode Require Import Theories ProofMode.
1010
1111Require Import Lia String List.
12- Import ListNotations.
1312
1413(* * Incompleteness of first-order logic *)
1514
Original file line number Diff line number Diff line change @@ -58,7 +58,7 @@ Notation "¬ A" := ((A → ⊥)%hoas) (at level 42) : hoas_scope.
5858Notation "A '↔' B" := ((A → B)%hoas ∧ (B → A)%hoas) (at level 43) : hoas_scope.
5959
6060Definition convert `{funcs_signature, preds_signature, operators} f := (@conv _ _ _ 0 f).
61- Arguments convert {_ _ _} f%hoas .
61+ Arguments convert {_ _ _} f%_hoas .
6262
6363Notation "<< f" := (ltac:(let y := eval cbn -[subst_form] in (convert f) in exact y)) (at level 200, only parsing).
6464
Original file line number Diff line number Diff 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+
816FullSyntax.v
917FragmentSyntax.v
1018Arithmetics.v
You can’t perform that action at this time.
0 commit comments