58 exprt decreases_clause,
61 const auto loop_head_location = loop_head->source_location();
62 const auto loop_number = loop_end->loop_number;
65 const auto &decreases_clause_exprs = decreases_clause.
operands();
69 std::vector<symbol_exprt> old_decreases_vars, new_decreases_vars;
132 invariant.
swap(replace_history_result.expression_after_replacement);
133 const auto &history_var_map = replace_history_result.parameter_to_history;
137 replace_history_result.history_construction;
141 const auto entered_loop =
144 id2string(loop_head_location.get_function()),
145 std::string(
ENTERED_LOOP) +
"__" + std::to_string(loop_number),
150 pre_loop_head_instrs.
add(
152 pre_loop_head_instrs.
add(
157 const auto initial_invariant_val =
160 id2string(loop_head_location.get_function()),
166 pre_loop_head_instrs.
add(
173 initial_invariant_val, invariant};
179 initial_invariant_value_assignment, pre_loop_head_instrs, mode);
186 id2string(loop_head_location.get_function()),
192 pre_loop_head_instrs.
add(
194 pre_loop_head_instrs.
add(
211 loop_head, loop_end, snapshot_instructions);
216 if(assigns_clause.
is_nil())
232 log.
debug() <<
"No loop assigns clause provided. Inferred targets: {";
234 bool ran_once =
false;
235 for(
const auto &target : to_havoc)
242 target, snapshot_instructions);
247 std::inserter(to_havoc, to_havoc.end()));
251 log.
error() <<
"Failed to infer variables being modified by the loop at "
252 << loop_head_location
253 <<
".\nPlease specify an assigns clause.\nReason:"
262 for(
const auto &target : assigns_clause.
operands())
264 to_havoc.insert(target);
277 pre_loop_head_instrs.
add(
284 const auto step_case_target =
297 "Check loop invariant before entry");
300 converter.
goto_convert(assertion, pre_loop_head_instrs, mode);
307 goto_function.body.destructive_insert(
314 const auto in_loop_havoc_block =
317 id2string(loop_head_location.get_function()),
323 pre_loop_head_instrs.
add(
325 pre_loop_head_instrs.
add(
330 pre_loop_head_instrs.
add(
337 goto_function.body.destructive_insert(loop_head, pre_loop_head_instrs);
347 converter.
goto_convert(assumption, pre_loop_head_instrs, mode);
352 for(
const auto &clause : decreases_clause.
operands())
354 const auto old_decreases_var =
357 id2string(loop_head_location.get_function()),
363 pre_loop_head_instrs.
add(
365 old_decreases_vars.push_back(old_decreases_var);
367 const auto new_decreases_var =
370 id2string(loop_head_location.get_function()),
376 pre_loop_head_instrs.
add(
378 new_decreases_vars.push_back(new_decreases_var);
382 if(loop_end->is_goto() && !loop_end->condition().is_true())
384 log.
error() <<
"Loop contracts are unsupported on do/while loops: "
395 if(!decreases_clause.
is_nil())
397 for(
size_t i = 0; i < old_decreases_vars.size(); i++)
400 old_decreases_vars[i], decreases_clause_exprs[i]};
405 old_decreases_assignment, pre_loop_head_instrs, mode);
408 goto_function.body.destructive_insert(
416 goto_function.body.destructive_insert(
431 pre_loop_end_instrs.
add(
437 step_case_target, in_base_case, loop_head_location));
451 "Check that loop invariant is preserved");
454 converter.
goto_convert(assertion, pre_loop_end_instrs, mode);
459 if(!decreases_clause.
is_nil())
461 for(
size_t i = 0; i < new_decreases_vars.size(); i++)
464 new_decreases_vars[i], decreases_clause_exprs[i]};
469 new_decreases_assignment, pre_loop_end_instrs, mode);
476 new_decreases_vars, old_decreases_vars)};
478 monotonic_decreasing_assertion.add_source_location().
set_comment(
479 "Check decreases clause on loop iteration");
483 monotonic_decreasing_assertion, pre_loop_end_instrs, mode);
486 for(
size_t i = 0; i < old_decreases_vars.size(); i++)
488 pre_loop_end_instrs.
add(
490 pre_loop_end_instrs.
add(
501 loop_end->turn_into_assume();
502 loop_end->condition_nonconst() =
boolean_negate(loop_end->condition());
504 std::set<goto_programt::targett, goto_programt::target_less_than>
508 for(
const auto &t : loop)
513 auto exit_target = t->get_target();
515 loop.contains(exit_target) ||
516 seen_targets.find(exit_target) != seen_targets.end())
519 seen_targets.insert(exit_target);
525 "Check that loop instrumentation was not truncated");
528 annotated_location));
530 pre_loop_exit_instrs.
add(
532 pre_loop_exit_instrs.
add(
534 for(
const auto &v : history_var_map)
536 pre_loop_exit_instrs.
add(
541 goto_function.body, exit_target, pre_loop_exit_instrs);
552 it.is_function_call() && it.call_function().id() == ID_symbol &&
558 it.source_location());
568 exprt &instantiated_clause,
594 is_fresh_update(constraint);
602 const std::string &function_str =
id2string(function);
603 const auto &function_symbol = ns.
lookup(function);
606 if(ns.
lookup(
"contract::" + function_str, contract_sym))
614 type == function_symbol.type,
615 "front-end should have rejected re-declarations with a different type");
626 const auto &const_target =
630 PRECONDITION(const_target->call_function().id() == ID_symbol);
645 std::optional<exprt> call_ret_opt = {};
648 bool call_ret_is_fresh_var =
false;
653 if(target->call_lhs().is_not_nil())
659 auto &lhs_expr = const_target->call_lhs();
660 call_ret_opt = lhs_expr;
661 instantiation_values.push_back(lhs_expr);
668 type.c_ensures().begin(),
669 type.c_ensures().end(),
671 return has_symbol_expr(
672 to_lambda_expr(e).where(), CPROVER_PREFIX
"return_value", true);
677 call_ret_is_fresh_var =
true;
681 "ignored_return_value",
682 const_target->source_location(),
687 call_ret_opt = fresh_sym_expr;
688 instantiation_values.push_back(fresh_sym_expr);
693 instantiation_values.push_back(
700 const auto &arguments = const_target->call_arguments();
701 instantiation_values.insert(
702 instantiation_values.end(), arguments.begin(), arguments.end());
704 const auto &mode = function_symbol.
mode;
715 for(
const auto &clause : type.c_requires())
717 auto instantiated_clause =
721 _location.
set_comment(std::string(
"Check requires clause of ")
722 .append(target_function.
c_str())
724 .append(function.
c_str()));
741 for(
auto clause : type.c_ensures())
743 auto instantiated_clause =
748 instantiated_ensures_clauses.push_back(instantiated_clause);
754 for(
auto &target : type.c_assigns())
755 targets.push_back(
to_lambda_expr(target).application(instantiation_values));
771 havocker.get_instructions(havoc_instructions);
774 if(call_ret_opt.has_value())
776 auto &call_ret = call_ret_opt.value();
777 auto &loc = call_ret.source_location();
778 auto &type = call_ret.type();
781 if(call_ret_is_fresh_var)
782 havoc_instructions.
add(
794 for(
auto &clause : instantiated_ensures_clauses)
796 if(clause.is_false())
799 std::string(
"Attempt to assume false at ")
800 .append(clause.source_location().as_string())
801 .append(
".\nPlease update ensures clause to avoid vacuity."));
819 if(call_ret_is_fresh_var)
823 target->output(mstream);
824 mstream << messaget::eom;
851 const bool may_have_loops = std::any_of(
852 goto_function.body.instructions.begin(),
853 goto_function.body.instructions.end(),
855 return instruction.is_backwards_goto();
867 "Recursive functions found during inlining");
885 struct loop_graph_nodet :
public graph_nodet<empty_edget>
889 exprt assigns_clause, invariant, decreases_clause;
895 const exprt &assigns,
897 const exprt &decreases)
901 assigns_clause(assigns),
903 decreases_clause(decreases)
909 std::list<size_t> to_check_contracts_on_children;
913 std::pair<goto_programt::targett, natural_loops_mutablet::loopt>,
917 for(
const auto &loop_head_and_content : natural_loops.
loop_map)
919 const auto &loop_body = loop_head_and_content.second;
921 if(loop_body.size() <= 1)
924 auto loop_head = loop_head_and_content.first;
925 auto loop_end = loop_head;
928 for(
const auto &t : loop_body)
931 t->is_goto() && t->get_target() == loop_head &&
932 t->location_number > loop_end->location_number)
936 if(loop_end == loop_head)
938 log.
error() <<
"Could not find end of the loop starting at: "
951 for(
const auto &i : loop_body)
954 loop_head->location_number > i->location_number ||
955 i->location_number > loop_end->location_number)
959 mstream <<
"Computed loop at " << loop_head->source_location()
960 <<
"contains an instruction beyond [loop_head, loop_end]:"
963 mstream << messaget::eom;
969 if(!loop_head_ends.emplace(loop_head, std::make_pair(loop_end, loop_body))
974 for(
auto &loop_head_end : loop_head_ends)
976 auto loop_head = loop_head_end.first;
977 auto loop_end = loop_head_end.second.first;
987 loop_end->set_target(loop_head);
992 exprt decreases_clause =
1003 <<
" does not have an invariant in its contract.\n"
1004 <<
"Hence, a default invariant ('true') is being used.\n"
1005 <<
"This choice is sound, but verification may fail"
1006 <<
" if it is be too weak to prove the desired properties."
1013 if(decreases_clause.
is_nil())
1017 <<
" does not have a decreases clause in its contract.\n"
1018 <<
"Termination of this loop will not be verified."
1023 const auto idx = loop_nesting_graph.
add_node(
1024 loop_head_end.second.second,
1033 decreases_clause.
is_nil())
1036 to_check_contracts_on_children.push_back(idx);
1039 for(
size_t outer = 0; outer < loop_nesting_graph.
size(); ++outer)
1041 for(
size_t inner = 0; inner < loop_nesting_graph.
size(); ++inner)
1046 if(loop_nesting_graph[outer].content.contains(
1047 loop_nesting_graph[inner].head_target))
1049 if(!loop_nesting_graph[outer].content.contains(
1050 loop_nesting_graph[inner].end_target))
1053 <<
"Overlapping loops at:\n"
1054 << loop_nesting_graph[outer].head_target->source_location()
1056 << loop_nesting_graph[inner].head_target->source_location()
1057 <<
"\nLoops must be nested or sequential for contracts to be "
1061 loop_nesting_graph.
add_edge(inner, outer);
1067 while(!to_check_contracts_on_children.empty())
1069 const auto loop_idx = to_check_contracts_on_children.front();
1070 to_check_contracts_on_children.pop_front();
1072 const auto &loop_node = loop_nesting_graph[loop_idx];
1074 loop_node.assigns_clause.is_nil() && loop_node.invariant.is_nil() &&
1075 loop_node.decreases_clause.is_nil())
1079 <<
" does not have contracts, but an enclosing loop does.\n"
1080 <<
"Please provide contracts for this loop, or unwind it first."
1086 to_check_contracts_on_children.push_back(child_idx);
1091 for(
const auto &idx : loop_nesting_graph.
topsort())
1093 const auto &loop_node = loop_nesting_graph[idx];
1095 loop_node.assigns_clause.is_nil() && loop_node.invariant.is_nil() &&
1096 loop_node.decreases_clause.is_nil())
1115 std::to_string(loop_node.end_target->loop_number) +
1123 loop_node.head_target,
1124 loop_node.end_target,
1125 updated_loops.
loop_map[loop_node.head_target],
1126 loop_node.assigns_clause,
1127 loop_node.invariant,
1128 loop_node.decreases_clause,
1140 "Function '" +
id2string(function) +
"'must exist in the goto program");
1142 const auto &goto_function = function_obj->second;
1143 auto &function_body = function_obj->second.body;
1175 "Loops remain in function '" +
id2string(function) +
1176 "', assigns clause checking instrumentation cannot be applied.");
1179 auto instruction_it = function_body.instructions.begin();
1183 function_body, instruction_it, snapshot_static_locals);
1192 instantiation_values.push_back(
exprt{ID_nil, function_type.
return_type()});
1193 for(
const auto ¶m : function_type.
parameters())
1195 instantiation_values.push_back(
1196 ns.
lookup(param.get_identifier()).symbol_expr());
1202 to_lambda_expr(target).application(instantiation_values), payload);
1208 for(
const auto ¶m : function_type.
parameters())
1212 ns.
lookup(param.get_identifier()).symbol_expr(), payload);
1221 function_body, instruction_it, function_body.instructions.end());
1231 std::stringstream ss;
1239 "Function to replace must exist in the program.");
1246 sl.
set_file(
"instrumented for code contracts");
1249 symbolt mangled_sym = *original_sym;
1250 mangled_sym.
name = mangled;
1255 mangled_found.second,
1256 "There should be no existing function called " + ss.str() +
1257 " in the symbol table because that name is a mangled name");
1263 "There should be no function called " +
id2string(function) +
1264 " in the function map because that function should have had its"
1270 "There should be a function called " + ss.str() +
1271 " in the function map because we inserted a fresh goto-program"
1272 " with that mangled name");
1311 std::optional<code_returnt> return_stmt;
1315 code_type.return_type(),
1319 function_symbol.
mode,
1327 instantiation_values.push_back(
r);
1331 goto_functionst::function_mapt::iterator f_it =
1336 for(
const auto ¶meter : gf.parameter_identifiers)
1341 parameter_symbol.
type,
1345 parameter_symbol.
mode,
1350 p, parameter_symbol.
symbol_expr(), source_location));
1354 instantiation_values.push_back(p);
1363 for(
const auto &clause : code_type.c_requires())
1365 auto instantiated_clause =
1370 std::string(
"Attempt to assume false at ")
1371 .append(clause.source_location().as_string())
1372 .append(
".\nPlease update requires clause to avoid vacuity."));
1381 instantiated_clause,
1382 function_symbol.
mode,
1384 visitor.update_requires(c_requires);
1392 for(
auto clause : code_type.c_ensures())
1394 auto instantiated_clause =
1399 instantiated_ensures_clauses.push_back(instantiated_clause);
1406 for(
auto &clause : instantiated_ensures_clauses)
1416 function_symbol.
mode,
1417 [&visitor](
goto_programt &ensures) { visitor.update_ensures(ensures); },
1425 return_stmt.value().return_value(), source_location));
1439 const std::set<std::string> &functions)
const
1441 for(
const auto &function : functions)
1448 "Function '" + function +
"' was not found in the GOTO program.");
1455 if(to_replace.empty())
1466 if(ins->is_function_call())
1468 if(ins->call_function().id() != ID_symbol)
1473 auto found = std::find(
1474 to_replace.begin(), to_replace.end(),
id2string(called_function));
1475 if(found == to_replace.end())
1479 goto_function.first,
1480 ins->source_location(),
1481 goto_function.second.body,
1494 const std::set<std::string> &to_exclude_from_nondet_init)
1499 log.
status() <<
"Adding nondeterministic initialization "
1500 "of static/global variables."
1518 auto &goto_function = goto_function_entry.second;
1519 bool is_in_loop_havoc_block =
false;
1521 unsigned loop_number_of_loop_havoc = 0;
1523 goto_function.body.instructions.begin();
1524 it_instr != goto_function.body.instructions.end();
1537 const auto &assign_lhs =
1540 id2string(assign_lhs->get_identifier()),
1553 is_in_loop_havoc_block = it_instr->assign_rhs() ==
true_exprt();
1554 const auto &assign_lhs =
1557 id2string(assign_lhs->get_identifier()),
1563 if(is_in_loop_havoc_block && it_instr->is_assign())
1575 const std::set<std::string> &to_enforce,
1576 const std::set<std::string> &to_exclude_from_nondet_init)
1578 if(to_enforce.empty())
1581 log.
status() <<
"Enforcing contracts" << messaget ::eom;
1585 for(
const auto &function : to_enforce)
1588 log.
status() <<
"Adding nondeterministic initialization "
1589 "of static/global variables."
API to expression classes that are internal to the C frontend.
const code_with_contract_typet & to_code_with_contract_type(const typet &type)
Cast a typet to a code_with_contract_typet.
Classes providing CFG-based information about symbols to guide simplifications in function and loop a...
Thrown when an unexpected error occurs during the analysis (e.g., when the SAT solver returns an erro...
A non-fatal assertion, which checks a condition then permits execution to continue.
A goto_instruction_codet representing an assignment in the program.
An assumption, which must hold in subsequent code.
void apply_function_contract(const irep_idt &function, const source_locationt &location, goto_programt &function_body, goto_programt::targett &target)
Replaces function calls with assertions based on requires clauses, non-deterministic assignments for ...
void enforce_contract(const irep_idt &function)
Enforce contract of a single function.
void check_apply_loop_contracts(const irep_idt &function_name, goto_functionst::goto_functiont &goto_function, const local_may_aliast &local_may_alias, goto_programt::targett loop_head, goto_programt::targett loop_end, const loopt &loop, exprt assigns_clause, exprt invariant, exprt decreases_clause, const irep_idt &mode)
void apply_loop_contract(const irep_idt &function, goto_functionst::goto_functiont &goto_function)
Apply loop contracts, whenever available, to all loops in function.
void check_all_functions_found(const std::set< std::string > &functions) const
Throws an exception if some function functions is found in the program.
void check_frame_conditions_function(const irep_idt &function)
Instrument functions to check frame conditions.
void apply_loop_contracts(const std::set< std::string > &to_exclude_from_nondet_init={})
Applies loop contract transformations.
symbol_tablet & symbol_table
void enforce_contracts(const std::set< std::string > &to_enforce, const std::set< std::string > &to_exclude_from_nondet_init={})
Turn requires & ensures into assumptions and assertions for each of the named functions.
void replace_calls(const std::set< std::string > &to_replace)
Replace all calls to each function in the to_replace set with that function's contract.
std::unordered_set< irep_idt > summarized
std::unordered_set< goto_programt::const_targett, const_target_hash > loop_havoc_set
Loop havoc instructions instrumented during applying loop contracts.
loop_contract_configt loop_contract_config
std::list< std::string > loop_names
Name of loops we are going to unwind.
goto_functionst & goto_functions
std::unordered_map< goto_programt::const_targett, unsigned, const_target_hash > original_loop_number_map
Store the map from instrumented instructions for loop contracts to their original loop numbers.
void add_contract_check(const irep_idt &wrapper_function, const irep_idt &mangled_function, goto_programt &dest)
Instruments wrapper_function adding assumptions based on requires clauses and assertions based on ens...
goto_instruction_codet representation of a function call statement.
goto_instruction_codet representation of a "return from afunction" statement.
const parameterst & parameters() const
const typet & return_type() const
dstringt has one field, an unsigned integer no which is an index into a static table of strings.
const char * c_str() const
Base class for all expressions.
std::vector< exprt > operandst
bool is_false() const
Return whether the expression is a constant representing false.
source_locationt & add_source_location()
The Boolean constant false.
void goto_convert(const codet &code, goto_programt &dest, const irep_idt &mode)
function_mapt function_map
::goto_functiont goto_functiont
A goto function, consisting of function body (see body) and parameter identifiers (see parameter_iden...
parameter_identifierst parameter_identifiers
The identifiers of the parameters of this function.
This class represents an instruction in the GOTO intermediate representation.
A generic container class for the GOTO intermediate representation of one function.
instructionst instructions
The list of instructions in the goto program.
static instructiont make_set_return_value(exprt return_value, const source_locationt &l=source_locationt::nil())
static instructiont make_dead(const symbol_exprt &symbol, const source_locationt &l=source_locationt::nil())
void insert_before_swap(targett target)
Insertion that preserves jumps to "target".
void destructive_insert(const_targett target, goto_programt &p)
Inserts the given program p before target.
static instructiont make_end_function(const source_locationt &l=source_locationt::nil())
void destructive_append(goto_programt &p)
Appends the given program p to *this. p is destroyed.
static instructiont make_assignment(const code_assignt &_code, const source_locationt &l=source_locationt::nil())
Create an assignment instruction.
instructionst::iterator targett
static instructiont make_skip(const source_locationt &l=source_locationt::nil())
instructionst::const_iterator const_targett
static instructiont make_function_call(const code_function_callt &_code, const source_locationt &l=source_locationt::nil())
Create a function call instruction.
targett add(instructiont &&instruction)
Adds a given instruction at the end.
static instructiont make_goto(targett _target, const source_locationt &l=source_locationt::nil())
static instructiont make_decl(const symbol_exprt &symbol, const source_locationt &l=source_locationt::nil())
static instructiont make_assertion(const exprt &g, const source_locationt &l=source_locationt::nil())
This class represents a node in a directed graph.
A generic directed graph with a parametric node type.
std::vector< node_indext > get_predecessors(const node_indext &n) const
node_indext add_node(arguments &&... values)
void add_edge(node_indext a, node_indext b)
std::list< node_indext > topsort() const
Find a topological order of the nodes if graph is DAG, return empty list for non-DAG or empty graph.
Class to generate havocking instructions for target expressions of a function contract's assign claus...
A class that further overrides the "safe" havoc utilities, and adds support for havocing pointer_obje...
void append_full_havoc_code(const source_locationt location, goto_programt &dest)
Append goto instructions to havoc the full assigns set.
Decorator for a message_handlert used during function inlining that collect names of GOTO functions c...
void throw_on_recursive_calls(messaget &log, const int error_code)
Throws the given error code if recursive call warnings happend during inlining.
const std::set< irep_idt > & get_recursive_call_set() const
A class that generates instrumentation for assigns clause checking.
void track_spec_target(const exprt &expr, goto_programt &dest)
Track an assigns clause target and generate snaphsot instructions and well-definedness assertions in ...
void track_stack_allocated(const symbol_exprt &symbol_expr, goto_programt &dest)
Track a stack-allocated object and generate snaphsot instructions in dest.
void track_static_locals(goto_programt &dest)
Searches the goto instructions reachable from the start to the end of the instrumented function's ins...
void instrument_instructions(goto_programt &body, goto_programt::targett instruction_it, const goto_programt::targett &instruction_end, const std::function< bool(const goto_programt::targett &)> &pred={})
Instruments a sequence of instructions with inclusion checks.
void track_static_locals_between(goto_programt::const_targett it, const goto_programt::const_targett end, goto_programt &dest)
Searches the goto instructions reachable between the given it and end target instructions to identify...
void get_static_locals(std::insert_iterator< C > inserter) const
Inserts the detected static local symbols into a target container.
Thrown when we can't handle something in an input source file.
void add_memory_map_decl(goto_programt &program)
void update_requires(goto_programt &requires_)
void add_memory_map_dead(goto_programt &program)
void update_ensures(goto_programt &ensures)
virtual void create_declarations()
virtual void create_declarations()
exprt application(const operandst &arguments) const
void erase_locals(std::set< exprt > &exprs)
A loop, specified as a set of instructions.
source_locationt source_location
message_handlert & get_message_handler()
mstreamt & warning() const
void conditional_output(mstreamt &mstream, const std::function< void(mstreamt &)> &output_generator) const
Generate output to message_stream using output_generator if the configured verbosity is at least as h...
mstreamt & status() const
A namespacet is essentially one or two symbol tables bound together, to allow for symbol lookups in t...
bool lookup(const irep_idt &name, const symbolt *&symbol) const override
See documentation for namespace_baset::lookup().
A side_effect_exprt that returns a non-deterministically chosen value.
void set_comment(const irep_idt &comment)
void set_property_class(const irep_idt &property_class)
const irep_idt & get_function() const
const irep_idt & get_line() const
const irep_idt & get_property_class() const
std::string as_string() const
void set_file(const irep_idt &file)
void set_line(const irep_idt &line)
void set_function(const irep_idt &function)
Expression to hold a symbol (variable)
const irep_idt & get_identifier() const
const symbolt * lookup(const irep_idt &name) const
Find a symbol in the symbol table for read-only access.
const symbolt & lookup_ref(const irep_idt &name) const
Find a symbol in the symbol table for read-only access.
virtual std::pair< symbolt &, bool > insert(symbolt symbol) override
Author: Diffblue Ltd.
irep_idt base_name
Base (non-scoped) name.
source_locationt location
Source code location of definition of symbol.
class symbol_exprt symbol_expr() const
Produces a symbol_exprt for a symbol.
typet type
Type of symbol.
irep_idt name
The unique identifier.
irep_idt mode
Language mode.
The Boolean constant true.
void parse_unwindset(const std::list< std::string > &unwindset, message_handlert &message_handler)
static void generate_contract_constraints(symbol_tablet &symbol_table, goto_convertt &converter, exprt &instantiated_clause, const irep_idt &mode, const std::function< void(goto_programt &)> &is_fresh_update, goto_programt &program, const source_locationt &location)
This function generates instructions for all contract constraint, i.e., assumptions and assertions ba...
static const code_with_contract_typet & get_contract(const irep_idt &function, const namespacet &ns)
static void throw_on_unsupported(const goto_programt &program)
Throws an exception if a contract uses unsupported constructs like:
Verify and use annotated invariants and pre/post-conditions.
static const std::map< dfcc_funt, int > to_unwind
set of functions that need to be unwound to assigns clause size with corresponding loop identifiers.
auto expr_try_dynamic_cast(TExpr &base) -> typename detail::expr_try_dynamic_cast_return_typet< T, TExpr >::type
Try to cast a reference to a generic exprt to a specific derived class.
bool has_subexpr(const exprt &expr, const std::function< bool(const exprt &)> &pred)
returns true if the expression has a subexpression that satisfies pred
exprt boolean_negate(const exprt &src)
negate a Boolean expression, possibly removing a not_exprt, and swapping false and true
Deprecated expression utility functions.
symbolt & get_fresh_aux_symbol(const typet &type, const std::string &name_prefix, const std::string &basename_prefix, const source_locationt &source_location, const irep_idt &symbol_mode, const namespacet &ns, symbol_table_baset &symbol_table)
Installs a fresh-named symbol with respect to the given namespace ns with the requested name pattern ...
Fresh auxiliary symbol creation.
void goto_function_inline(goto_modelt &goto_model, const irep_idt function, message_handlert &message_handler, bool adjust_function, bool caching)
Transitively inline all function calls made from a particular function.
Function Inlining This gives a number of different interfaces to the function inlining functionality ...
#define Forall_goto_program_instructions(it, program)
A Template Class for Graphs.
Havoc function assigns clauses.
Utilities for building havoc code for expressions.
std::set< exprt > assignst
std::optional< code_with_contract_typet > get_contract(const irep_idt &function_identifier, const namespacet &ns)
void add_pragma_disable_assigns_check(source_locationt &location)
Adds a pragma on a source_locationt to disable inclusion checking.
Specify write set in function contracts.
const std::string & id2string(const irep_idt &d)
Field-insensitive, location-sensitive may-alias analysis.
natural_loops_mutablet::natural_loopt loopt
API to expression classes for 'mathematical' expressions.
const lambda_exprt & to_lambda_expr(const exprt &expr)
Cast an exprt to a lambda_exprt.
Predicates to specify memory footprint in function contracts.
static void nondet_static(const namespacet &ns, goto_modelt &goto_model, const irep_idt &fct_name)
Nondeterministically initializes global scope variables in a goto-function.
Nondeterministically initializes global scope variables, except for constants (such as string literal...
void remove_skip(goto_programt &goto_program, goto_programt::targett begin, goto_programt::targett end)
remove unnecessary skip statements
#define UNREACHABLE
This should be used to mark dead code.
#define DATA_INVARIANT(CONDITION, REASON)
This condition should be used to document that assumptions that are made on goto_functions,...
#define PRECONDITION(CONDITION)
#define INVARIANT(CONDITION, REASON)
This macro uses the wrapper function 'invariant_violated_string'.
exprt conjunction(const exprt::operandst &op)
1) generates a conjunction for two or more operands 2) for one operand, returns the operand 3) return...
const symbol_exprt & to_symbol_expr(const exprt &expr)
Cast an exprt to a symbol_exprt.
const code_typet & to_code_type(const typet &type)
Cast a typet to a code_typet.
A total order over targett and const_targett.
bool unwind_transformed_loops
void generate_history_variables_initialization(symbol_table_baset &symbol_table, exprt &clause, const irep_idt &mode, goto_programt &program)
This function generates all the instructions required to initialize history variables.
bool is_assignment_to_instrumented_variable(const goto_programt::const_targett &target, std::string var_name)
Return true if target is an assignment to an instrumented variable with name var_name.
void insert_before_and_update_jumps(goto_programt &destination, goto_programt::targett &target, const goto_programt::instructiont &i)
Insert a goto instruction before a target instruction iterator and update targets of all jumps that p...
void add_quantified_variable(symbol_table_baset &symbol_table, exprt &expression, const irep_idt &mode)
This function recursively searches expression to find nested or non-nested quantified expressions.
void infer_loop_assigns(const local_may_aliast &local_may_alias, const loopt &loop, assignst &assigns)
Infer loop assigns using alias analysis result local_may_alias.
bool is_loop_free(const goto_programt &goto_program, namespacet &ns, messaget &log)
Returns true iff the given program is loop-free, i.e.
exprt get_loop_assigns(const goto_programt::const_targett &loop_end)
replace_history_parametert replace_history_loop_entry(symbol_table_baset &symbol_table, const exprt &expr, const source_locationt &location, const irep_idt &mode)
This function recursively identifies the "loop_entry" expressions within expr and replaces them with ...
bool is_transformed_loop_head(const goto_programt::const_targett &target)
Return true if target is the head of some transformed loop.
void insert_before_swap_and_advance(goto_programt &destination, goto_programt::targett &target, goto_programt &payload)
Insert a goto program before a target instruction iterator and advance the iterator.
void widen_assigns(assignst &assigns, const namespacet &ns)
Widen expressions in assigns with the following strategy.
exprt get_loop_invariants(const goto_programt::const_targett &loop_end, const bool check_side_effect)
bool is_transformed_loop_end(const goto_programt::const_targett &target)
Return true if target is the end of some transformed loop.
void simplify_gotos(goto_programt &goto_program, namespacet &ns)
Turns goto instructions IF cond GOTO label where the condition statically simplifies to false into SK...
exprt get_loop_decreases(const goto_programt::const_targett &loop_end, const bool check_side_effect)
Extract loop invariants from annotated loop end.
unsigned get_suffix_unsigned(const std::string &str, const std::string &prefix)
Convert the suffix digits right after prefix of str into unsigned.
exprt generate_lexicographic_less_than_check(const std::vector< symbol_exprt > &lhs, const std::vector< symbol_exprt > &rhs)
Generate a lexicographic less-than comparison over ordered tuples.
#define IN_LOOP_HAVOC_BLOCK