Skip to content
Merged
Show file tree
Hide file tree
Changes from all commits
Commits
File filter

Filter by extension

Filter by extension

Conversations
Failed to load comments.
Loading
Jump to
Jump to file
Failed to load files.
Loading
Diff view
Diff view
7 changes: 5 additions & 2 deletions backend/Inlining.v
Original file line number Diff line number Diff line change
Expand Up @@ -293,10 +293,13 @@ Inductive inline_decision (ros: reg + ident) : Type :=
| Cannot_inline
| Can_inline (id: ident) (f: function) (P: ros = inr reg id) (Q: fenv!id = Some f).

Arguments Cannot_inline {ros}.
Arguments Can_inline {ros}.

Program Definition can_inline (ros: reg + ident): inline_decision ros :=
match ros with
| inl r => Cannot_inline _
| inr id => match fenv!id with Some f => Can_inline _ id f _ _ | None => Cannot_inline _ end
| inl r => Cannot_inline
| inr id => match fenv!id with Some f => Can_inline id f _ _ | None => Cannot_inline end
end.

(** Inlining of a call to function [f]. An appropriate context is
Expand Down
2 changes: 2 additions & 0 deletions cfrontend/Ctypes.v
Original file line number Diff line number Diff line change
Expand Up @@ -20,6 +20,8 @@ Require Import Axioms Coqlib Maps Errors.
Require Import AST Linking.
Require Archi.

Set Asymmetric Patterns.

Local Open Scope error_monad_scope.

(** * Syntax of types *)
Expand Down
1 change: 1 addition & 0 deletions common/Behaviors.v
Original file line number Diff line number Diff line change
Expand Up @@ -25,6 +25,7 @@ Require Import Integers.
Require Import Smallstep.

Set Implicit Arguments.
Set Asymmetric Patterns.

(** * Behaviors for program executions *)

Expand Down
2 changes: 1 addition & 1 deletion common/Linking.v
Original file line number Diff line number Diff line change
Expand Up @@ -869,7 +869,7 @@ Infix ":::" := pass_cons (at level 60, right associativity) : linking_scope.
Fixpoint compose_passes (l l': Language) (passes: Passes l l') : Pass l l' :=
match passes in Passes l l' return Pass l l' with
| pass_nil l => pass_identity l
| pass_cons l1 l2 l3 pass1 passes => pass_compose pass1 (compose_passes passes)
| pass_cons pass1 passes => pass_compose pass1 (compose_passes passes)
end.

(** Some more lemmas about [nlist_forall2]. *)
Expand Down
2 changes: 0 additions & 2 deletions lib/Coqlib.v
Original file line number Diff line number Diff line change
Expand Up @@ -25,8 +25,6 @@ Require Export List.
Require Export Bool.
Require Export Lia.

Global Set Asymmetric Patterns.

(** * Useful tactics *)

Ltac inv H := inversion H; clear H; subst.
Expand Down
1 change: 1 addition & 0 deletions lib/Floats.v
Original file line number Diff line number Diff line change
Expand Up @@ -26,6 +26,7 @@ Import ListNotations.

Close Scope R_scope.
Open Scope Z_scope.
Set Asymmetric Patterns.

Definition float := binary64. (**r the type of IEE754 double-precision FP numbers *)
Definition float32 := binary32. (**r the type of IEE754 single-precision FP numbers *)
Expand Down
2 changes: 2 additions & 0 deletions lib/Iteration.v
Original file line number Diff line number Diff line change
Expand Up @@ -20,6 +20,8 @@ Require Import Axioms.
Require Import Coqlib.
Require Import Wfsimpl.

Set Asymmetric Patterns.

(** This modules defines several Coq encodings of a general "while" loop.
The loop is presented in functional style as the iteration
of a [step] function of type [A -> B + A]:
Expand Down
1 change: 1 addition & 0 deletions lib/UnionFind.v
Original file line number Diff line number Diff line change
Expand Up @@ -21,6 +21,7 @@ Require Import Coqlib.

Open Scope nat_scope.
Set Implicit Arguments.
Set Asymmetric Patterns.

(* To avoid useless definitions of inductors in extracted code. *)
Local Unset Elimination Schemes.
Expand Down