Theory mere_addition_lewis
section ‹The Mere Addition Paradox: Lewis' rule›
text ‹We run the same queries as before, but using Lewis' rule. The outcome is pretty
much the same. Thus, the choice between the opt rule and Lewis' rule does not make a difference.›
theory mere_addition_lewis
imports DDLcube
begin
consts a::σ aplus::σ b::σ
axiomatization where
PPP0: "⌊(❙¬∘<❙¬a|a❙∨b>❙∧∘<❙¬b|a❙∨b>)⌋" and
PPP1: "⌊❙¬∘<❙¬aplus|a❙∨aplus>⌋" and
PPP2: "⌊(❙¬∘<❙¬b|aplus❙∨b> ❙∧ ∘<❙¬aplus|aplus❙∨b>)⌋"
text ‹Sledgehammer finds PPP0-PPP2 inconsistent given transitivity of the betterness relation in the models:›
theorem T0:
assumes transitivity
shows False
by (metis PPP0 PPP1 PPP2 assms)
text ‹Nitpick shows consistency in the absence of transitivity:›
lemma T1:
True
nitpick [satisfy,expect=genuine,card i=3,show_all]
oops
text ‹Sledgehammer confirms inconsistency in the presence of the interval order condition:›
theorem T2:
assumes reflexivity Ferrers
shows False
by (metis PPP0 PPP1 PPP2 assms(1) assms(2))
text ‹Nitpick shows consistency if transitivity is weakened into acyclicity
or quasi-transitivity:›
theorem T3:
assumes loopfree
shows True
nitpick [satisfy,expect=genuine,card=3]
oops
theorem T4:
assumes Quasitransit
shows True
nitpick [satisfy,expect=genuine,card=4]
oops
end