Axiomatization of Logic. Truth and Proof. Resolution

Axiomatization of Logic. Truth and Proof. Resolution

H250: Honors Colloquium – Introduction to Computation Axiomatization of Logic. Truth and Proof. Resolution Marius Minea [email protected] How many do we need? (best: few) Are they enough? Can we prove everything? Axiomatization helps answer these questions Motivation: Determining Truth In CS250, we started with truth table proofs. Propositional formula: can always do truth table (even if large) Predicate formula: can’t do truth tables (infinite possibilities) ⇒ must use other proof rules Motivation: Determining Truth In CS250, we started with truth table proofs. Propositional formula: can always do truth table (even if large) Predicate formula: can’t do truth tables (infinite possibilities) ⇒ must use other proof rules How many do we need? (best: few) Are they enough? Can we prove everything? Axiomatization helps answer these questions Symbols of propositional logic: propositions: p, q, r (usually lowercase letters) operators (logical connectives): negation ¬, implication → parentheses () Formulas of propositional logic: defined by structural induction (how to build complex formulas from simpler ones) A formula (compound proposition) is: any proposition (aka atomic formula or variable) (¬α) where α is a formula (α → β) if α and β are formulas Implication and negation suffice! First, Define Syntax We define a language by its symbols and the rules to correctly combine symbols (the syntax) Formulas of propositional logic: defined by structural induction (how to build complex formulas from simpler ones) A formula (compound proposition) is: any proposition (aka atomic formula or variable) (¬α) where α is a formula (α → β) if α and β are formulas Implication and negation suffice! First, Define Syntax We define a language by its symbols and the rules to correctly combine symbols (the syntax) Symbols of propositional logic: propositions: p, q, r (usually lowercase letters) operators (logical connectives): negation ¬, implication → parentheses () Implication and negation suffice! First, Define Syntax We define a language by its symbols and the rules to correctly combine symbols (the syntax) Symbols of propositional logic: propositions: p, q, r (usually lowercase letters) operators (logical connectives): negation ¬, implication → parentheses () Formulas of propositional logic: defined by structural induction (how to build complex formulas from simpler ones) A formula (compound proposition) is: any proposition (aka atomic formula or variable) (¬α) where α is a formula (α → β) if α and β are formulas First, Define Syntax We define a language by its symbols and the rules to correctly combine symbols (the syntax) Symbols of propositional logic: propositions: p, q, r (usually lowercase letters) operators (logical connectives): negation ¬, implication → parentheses () Formulas of propositional logic: defined by structural induction (how to build complex formulas from simpler ones) A formula (compound proposition) is: any proposition (aka atomic formula or variable) (¬α) where α is a formula (α → β) if α and β are formulas Implication and negation suffice! Definitions Should Be Minimal Fewest cases ⇒ simplicity (all future reasoning must cover all cases) Can define all other connectives in terms of ¬ and →: def α ∧ β = ¬(α → ¬β)(AND) α ∨ β def= ¬α → β (OR) α ↔ β def= (α → β) ∧ (β → α) (equivalence) Which inference rules to use? (again, few is good!) AA → B modus ponens B (from A and A → B we derive/infer B Modus Ponens is enough for propositional (and predicate) logic What is a Proof? (First Try) Let H be a set of formulas (hypotheses, premises). A deduction (or proof) from H is a sequence of formulas (statements) S1,..., Sn, such that every formula Sk is I a premise : Sk ∈ H I or follows from previous statements by a inference rule Modus Ponens is enough for propositional (and predicate) logic What is a Proof? (First Try) Let H be a set of formulas (hypotheses, premises). A deduction (or proof) from H is a sequence of formulas (statements) S1,..., Sn, such that every formula Sk is I a premise : Sk ∈ H I or follows from previous statements by a inference rule Which inference rules to use? (again, few is good!) AA → B modus ponens B (from A and A → B we derive/infer B What is a Proof? (First Try) Let H be a set of formulas (hypotheses, premises). A deduction (or proof) from H is a sequence of formulas (statements) S1,..., Sn, such that every formula Sk is I a premise : Sk ∈ H I or follows from previous statements by a inference rule Which inference rules to use? (again, few is good!) AA → B modus ponens B (from A and A → B we derive/infer B Modus Ponens is enough for propositional (and predicate) logic Proof Axioms What about statements that need no premises at all ? Need a base case for our reasoning: axioms Actual definition: A deduction (or proof) from H is a sequence of formulas S1,..., Sn, such that every formula Sk is I an axiom I a premise : Sk ∈ H I or follows from previous statements by a deduction rule Notation: H ` Sn (Sn can be derived from H) Axioms of propositional logic: A1: α → (β → α) A2: (α → (β → γ)) → ((α → β) → (α → γ)) A3: (¬β → ¬α) → (α → β) α, β, γ are any formulas ((2) A → ((A → A) → A)) → ((A → (A → A)) → (A → A)) A2, α = γ = A, β = A → A (3) (A → (A → A)) → (A → A) MP(1,2) (4) A → (A → A) A1, α = β = A (5) A → A MP(3,4) We can also show the Deduction Theorem If H ∪ {A} ` B then H ` A → B (assuming premise and proving conclusion shows implication) A Sample Deduction We prove A → A for any formula A (this is an axiom in some systems, but we can do without it) (1) A → ((A → A) → A)) A1, α = A, β = A → A (3) (A → (A → A)) → (A → A) MP(1,2) (4) A → (A → A) A1, α = β = A (5) A → A MP(3,4) We can also show the Deduction Theorem If H ∪ {A} ` B then H ` A → B (assuming premise and proving conclusion shows implication) A Sample Deduction We prove A → A for any formula A (this is an axiom in some systems, but we can do without it) (1) A → ((A → A) → A)) A1, α = A, β = A → A ((2) A → ((A → A) → A)) → ((A → (A → A)) → (A → A)) A2, α = γ = A, β = A → A (4) A → (A → A) A1, α = β = A (5) A → A MP(3,4) We can also show the Deduction Theorem If H ∪ {A} ` B then H ` A → B (assuming premise and proving conclusion shows implication) A Sample Deduction We prove A → A for any formula A (this is an axiom in some systems, but we can do without it) (1) A → ((A → A) → A)) A1, α = A, β = A → A ((2) A → ((A → A) → A)) → ((A → (A → A)) → (A → A)) A2, α = γ = A, β = A → A (3) (A → (A → A)) → (A → A) MP(1,2) (5) A → A MP(3,4) We can also show the Deduction Theorem If H ∪ {A} ` B then H ` A → B (assuming premise and proving conclusion shows implication) A Sample Deduction We prove A → A for any formula A (this is an axiom in some systems, but we can do without it) (1) A → ((A → A) → A)) A1, α = A, β = A → A ((2) A → ((A → A) → A)) → ((A → (A → A)) → (A → A)) A2, α = γ = A, β = A → A (3) (A → (A → A)) → (A → A) MP(1,2) (4) A → (A → A) A1, α = β = A We can also show the Deduction Theorem If H ∪ {A} ` B then H ` A → B (assuming premise and proving conclusion shows implication) A Sample Deduction We prove A → A for any formula A (this is an axiom in some systems, but we can do without it) (1) A → ((A → A) → A)) A1, α = A, β = A → A ((2) A → ((A → A) → A)) → ((A → (A → A)) → (A → A)) A2, α = γ = A, β = A → A (3) (A → (A → A)) → (A → A) MP(1,2) (4) A → (A → A) A1, α = β = A (5) A → A MP(3,4) A Sample Deduction We prove A → A for any formula A (this is an axiom in some systems, but we can do without it) (1) A → ((A → A) → A)) A1, α = A, β = A → A ((2) A → ((A → A) → A)) → ((A → (A → A)) → (A → A)) A2, α = γ = A, β = A → A (3) (A → (A → A)) → (A → A) MP(1,2) (4) A → (A → A) A1, α = β = A (5) A → A MP(3,4) We can also show the Deduction Theorem If H ∪ {A} ` B then H ` A → B (assuming premise and proving conclusion shows implication) Proofs are purely syntactic! We have done this without defining truth values, truth tables, etc. Finding a proof may be difficult (creativity, heuristics/tactics, etc.) Checking a proof is mechanical, based on simple string operations (check that formulas “pattern match” structure of axioms/rules) ( T if v(α) = F v(¬α) = F if v(α) = T ( F if v(α) = T and v(β) = F v(α → β) = T otherwise An interpretation is a truth assignment for the propositions of a formula. Semantics of Logic Truth assignment (valuation): gives a value (T, F) to any formula: v(p) defined for any atomic proposition p ( F if v(α) = T and v(β) = F v(α → β) = T otherwise An interpretation is a truth assignment for the propositions of a formula. Semantics of Logic Truth assignment (valuation): gives a value (T, F) to any formula: v(p) defined for any atomic proposition p ( T if v(α) = F v(¬α) = F if v(α) = T An interpretation is a truth assignment for the propositions of a formula. Semantics of Logic Truth assignment (valuation): gives a value (T, F) to any formula: v(p) defined for any atomic proposition p ( T if v(α) = F v(¬α) = F if v(α) = T ( F if v(α) = T and v(β) = F v(α → β) = T otherwise Semantics of Logic Truth assignment (valuation): gives a value (T, F) to any formula: v(p) defined for any atomic proposition p ( T if v(α) = F v(¬α) = F if v(α) = T ( F if v(α) = T and v(β) = F v(α → β) = T otherwise An interpretation is a truth assignment for the propositions of a formula.

View Full Text

Details

  • File Type
    pdf
  • Upload Time
    -
  • Content Languages
    English
  • Upload User
    Anonymous/Not logged-in
  • File Pages
    56 Page
  • File Size
    -

Download

Channel Download Status
Express Download Enable

Copyright

We respect the copyrights and intellectual property rights of all users. All uploaded documents are either original works of the uploader or authorized works of the rightful owners.

  • Not to be reproduced or distributed without explicit permission.
  • Not used for commercial purposes outside of approved use cases.
  • Not used to infringe on the rights of the original creators.
  • If you believe any content infringes your copyright, please contact us immediately.

Support

For help with questions, suggestions, or problems, please contact us