def add(n, m):
return nat_rect(
lambda x: nat, # The motive: the property we're defining
# Base case: 0 + m = m
m, lambda k, rec: S(rec) # Inductive case: S(k) + m = S(k + m)
)(n)
Introduction
In the Induction post, we were able to build some simple inductive types and write some (very simple proofs). However, the actual process of defining the inductive types and writing the proofs was clunky and difficult. Most theorem provers introduce a Match construct to simplify the process of defining and working complex inductive types. We can use Match constructions both as syntactic sugar to help define inductive types and to more easily define functions that manipulate inductive types by pattern matching against their constructors.
This post follows several other posts about implementing a theorem prover in Python. The first post is here. In this post I’ll attempt to get some basic Match functionality working in conjunction with the previous posts theorem prover implementation in Python. Match constructions can get quite complicated. This post will not implement the full functionality that you would find in a production proof assistant, but will try to get the base functionality working.
Elimination Principles vs Match
In our previous implementation of induction, we automatically generated elimination principles for inductive types. For example, with natural numbers, we created nat_rect
, which has the following type:
∀P_nat:(Constant(nat)->Type(0)),((Var(P_nat) Constant(O))->((Constant(nat)->((Var(P_nat) Var(n))->(Var(P_nat) Constant(S))))->∀target_nat:Constant(nat),(Var(P_nat) Var(target_nat))))
This is very intimidating, and hard to parse, but it encodes the standard induction principle for natural numbers. To prove a property P for all natural numbers, you need to:
Prove \(P(0)\) (the base case).
Prove that for any \(n\), if \(P(n)\) holds, then \(P(S(n))\) also holds (the inductive step).
Here’s an intuitive look at what it would look like to define addition in terms of nat_rect
:
In our current language, this gets pretty ugly:
def define_plus(env: Environment) -> Environment:
# Type is: nat -> nat -> nat
= ProductType(
plus_type "n"),
Variable("nat"),
Constant(
ProductType("m"),
Variable("nat"),
Constant("nat")
Constant(
)
)
= Variable("n")
n = Variable("m")
m
# The function needs to do recursion on the first argument:
# plus := λ n. λ m. nat_rect (λ _. nat) m (λ k rec. S rec) n
= FunctionType(
plus_body "nat"),
n, Constant(
FunctionType("nat"),
m, Constant(
Application(
Application(
Application("nat_rect"),
Constant(# Motive: λ _. nat
"_"), Constant("nat"), Constant("nat"))
FunctionType(Variable(
),# Base: m
m
),# Step: λ k rec. S rec
FunctionType("k"), Constant("nat"),
Variable(
FunctionType("rec"), Constant("nat"),
Variable("S"), Variable("rec"))
Application(Constant(
)
)
)
)
)
return w_global_def(
env,"plus"),
Constant(
Hypothesis(env, plus_body, plus_type) )
Yikes1. A more complex inductive type would be extremely unwieldy. We can use the Match
construction to cut through some of the complexity using functional-programming-like pattern matching (this is pseudocode):
def add(n, m):
match n with
| O => m
| S(k) => S(add(k, m))
We can also use match to handle “enum-like” definitions. For example, say we want to prove theorems about the days of the week. We can define an inductive type as follows:
def define_weekday(env: Environment) -> Environment:
= InductiveType(
weekday_type ="weekday",
name=[],
params=[],
indices=Set(),
returnType=[
constructors"weekday"))
InductiveTypeConstructor(day, Constant(for day in ["sunday", "monday", "tuesday", "wednesday",
"thursday", "friday", "saturday"]
]
)
return define_inductive(env, weekday_type), weekday_type
You can imagine this (pseudocode) function implementation of is_weekend
:
def is_weekend(day):
return weekday_rect(
lambda d: bool, # Motive
False, # Monday case
False, # Tuesday case
False, # Wednesday case
False, # Thursday case
False, # Friday case
True, # Saturday case
True # Sunday case
)(day)
with Match
we can simplify this:
def is_weekend(day):
match day with
| Saturday => True
| Sunday => True
| _ => False
Ditto a function like “tomorrow”:
def tomorrow(day):
match day with
| Monday => Tuesday
| Tuesday => Wednesday
| Wednesday => Thursday
| Thursday => Friday
| Friday => Saturday
| Saturday => Sunday
| Sunday => Monday
So we have three use cases we might want out of Match
2:
- simplifying the definition of inductive types
- handling case-by-case proofs (for inductive types)
- simplifying the definition of functions on inductive types
We won’t handle 1 in this blog post (since we’ve got a perfectly good way of defining inductive types already) but we will try to handle 2 and 3.
Match Construct
Let’s start to implement our Match
construct. We’ll start with the extension to our grammar
class MatchBranch:
__match_args__ = ('constructor', 'bound_vars', 'body')
def __init__(self, constructor: Constant, bound_vars: List[Variable], body: Term):
self.constructor = constructor
self.bound_vars = bound_vars
self.body = body
def __repr__(self):
return f"MatchBranch({self.constructor}->{self.body})"
class Match:
__match_args__ = ('name', 'scrutinee', 'motive', 'branches')
def __init__(self, name:str, scrutinee: Term, motive: Term, branches: List[MatchBranch]):
self.name = name
self.scrutinee = scrutinee
self.motive = motive
self.branches = branches
def __repr__(self):
= '\n'.join(
branches_str f"| {b.constructor} {' '.join(str(v) for v in b.bound_vars)} => {b.body}"
for b in self.branches
)return f"match {self.scrutinee} return {self.motive} with\n{branches_str}\nend"
There’s two main classes. The first is for each branch of a Match
construct. This has three components:
- constructor: A Constant representing the constructor pattern being matched (like O or S for natural numbers)
- bound_vars: A list of Variables that will be bound to the constructor’s arguments
- body: A Term representing the result expression when this branch matches
The Match
construct follows. Here, the constructor takes four parameters:
- name: A string identifier for the match expression
- scrutinee: The term being matched against (the value we’re examining) motive: The return type of the match - expression (similar to the motive in elimination principles)
- branches: A list of
MatchBranch
objects representing the different cases
Proofs of Inductive Types with Match
Next, let’s try to handle case-by-case proofs for inductive types using the match
construct.
Match Rule
Given a valid match object, to view the theorem as “proven” we need to produce a valid hypothesis out of the elimination rules. Let’s take a look at how to do this:
def match_rule(env: Environment, match_: Match, inductive_type: InductiveType) -> Term:
# Find the elimination principle for this inductive type
= f"{inductive_type.name}_rect"
eliminator_name
# Apply eliminator applied to motive, branches, and scrutinee
= Constant(eliminator_name)
result = Application(result, match_.motive)
result for branch in match_.branches:
= Application(result, branch.body.term_)
result = Application(result, match_.scrutinee)
result
# Return type (motive applied to scrutinee)
= Application(match_.motive, match_.scrutinee)
return_type return Hypothesis(env, result, beta_reduce(return_type))
The match_rule
function builds the correct expression using elimination principles. We take the appropriate eliminator (nat_rect
in this case), then systematically apply it to the motive, each branch implementation, and the scrutinee value being matched against3.
Proof Example
Let’s now look at a proof example using match. This is a proof we previously handled in the induction post. Here, we will prove it using Match
:
def prove_plus_zero_via_match():
= w_empty()
env = define_nat(env)
env, nat_type = define_plus(env)
env = define_equality(env, Set())
env, _
= const(env, Constant("O"))
zero = const(env, Constant("plus"))
plus = const(env, Constant("eq"))
eq = const(env, Constant("nat"))
nat
= Variable("n")
n = w_local_assum(env, n, nat)
env = var(env, n)
hyp_n
# n + 0 = n
= app(env, app(env, plus, hyp_n), zero)
n_plus_zero
= app(env, eq, nat)
eq_nat = app(env, eq_nat, n_plus_zero)
eq_n = app(env, eq_n, hyp_n)
eq_type
# 0 + 0 = 0
= app(env, eq_nat, zero)
eq_0 = app(env, eq_0, zero)
eq_0_0
# Zero branch
= MatchBranch(
zero_branch =Constant("O"),
constructor=[],
bound_vars=eq_0_0
body
)
= Variable("s")
s = w_local_assum(env, s, nat)
env = const(env, Constant("S"))
succ = var(env, s)
s_term = app(env, succ, s_term)
succ_s = app(env, app(env, plus, succ_s), zero)
succ_s_plus_zero
= app(env, eq_nat, succ_s_plus_zero)
eq_succ_s = app(env, eq_succ_s, succ_s)
eq_succ_s_succ_s
= MatchBranch(
succ_branch =Constant("S"),
constructor=[s],
bound_vars=eq_succ_s_succ_s
body
)
= Variable('m')
m = w_local_assum(env, m, nat)
env = FunctionType(n, nat.term_, eq_type.term_)
motive
# Create match expression with name related to the type
= Match(
match_expr ="nat_match",
name=m,
scrutinee=motive,
motive=[zero_branch, succ_branch]
branches
)
= match_rule(env, n, match_expr, nat_type)
theorem return theorem
How does it work?
If we look at the output of this:
E[Gamma]⊢((((Constant(nat_rect) λn:Constant(nat).(((Constant(eq) Constant(nat)) ((Constant(plus) Var(n)) Constant(O))) Var(n))) (((Constant(eq) Constant(nat)) Constant(O)) Constant(O))) (((Constant(eq) Constant(nat)) ((Constant(plus) (Constant(S) Var(s))) Constant(O))) (Constant(S) Var(s)))) Var(m)):(((Constant(eq) Constant(nat)) ((Constant(plus) Var(m)) Constant(O))) Var(m))
It’s almost the same4 as the output of the example from the induction post.
Defining Functions Using Match
Weekday
I alluded to this earlier. Let’s say we have a weekday
enum defined as an inductive type:
def define_weekday(env: Environment) -> Environment:
= InductiveType(
weekday_type ="weekday",
name=[],
params=[],
indices=Set(),
returnType=[
constructors"weekday"))
InductiveTypeConstructor(day, Constant(for day in ["sunday", "monday", "tuesday", "wednesday",
"thursday", "friday", "saturday"]
]
)
return define_inductive(env, weekday_type), weekday_type
Now let’s define functions on top of weekday. This function adds yesterday
and tomorrow
to our global environment.
def define_weekday_operations(env: Environment, weekday:InductiveType) -> Environment:
= ["sunday", "monday", "tuesday", "wednesday", "thursday", "friday", "saturday"]
days
# Get the weekday type from environment
= Variable("w_weekday")
w_weekday = const(env, weekday)
ind_weekday
= Variable("d_tomorrow")
d_tomorrow = Variable("d_yesterday")
d_yesterday = w_local_assum(env, d_tomorrow, ind_weekday)
env = w_local_assum(env, d_yesterday, ind_weekday)
env
# Create motive - maps weekday to weekday
= ProductType(
motive
w_weekday,
weekday,
weekday
)
# Create branches for tomorrow
= []
branches_tomorrow for ind, day in enumerate(days):
= days[(ind + 1) % 7]
tomorrow_day
branches_tomorrow.append(
MatchBranch(=Constant(day),
constructor=[],
bound_vars=Constant(tomorrow_day)
body
)
)
# Create branches for yesterday
= []
branches_yesterday for ind, day in enumerate(days):
= days[(ind - 1) % 7]
yesterday_day
branches_yesterday.append(
MatchBranch(=Constant(day),
constructor=[],
bound_vars=Constant(yesterday_day)
body
)
)
# Create match expressions
= Match(
tomorrow ="tomorrow",
name=d_tomorrow,
scrutinee=motive,
motive=branches_tomorrow
branches
)
= Match(
yesterday ="yesterday",
name=d_yesterday,
scrutinee=motive,
motive=branches_yesterday
branches
)
# Add functions to environment
= w_global_def(
env
env,"tomorrow"),
Constant(
Hypothesis(env, tomorrow, tomorrow)
)= w_global_def(
env
env,"yesterday"),
Constant(
Hypothesis(env, yesterday, yesterday)
)
return env
Reduce Match
Now, say we have Application
of yesterday
to a day of the week. We need a way to reduce it:
def reduce_match(term: Term) -> Term:
if isinstance(term, Application) and isinstance(term.first, Match):
= term.first
match_expr = term.second
arg
for branch in match_expr.branches:
if isinstance(arg, Constant) and arg.name == branch.constructor.name:
return branch.body
return term
This is a pretty naive implementation, but it reduces an application of Match
by running through all the branches.
At this point, in theory, you could add reduce_match
(or similar rules) to our other conversion rules, which would let us prove theorems like \(\forall \text{day}: \text{weekday}, \text{yesterday}(\text{tomorrow}(\text{day})) = \text{day}\).
Conclusion and Next Steps
In this post, we’ve implemented a basic Match
construct that provides a more intuitive interface to the elimination principles. Though this implementation covers only the essentials it does demonstrate the core principles for handling Match
.
We’re pretty far along in terms of a proof assistant. There is more that can be done with Match
, but it’s out of scope of this post
In the game plan this post is the second half of step five. I’ve now implemented at least toy versions for most of the major aspects of a theorem prover, and proved a fair number of (trivial) theorems.
Probably I will have one more post on this Python implementation (the second half of step six, where I will attempt to tie our tactics back to the typing rules) and then a retrospective.
Footnotes
In general, this post is where the wheels started to fall off of this codebase. I’ll get into this in my proof assistant retrospective post.↩︎
At least. Presumably there are many tactics that can use matching, but that’s outside the scope of this post.↩︎
Note that I’ve fudged this a bit: we are getting away from the typing rules and just constructing the appropriate term. More on this in the next two posts.↩︎
I flipped the equal sign, so this proves \(n + 0 = n\) whereas the other proves \(n = n + 0\).↩︎