Skip to content

Commit 3edeccf

Browse files
authored
Merge pull request #232 from DmxLarchey/notation-overridden-2
Cleanup for overridden notations
2 parents f87cc31 + 12807df commit 3edeccf

29 files changed

+108
-107
lines changed

theories/FOL/FOL.v

Lines changed: 4 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -19,11 +19,13 @@ From Undecidability.FOL Require Deduction.FullND.
1919
| quant {b} : quantop -> form b -> form b.
2020
*)
2121

22-
22+
(*
2323
2424
Import FragmentSyntax.
2525
Export FragmentSyntax.
2626
27+
*)
28+
2729
(* ** Instantiation to signature with 1 constant, 2 unary functions, 1 prop constant, 1 binary relation *)
2830

2931
Inductive syms_func := s_f : bool -> syms_func | s_e.
@@ -66,7 +68,7 @@ Definition FOL_prv_class := @prv _ _ falsity_on class nil.
6668

6769
(* ** List of decision problems concerning validity, satisfiability and provability *)
6870

69-
Import BinSig Semantics.Tarski.FullCore.
71+
Import BinSig (* Semantics.Tarski.FullCore *) .
7072

7173
(* Validity of formulas with falsity in Tarski semantics *)
7274
Definition binFOL_valid := @FullCore.valid sig_empty sig_binary falsity_on.

theories/FOL/Reductions/H10UPC_to_FOL_friedman.v

Lines changed: 4 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -53,7 +53,11 @@ Section Fr_validity.
5353
- exact (H10UPC_SAT h10).
5454
- exact (dom_rel' (Vector.hd v) (Vector.hd (Vector.tl v))).
5555
Defined.
56+
57+
(* [DLW] This one is overridden by a new definition, may be change the notation slightly
58+
would be better? *)
5659
#[local] Notation "rho ⊨ phi" := (sat rho (Fr phi)) (at level 20).
60+
5761
(* Now we need rewrite helpers which transform our syntactic sugar into useful statements in the model *)
5862
Lemma IB_sFalse rho : rho ⊨ (∀ ∀ Pr $0 $1) <-> H10UPC_SAT h10.
5963
Proof.

theories/FOL/Reductions/H10p_to_FA.v

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -96,7 +96,7 @@ Section FA_ext_Model.
9696
Hypothesis ext_model : extensional I.
9797
Hypothesis FA_model : forall ax rho, In ax FA -> rho ⊨ ax.
9898

99-
Notation "'iO'" := (i_func (f:=Zero) (Vector.nil D)) (at level 2) : PA_Notation.
99+
(* Notation "'iO'" := (i_func (f:=Zero) (Vector.nil D)) (at level 2) : PA_Notation. *)
100100

101101
Fact eval_poly sigma p : eval (sigma >> iμ) (embed_poly p) = iμ (dp_eval_pfree sigma p).
102102
Proof using ext_model FA_model.
@@ -137,7 +137,7 @@ Section FA_Model.
137137

138138
Hypothesis FA_model : forall rho ax, In ax FAeq -> rho ⊨ ax.
139139

140-
Notation "'iO'" := (i_func (f:=Zero) (Vector.nil D)) (at level 2) : PA_Notation.
140+
(* Notation "'iO'" := (i_func (f:=Zero) (Vector.nil D)) (at level 2) : PA_Notation. *)
141141

142142
Lemma problem_to_model E sigma : H10p_sem E sigma -> (sigma >> iμ) ⊨ embed_problem E.
143143
Proof using FA_model.

theories/FOL/Reductions/PCPb_to_FSTD.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -26,7 +26,7 @@ Section FST.
2626

2727
Context { p : peirce }.
2828

29-
Close Scope sem.
29+
Close Scope FSTsem.
3030

3131
Lemma FST_eset x :
3232
FSTeq ⊢ ¬ (x ∈ ∅).

theories/FOL/Reductions/PCPb_to_HF.v

Lines changed: 0 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -15,8 +15,6 @@ Import ListAutomationNotations ListAutomationHints.
1515
Local Set Implicit Arguments.
1616
Local Unset Strict Implicit.
1717

18-
19-
2018
(* ** Reduction function *)
2119

2220
Local Definition BSRS := list(card bool).

theories/FOL/Reductions/PCPb_to_HFD.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -26,7 +26,7 @@ Section HF.
2626

2727
Context { p : peirce }.
2828

29-
Close Scope sem.
29+
Close Scope HFsem.
3030

3131
Lemma HF_eset x :
3232
HFeq ⊢ ¬ (x ∈ ∅).

theories/FOL/Reductions/PCPb_to_ZF.v

Lines changed: 0 additions & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -16,7 +16,6 @@ Import ListAutomationNotations ListAutomationHints.
1616
Local Set Implicit Arguments.
1717
Local Unset Strict Implicit.
1818

19-
2019
(* ** Reduction function *)
2120

2221
Local Definition BSRS := list(card bool).

theories/FOL/Reductions/PCPb_to_ZFD.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -26,7 +26,7 @@ Section ZF.
2626

2727
Context { p : peirce }.
2828

29-
Close Scope sem.
29+
Close Scope ZFsem.
3030

3131
Lemma ZF_eset x :
3232
ZFeq' ⊢ ¬ (x ∈ ∅).

theories/FOL/Reductions/PCPb_to_binZF.v

Lines changed: 2 additions & 2 deletions
Original file line numberDiff line numberDiff line change
@@ -152,7 +152,7 @@ From Undecidability.FOL Require Import Reductions.PCPb_to_ZFeq.
152152

153153
Section Model.
154154

155-
Open Scope sem.
155+
Open Scope ZFsem.
156156

157157
Context {V : Type} {I : interp V}.
158158

@@ -218,7 +218,7 @@ Section Model.
218218
erewrite sat_comp, sat_ext. reflexivity. now intros [].
219219
Qed.
220220

221-
Notation "x ≈ y" := (forall z, (x ∈ z -> y ∈ z) /\ (y ∈ z -> x ∈ z)) (at level 35) : sem.
221+
Notation "x ≈ y" := (forall z, (x ∈ z -> y ∈ z) /\ (y ∈ z -> x ∈ z)) (at level 35) : ZFsem.
222222

223223
Lemma eq_equiv x y :
224224
x ≈ y <-> x ≡ y.

theories/FOL/Reductions/PCPb_to_minZF.v

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -129,7 +129,7 @@ Qed.
129129

130130
Section Model.
131131

132-
Open Scope sem.
132+
Open Scope ZFsem.
133133

134134
Context {V : Type} {I : interp V}.
135135

0 commit comments

Comments
 (0)