aboutsummaryrefslogtreecommitdiffstats
path: root/src/Misc.v
diff options
context:
space:
mode:
Diffstat (limited to 'src/Misc.v')
-rw-r--r--src/Misc.v2
1 files changed, 2 insertions, 0 deletions
diff --git a/src/Misc.v b/src/Misc.v
index b3a0fc4..5ea1d14 100644
--- a/src/Misc.v
+++ b/src/Misc.v
@@ -14,6 +14,8 @@ Require Import Bool List PArray Int63 Ring63 ZArith Psatz.
Local Open Scope int63_scope.
Local Open Scope array_scope.
+Global Notation "[| x |]" := (φ x).
+
(** Lemmas about Bool *)