theory FOL_Extra imports Type_Instances_Impl "FOL-Fitting.FOL_Fitting" "HOL-Library.FSet" begin section ‹Additional support for FOL-Fitting› subsection ‹Iff› definition Iff where "Iff p q = And (Impl p q) (Impl q p)" lemma eval_Iff: "eval e f g (Iff p q) ⟷ (eval e f g p ⟷ eval e f g q)" by (auto simp: Iff_def) subsection ‹Replacement of subformulas›