Skip to content

Commit

Permalink
feat(model_theory/satisfiability): Definition of categorical theories (
Browse files Browse the repository at this point in the history
…#14038)

Defines that a first-order theory is `κ`-categorical when all models of cardinality `κ` are isomorphic.
Shows that all theories in the empty language are `κ`-categorical for all cardinals `κ`.
  • Loading branch information
awainverse committed May 9, 2022
1 parent 5d8b432 commit 31af0e8
Showing 1 changed file with 16 additions and 0 deletions.
16 changes: 16 additions & 0 deletions src/model_theory/satisfiability.lean
Expand Up @@ -20,6 +20,7 @@ every finite subset of `T` is satisfiable.
models each sentence or its negation.
* `first_order.language.Theory.semantically_equivalent`: `T.semantically_equivalent φ ψ` indicates
that `φ` and `ψ` are equivalent formulas or sentences in models of `T`.
* `cardinal.categorical`: A theory is `κ`-categorical if all models of size `κ` are isomorphic.
## Main Results
* The Compactness Theorem, `first_order.language.Theory.is_satisfiable_iff_is_finitely_satisfiable`,
Expand Down Expand Up @@ -395,3 +396,18 @@ lemma induction_on_exists_not {P : Π {m}, L.bounded_formula α m → Prop} (φ
end bounded_formula
end language
end first_order

namespace cardinal
open first_order first_order.language

variables {L : language.{u v}} (κ : cardinal.{w}) (T : L.Theory)

/-- A theory is `κ`-categorical if all models of size `κ` are isomorphic. -/
def categorical : Prop :=
∀ (M N : T.Model), # M = κ → # N = κ → nonempty (M ≃[L] N)

theorem empty_Theory_categorical (T : language.empty.Theory) :
κ.categorical T :=
λ M N hM hN, by rw [empty.nonempty_equiv_iff, hM, hN]

end cardinal

0 comments on commit 31af0e8

Please sign in to comment.