aboutsummaryrefslogtreecommitdiff
path: root/src/Util/CaseUtil.v
diff options
context:
space:
mode:
authorGravatar Andres Erbsen <andreser@mit.edu>2017-04-06 15:47:12 -0400
committerGravatar Andres Erbsen <andreser@mit.edu>2017-04-06 15:47:12 -0400
commitf8cc64c7ca411828cac5cad2958959b0d779d683 (patch)
tree1c74a6bf6bc92522db7451e3c0dd748c57a2ece3 /src/Util/CaseUtil.v
parent33b1e92e1a71f284461e0c8d1d22b1d28b29bd7a (diff)
start removing BaseSystem
Diffstat (limited to 'src/Util/CaseUtil.v')
-rw-r--r--src/Util/CaseUtil.v18
1 files changed, 0 insertions, 18 deletions
diff --git a/src/Util/CaseUtil.v b/src/Util/CaseUtil.v
deleted file mode 100644
index 2d1ab6c58..000000000
--- a/src/Util/CaseUtil.v
+++ /dev/null
@@ -1,18 +0,0 @@
-Require Import Coq.Arith.Arith Coq.Arith.Max.
-
-Ltac case_max :=
- match goal with [ |- context[max ?x ?y] ] =>
- destruct (le_dec x y);
- match goal with
- | [ H : (?x <= ?y)%nat |- context[max ?x ?y] ] => rewrite max_r by
- (exact H)
- | [ H : ~ (?x <= ?y)%nat |- context[max ?x ?y] ] => rewrite max_l by
- (exact (le_Sn_le _ _ (not_le _ _ H)))
- end
- end.
-
-Lemma pull_app_if_sumbool {A B X Y} (b : sumbool X Y) (f g : A -> B) (x : A)
- : (if b then f x else g x) = (if b then f else g) x.
-Proof.
- destruct b; reflexivity.
-Qed.