aboutsummaryrefslogtreecommitdiff
path: root/theories/Program
diff options
context:
space:
mode:
authorEmilio Jesus Gallego Arias2018-09-11 11:04:11 +0200
committerEmilio Jesus Gallego Arias2018-09-11 11:04:11 +0200
commitf3475cd1a68f632b1e6522975354c7dcc1acd6bb (patch)
tree6ea45570f34dd67e422b946b0781013692a24709 /theories/Program
parent3dceb51345662b4ceda4214be5ae2d17459f48f3 (diff)
parent0aa164f8fc8adf2cd57681ef64ff598c71b5d9f8 (diff)
Merge PR #7135: Introducing an explicit `Declare Scope` command
Diffstat (limited to 'theories/Program')
-rw-r--r--theories/Program/Basics.v2
-rw-r--r--theories/Program/Utils.v5
2 files changed, 5 insertions, 2 deletions
diff --git a/theories/Program/Basics.v b/theories/Program/Basics.v
index f55093ed48..c2316689fc 100644
--- a/theories/Program/Basics.v
+++ b/theories/Program/Basics.v
@@ -28,6 +28,8 @@ Definition compose {A B C} (g : B -> C) (f : A -> B) :=
Hint Unfold compose.
+Declare Scope program_scope.
+
Notation " g ∘ f " := (compose g f)
(at level 40, left associativity) : program_scope.
diff --git a/theories/Program/Utils.v b/theories/Program/Utils.v
index 78c36dc7d1..c51cacac68 100644
--- a/theories/Program/Utils.v
+++ b/theories/Program/Utils.v
@@ -20,12 +20,13 @@ Notation "{ ( x , y ) : A | P }" :=
(sig (fun anonymous : A => let (x,y) := anonymous in P))
(x ident, y ident, at level 10) : type_scope.
+Declare Scope program_scope.
+Delimit Scope program_scope with prg.
+
(** Generates an obligation to prove False. *)
Notation " ! " := (False_rect _ _) : program_scope.
-Delimit Scope program_scope with prg.
-
(** Abbreviation for first projection and hiding of proofs of subset objects. *)
Notation " ` t " := (proj1_sig t) (at level 10, t at next level) : program_scope.