-
Notifications
You must be signed in to change notification settings - Fork 1
/
Copy pathexamples_4.v
38 lines (33 loc) · 1.08 KB
/
examples_4.v
1
2
3
4
5
6
7
8
9
10
11
12
13
14
15
16
17
18
19
20
21
22
23
24
25
26
27
28
29
30
31
32
33
34
35
36
37
38
(***************************************************************************)
(* Formalization of the Chou, Gao and Zhang's decision procedure. *)
(* Julien Narboux (Julien@narboux.fr) *)
(* LIX/INRIA FUTURS 2004-2006 *)
(* University of Strasbourg 2008 *)
(***************************************************************************)
Require Import area_method.
(** The Pappus line theorem *)
Theorem Pappus : forall A B C A' B' C' P Q R :Point,
on_line C A B ->
on_line C' A' B' ->
inter_ll P A' B A B' ->
inter_ll Q A C' A' C ->
inter_ll R B' C B C' ->
Col P Q R.
Proof.
area_method.
Qed.
(** This version uses an extra point *)
Theorem Pappus_2 : forall A B C A' B' C' P Q R T:Point,
on_line C A B ->
on_line C' A' B' ->
inter_ll P A' B A B' ->
inter_ll Q A C' A' C ->
inter_ll R B' C B C' ->
inter_ll T B' C P Q ->
C<>R -> C<>T ->
parallel B' R C R ->
parallel B' T C T ->
B'**R / C**R = B'**T / C**T.
Proof.
area_method.
Qed.