Documentation

Mathlib.ModelTheory.Bundled

Bundled First-Order Structures #

This file bundles types together with their first-order structure.

Main Definitions #

TODO #

@[simp]

A type bundled with the structure induced by an equivalence.

Equations
Instances For

    An equivalence of types as a first-order equivalence to the bundled structure on the codomain.

    Equations
    Instances For

      The equivalence relation on bundled L.Structures indicating that they are isomorphic.

      Equations

      The type of nonempty models of a first-order theory.

      Instances For

        The object in the category of R-algebras associated to a type equipped with the appropriate typeclasses.

        Equations
        Instances For
          @[simp]
          theorem FirstOrder.Language.Theory.ModelType.defaultExpansion_Carrier {L : FirstOrder.Language} {T : FirstOrder.Language.Theory L} {L' : FirstOrder.Language} {φ : L →ᴸ L'} (h : FirstOrder.Language.LHom.Injective φ) [(n : ) → (f : L'.Functions n) → Decidable (f Set.range fun (f : L.Functions n) => φ.onFunction f)] [(n : ) → (r : L'.Relations n) → Decidable (r Set.range fun (r : L.Relations n) => φ.onRelation r)] (M : FirstOrder.Language.Theory.ModelType T) [Inhabited M] :
          @[simp]
          theorem FirstOrder.Language.Theory.ModelType.defaultExpansion_struc {L : FirstOrder.Language} {T : FirstOrder.Language.Theory L} {L' : FirstOrder.Language} {φ : L →ᴸ L'} (h : FirstOrder.Language.LHom.Injective φ) [(n : ) → (f : L'.Functions n) → Decidable (f Set.range fun (f : L.Functions n) => φ.onFunction f)] [(n : ) → (r : L'.Relations n) → Decidable (r Set.range fun (r : L.Relations n) => φ.onRelation r)] (M : FirstOrder.Language.Theory.ModelType T) [Inhabited M] :
          noncomputable def FirstOrder.Language.Theory.ModelType.defaultExpansion {L : FirstOrder.Language} {T : FirstOrder.Language.Theory L} {L' : FirstOrder.Language} {φ : L →ᴸ L'} (h : FirstOrder.Language.LHom.Injective φ) [(n : ) → (f : L'.Functions n) → Decidable (f Set.range fun (f : L.Functions n) => φ.onFunction f)] [(n : ) → (r : L'.Relations n) → Decidable (r Set.range fun (r : L.Relations n) => φ.onRelation r)] (M : FirstOrder.Language.Theory.ModelType T) [Inhabited M] :

          When φ is injective, defaultExpansion expands a model of T to a model of φ.onTheory T arbitrarily.

          Equations
          Instances For