Skip to content

Commit 88ce072

Browse files
2 parents a1bda00 + 85bb89c commit 88ce072

File tree

2 files changed

+7
-1
lines changed

2 files changed

+7
-1
lines changed

Mathlib/ModelTheory/Semantics.lean

Lines changed: 6 additions & 0 deletions
Original file line numberDiff line numberDiff line change
@@ -568,6 +568,12 @@ theorem realize_graph {f : L.Functions n} {x : Fin n → M} {y : M} :
568568
simp only [Formula.graph, Term.realize, realize_equal, Fin.cons_zero, Fin.cons_succ]
569569
rw [eq_comm]
570570

571+
theorem boundedFormula_realize_eq_realize (φ : L.Formula α) (x : α → M) (y : Fin 0 → M) :
572+
BoundedFormula.Realize φ x y ↔ φ.Realize x := by
573+
rw [Formula.Realize, iff_iff_eq]
574+
congr
575+
ext i; exact Fin.elim0 i
576+
571577
end Formula
572578

573579
@[simp]

lake-manifest.json

Lines changed: 1 addition & 1 deletion
Original file line numberDiff line numberDiff line change
@@ -65,7 +65,7 @@
6565
"type": "git",
6666
"subDir": null,
6767
"scope": "leanprover-community",
68-
"rev": "d3a45c11f470e814978c1e939a60509e3420c0b5",
68+
"rev": "8510de1dc4a6a573fc9e6c0980315fc1088da4db",
6969
"name": "batteries",
7070
"manifestFile": "lake-manifest.json",
7171
"inputRev": "union-darray",

0 commit comments

Comments
 (0)