Skip to content

Commit

Permalink
fix Intprop.Heyting
Browse files Browse the repository at this point in the history
  • Loading branch information
iehality committed Nov 24, 2024
1 parent 7133522 commit 4887553
Showing 1 changed file with 6 additions and 7 deletions.
13 changes: 6 additions & 7 deletions Foundation/IntProp/Heyting/Semantics.lean
Original file line number Diff line number Diff line change
Expand Up @@ -4,7 +4,7 @@ import Foundation.Logic.LindenbaumAlgebra

namespace LO.IntProp

variable {α : Type u} [DecidableEq α]
variable {α : Type u}

namespace Formula

Expand Down Expand Up @@ -94,9 +94,9 @@ lemma val_not (φ : Formula α) : ℍ ⊧ ∼φ ↔ (ℍ ⊧ₕ φ) = ⊥ := by

def mod (H : Hilbert α) : Set (HeytingSemantics α) := Semantics.models (HeytingSemantics α) H.axioms

variable {H : Hilbert α} [H.IncludeEFQ]
variable {H : Hilbert α}

instance : System.Intuitionistic H where
instance [H.IncludeEFQ] : System.Intuitionistic H where

lemma mod_models_iff {φ : Formula α} :
mod.{_,w} H ⊧ φ ↔ ∀ ℍ : HeytingSemantics.{_,w} α, ℍ ⊧* H.axioms → ℍ ⊧ φ := by
Expand Down Expand Up @@ -129,8 +129,7 @@ section

open System.LindenbaumAlgebra

variable (H)
variable [System.Consistent H]
variable [DecidableEq α] (H) [H.IncludeEFQ] [System.Consistent H]

def lindenbaum : HeytingSemantics α where
Algebra := System.LindenbaumAlgebra H
Expand Down Expand Up @@ -159,12 +158,12 @@ end

open Hilbert.Deduction

lemma complete {φ : Formula α} (h : mod.{_,u} H ⊧ φ) : H ⊢! φ := by
lemma complete [DecidableEq α] {φ : Formula α} [H.IncludeEFQ] (h : mod.{_,u} H ⊧ φ) : H ⊢! φ := by
wlog Con : System.Consistent H
· exact System.not_consistent_iff_inconsistent.mp Con φ
exact lindenbaum_complete_iff.mp <|
mod_models_iff.mp h (lindenbaum H) ⟨fun ψ hq ↦ lindenbaum_complete_iff.mpr <| eaxm! hq⟩

instance : Complete H (mod.{_,u} H) := ⟨complete⟩
instance [DecidableEq α] [H.IncludeEFQ] : Complete H (mod.{_,u} H) := ⟨complete⟩

end HeytingSemantics

0 comments on commit 4887553

Please sign in to comment.