aboutsummaryrefslogtreecommitdiffhomepage
path: root/coq/example.v
diff options
context:
space:
mode:
Diffstat (limited to 'coq/example.v')
-rw-r--r--coq/example.v16
1 files changed, 8 insertions, 8 deletions
diff --git a/coq/example.v b/coq/example.v
index 5c6894c7..27ccd26d 100644
--- a/coq/example.v
+++ b/coq/example.v
@@ -6,13 +6,13 @@
Module Example.
-Goal forall (A B:Prop),(A /\ B) -> (B /\ A).
- intros A B.
- intros H.
- elim H.
- split.
- assumption.
- assumption.
-Save and_comms.
+ Lemma and_commutative : forall (A B:Prop),(A /\ B) -> (B /\ A).
+ Proof.
+ intros A B H.
+ destruct H.
+ split.
+ trivial.
+ trivial.
+ Qed.
End Example.