Library GeoCoq.Axioms.continuity_axioms

In this file, we introduce elementary continuity properties. These properties are different variant to assert that the intersection of line, segment and circles exists under some assumptions. Adding one of these properties as axiom to the Tarski_2D type class gives us a definition of ruler and compass geometry. The links between these properties are in file elementary_continuity_props.v
If there is a point P inside a circle, and Q outside then there is a point Z of the segment PQ which is on the circle.

Definition segment_circle := A B P Q,
  InCircle P A B
  OutCircle Q A B
   Z, Bet P Z Q OnCircle Z A B.

Given a line UV which contains a point inside the circle, there is a point of line UV which is on the circle.

Definition one_point_line_circle := A B U V P,
  Col U V P U V Bet A P B
   Z, Col U V Z OnCircle Z A B.

Given a line UV which contains a point P inside the circle, there are two points on line UV which belong to the circle and they are distinct if if P is strictly inside the circle.

Definition two_points_line_circle := A B U V P,
  Col U V P U V Bet A P B
   Z1 Z2, Col U V Z1 OnCircle Z1 A B
                Col U V Z2 OnCircle Z2 A B
                Bet Z1 P Z2 (P B Z1 Z2).

Given two circles (A,B) and (C,D), if there are two points of (C,D) one inside and one outside (A,B) then there is a point of intersection of the two circles.

Definition circle_circle := A B C D P Q,
  OnCircle P C D
  OnCircle Q C D
  InCircle P A B
  OutCircle Q A B
   Z, OnCircle Z A B OnCircle Z C D.

Given two circles (A,B) and (C,D), if there is a point of (A,B) which is inside (C,D) and vice-versa, then there is a point of intersection of the two circles.

Definition circle_circle_bis := A B C D P Q,
  OnCircle P C D
  InCircle P A B
  OnCircle Q A B
  InCircle Q C D
   Z, OnCircle Z A B OnCircle Z C D.

Given two circles (A,B) and (C,D), if there are two points of (C,D) one inside and one outside (A,B) then there are two points of intersection of the two circles. They are distinct if the inside and outside properties are strict.

Definition circle_circle_two := A B C D P Q,
  OnCircle P C D
  OnCircle Q C D
  InCircle P A B
  OutCircle Q A B
   Z1 Z2,
    OnCircle Z1 A B OnCircle Z1 C D
    OnCircle Z2 A B OnCircle Z2 C D
    (InCircleS P A B OutCircleS Q A B Z1Z2).


Nested A B describes the fact that the sequences A and B form the end points of nested non-degenerate segments

Definition Nested (A B:nat Tpoint Prop) :=
  ( n, An, A n An) ( n, Bn, B n Bn)
   n An Am Bm Bn,
    A n An A (S n) Am B (S n) Bm B n Bn Bet An Am Bm Bet Am Bm Bn Am Bm.

Definition cantor_s_axiom := A B, Nested A B
   X, n An Bn, A n An B n Bn Bet An X Bn.

Definition dedekind_s_axiom := (Xi Upsilon : Tpoint Prop),
  ( A, X Y, Xi X Upsilon Y Bet A X Y)
  ( B, X Y, Xi X Upsilon Y Bet X B Y).

First-order formula

Inductive FOF : Prop Prop :=
| eq_fof : A B:Tpoint, FOF (A = B)
| bet_fof : A B C, FOF (Bet A B C)
| cong_fof : A B C D, FOF (Cong A B C D)
| not_fof : P, FOF P FOF (¬ P)
| and_fof : P Q, FOF P FOF Q FOF (P Q)
| or_fof : P Q, FOF P FOF Q FOF (P Q)
| implies_fof : P Q, FOF P FOF Q FOF (P Q)
| forall_fof : P, ( (A:Tpoint), FOF (P A)) FOF ( A, P A)
| exists_fof : P, ( (A:Tpoint), FOF (P A)) FOF ( A, P A).

Definition first_order_dedekind := Xi Upsilon,
  ( X, FOF (Xi X)) ( Y, FOF (Upsilon Y))
  ( A, X Y, Xi X Upsilon Y Bet A X Y)
  ( B, X Y, Xi X Upsilon Y Bet X B Y).

Definition archimedes_axiom := A B C D, A B Reach A B C D.

Definition aristotle_s_axiom := P Q A B C,
  ¬ Col A B C Acute A B C
   X, Y, Out B A X Out B C Y Per B X Y Lt P Q X Y.

Definition greenberg_s_axiom := P Q R A B C,
  ¬ Col A B C
  Acute A B C Q R Per P Q R
   S, LtA P S Q A B C Out Q S R.

End Continuity_Defs.