(* Author: Stefan Berghofer, TU Muenchen, 2003 Author: Asta Halkjær From, DTU Compute, 2019 Thanks to John Bruntse Larsen, Anders Schlichtkrull & Jørgen Villadsen See also the Natural Deduction Assistant: https://nadea.compute.dtu.dk/ *) section ‹First-Order Logic According to Fitting› theory FOL_Fitting imports "HOL-Library.Countable" begin section ‹Miscellaneous Utilities› text ‹Some facts about (in)finite sets› theorem set_inter_compl_diff [simp]: ‹- A ∩ B = B - A› by blast section ‹Terms and formulae› text ‹ \label{sec:terms} The datatypes of terms and formulae in {\em de Bruijn notation} are defined as follows: ›