aboutsummaryrefslogtreecommitdiff
path: root/mathcomp/ssrtest/caseview.v
diff options
context:
space:
mode:
authorEnrico Tassi2015-03-09 11:07:53 +0100
committerEnrico Tassi2015-03-09 11:24:38 +0100
commitfc84c27eac260dffd8f2fb1cb56d599f1e3486d9 (patch)
treec16205f1637c80833a4c4598993c29fa0fd8c373 /mathcomp/ssrtest/caseview.v
Initial commit
Diffstat (limited to 'mathcomp/ssrtest/caseview.v')
-rw-r--r--mathcomp/ssrtest/caseview.v4
1 files changed, 4 insertions, 0 deletions
diff --git a/mathcomp/ssrtest/caseview.v b/mathcomp/ssrtest/caseview.v
new file mode 100644
index 0000000..108cf46
--- /dev/null
+++ b/mathcomp/ssrtest/caseview.v
@@ -0,0 +1,4 @@
+Require Import ssreflect.
+
+Lemma test (A B : Prop) : A /\ B -> True.
+Proof. by case=> _ /id _. Qed. \ No newline at end of file