Skip to content

Commit

Permalink
fix(ModelTheory): make some defs into abbrevs (#6171)
Browse files Browse the repository at this point in the history
  • Loading branch information
ChrisHughes24 authored and semorrison committed Aug 3, 2023
1 parent 100debf commit 283325a
Showing 1 changed file with 3 additions and 3 deletions.
6 changes: 3 additions & 3 deletions Mathlib/ModelTheory/Syntax.lean
Original file line number Diff line number Diff line change
Expand Up @@ -1020,17 +1020,17 @@ def graph (f : L.Functions n) : L.Formula (Fin (n + 1)) :=
#align first_order.language.formula.graph FirstOrder.Language.Formula.graph

/-- The negation of a formula. -/
protected nonrec def not (φ : L.Formula α) : L.Formula α :=
protected nonrec abbrev not (φ : L.Formula α) : L.Formula α :=
φ.not
#align first_order.language.formula.not FirstOrder.Language.Formula.not

/-- The implication between formulas, as a formula. -/
protected def imp : L.Formula α → L.Formula α → L.Formula α :=
protected abbrev imp : L.Formula α → L.Formula α → L.Formula α :=
BoundedFormula.imp
#align first_order.language.formula.imp FirstOrder.Language.Formula.imp

/-- The biimplication between formulas, as a formula. -/
protected nonrec def iff (φ ψ : L.Formula α) : L.Formula α :=
protected nonrec abbrev iff (φ ψ : L.Formula α) : L.Formula α :=
φ.iff ψ
#align first_order.language.formula.iff FirstOrder.Language.Formula.iff

Expand Down

0 comments on commit 283325a

Please sign in to comment.