Skip to content

Commit

Permalink
moved putnam_2003_b5 to commented_problems.v
Browse files Browse the repository at this point in the history
  • Loading branch information
leejasper851 committed Jul 17, 2024
1 parent 8d20f3f commit 8bd422d
Show file tree
Hide file tree
Showing 2 changed files with 26 additions and 25 deletions.
27 changes: 26 additions & 1 deletion coq/src/commented_problems.v
Original file line number Diff line number Diff line change
Expand Up @@ -76,4 +76,29 @@ Theorem putnam_2010_a5:
forall (a b: R -> R -> R),
cross_product a b = a.
Proof. Admitted.
End putnam_2010_a5. *)
End putnam_2010_a5. *)

(* Require Import Reals
GeoCoq.Main.Tarski_dev.Ch16_coordinates_with_functions
GeoCoq.Axioms.Definitions
GeoCoq.Main.Highschool.triangles.
Context `{T2D:Tarski_2D} `{TE:@Tarski_euclidean Tn TnEQD}.
Open Scope R.
Definition putnam_2003_b5_solution (pt_to_R : Tpoint -> (R * R)) (dist : Tpoint -> Tpoint -> R) (P Op : Tpoint) := sqrt 3 * (1 - (dist P Op) ^ 2 - 1).
Theorem putnam_2003_b5
(pt_to_R : Tpoint -> (R * R))
(F_to_R : F -> R)
(dist : Tpoint -> Tpoint -> R := fun A B => let (a, b) := pt_to_R A in let (c, d) := pt_to_R B in dist_euc a b c d)
(Triangle : Tpoint -> Tpoint -> Tpoint -> Prop := fun x y z => ~ Col x y z) (* copied from GeoCoq.Axioms.euclidean_axioms *)
(A B C Op Op' P: Tpoint)
(fixpoint : dist Op Op' = R1)
(hABC : OnCircle A Op Op' /\ OnCircle B Op Op' /\ OnCircle C Op Op')
(hABC' : Main.Highschool.triangles.equilateral A B C)
(hp : InCircle P Op Op')
(a : R := dist P A)
(b : R := dist P B)
(c : R := dist P C)
: exists (A' B' C' : Tpoint) (D: Cs O E A' B' C'),
Triangle A' B' C' /\ dist A' B' = a /\ dist B' C' = b /\ dist C' A' = c /\
F_to_R (signed_area A' B' C' D A' B' C') = (putnam_2003_b5_solution pt_to_R dist P Op).
Proof. Admitted. *)
24 changes: 0 additions & 24 deletions coq/src/putnam_2003_b5.v

This file was deleted.

0 comments on commit 8bd422d

Please sign in to comment.