2f88d6710c
Signed-off-by: Leonardo de Moura <leonardo@microsoft.com>
118 lines
3.7 KiB
C++
118 lines
3.7 KiB
C++
/*
|
|
Copyright (c) 2013 Microsoft Corporation. All rights reserved.
|
|
Released under Apache 2.0 license as described in the file LICENSE.
|
|
|
|
Author: Leonardo de Moura
|
|
*/
|
|
#pragma once
|
|
#include <tuple>
|
|
#include "util/buffer.h"
|
|
#include "util/interrupt.h"
|
|
#include "kernel/expr.h"
|
|
#include "kernel/expr_maps.h"
|
|
|
|
namespace lean {
|
|
/**
|
|
\brief Default replace_fn postprocessor functional object. It is a
|
|
do-nothing object.
|
|
*/
|
|
class default_replace_postprocessor {
|
|
public:
|
|
void operator()(expr const &, expr const &) {}
|
|
};
|
|
|
|
/**
|
|
\brief Functional for applying <tt>F</tt> to the subexpressions of a given expression.
|
|
|
|
The signature of \c F is
|
|
expr const &, unsigned -> expr
|
|
|
|
F is invoked for each subexpression \c s of the input expression e.
|
|
In a call <tt>F(s, n)</tt>, n is the scope level, i.e., the number of
|
|
bindings operators that enclosing \c s.
|
|
|
|
P is a "post-processing" functional object that is applied to each
|
|
pair (old, new)
|
|
*/
|
|
template<typename F, typename P = default_replace_postprocessor>
|
|
class replace_fn {
|
|
static_assert(std::is_same<typename std::result_of<F(expr const &, unsigned)>::type, expr>::value,
|
|
"replace_fn: return type of F is not expr");
|
|
// the return type of P()(e1, e2) should be void
|
|
static_assert(std::is_same<typename std::result_of<decltype(std::declval<P>())(expr const &, expr const &)>::type,
|
|
void>::value,
|
|
"The return type of P()(e1, e2) is not void");
|
|
|
|
expr_cell_offset_map<expr> m_cache;
|
|
F m_f;
|
|
P m_post;
|
|
|
|
optional<expr> apply(optional<expr> const & e, unsigned offset) {
|
|
if (e)
|
|
return some_expr(apply(*e, offset));
|
|
else
|
|
return none_expr();
|
|
}
|
|
|
|
expr apply(expr const & e, unsigned offset) {
|
|
check_system("expression replacer");
|
|
bool sh = false;
|
|
if (is_shared(e)) {
|
|
expr_cell_offset p(e.raw(), offset);
|
|
auto it = m_cache.find(p);
|
|
if (it != m_cache.end())
|
|
return it->second;
|
|
sh = true;
|
|
}
|
|
|
|
expr r = m_f(e, offset);
|
|
if (is_eqp(e, r)) {
|
|
switch (e.kind()) {
|
|
case expr_kind::Constant:
|
|
if (const_type(e))
|
|
r = update_const(e, apply(const_type(e), offset));
|
|
break;
|
|
case expr_kind::Type: case expr_kind::Value:
|
|
case expr_kind::Var: case expr_kind::MetaVar:
|
|
break;
|
|
case expr_kind::App:
|
|
r = update_app(e, [=](expr const & c) { return apply(c, offset); });
|
|
break;
|
|
case expr_kind::Eq:
|
|
r = update_eq(e, [=](expr const & l, expr const & r) { return std::make_pair(apply(l, offset), apply(r, offset)); });
|
|
break;
|
|
case expr_kind::Lambda:
|
|
case expr_kind::Pi:
|
|
r = update_abst(e, [=](expr const & t, expr const & b) { return std::make_pair(apply(t, offset), apply(b, offset+1)); });
|
|
break;
|
|
case expr_kind::Let:
|
|
r = update_let(e, [=](optional<expr> const & t, expr const & v, expr const & b) {
|
|
return std::make_tuple(apply(t, offset), apply(v, offset), apply(b, offset+1));
|
|
});
|
|
break;
|
|
}
|
|
}
|
|
|
|
if (sh)
|
|
m_cache.insert(std::make_pair(expr_cell_offset(e.raw(), offset), r));
|
|
|
|
m_post(e, r);
|
|
|
|
return r;
|
|
}
|
|
|
|
public:
|
|
replace_fn(F const & f, P const & p = P()):
|
|
m_f(f),
|
|
m_post(p) {
|
|
}
|
|
|
|
expr operator()(expr const & e) {
|
|
return apply(e, 0);
|
|
}
|
|
|
|
void clear() {
|
|
m_cache.clear();
|
|
}
|
|
};
|
|
}
|