Created
September 24, 2016 03:29
-
-
Save mukeshtiwari/1927382c67de68d55776c5883d95ef5a to your computer and use it in GitHub Desktop.
This file contains hidden or bidirectional Unicode text that may be interpreted or compiled differently than what appears below. To review, open the file in an editor that reveals hidden Unicode characters.
Learn more about bidirectional Unicode characters
| Theorem path_lfp : forall (c d : cand) (k : nat), | |
| Fixpoints.least_fixed_point | |
| (cand * cand) (all_pairs cand_all) | |
| (all_pairs_universal cand_all cand_fin) (O k) (monotone_operator k) (c, d) = true | |
| <-> Path k c d. | |
| Proof. | |
| split. intros H. apply wins_evi. exists (length (all_pairs cand_all)). assumption. | |
| intros H. apply wins_evi in H. destruct H as [n H]. unfold Fixpoints.least_fixed_point. | |
| unfold Fixpoints.empty_ss. remember (length (all_pairs cand_all)) as v. | |
| specialize (Fixpoints.iter_fin v (O k) (monotone_operator k)). intros. | |
| unfold Fixpoints.bounded_card in H0. | |
| assert (Ht : (exists l : list (cand * cand), (forall a : cand * cand, In a l) /\ length l <= v)). | |
| { | |
| exists (all_pairs cand_all). split. apply (all_pairs_universal cand_all cand_fin). | |
| omega. | |
| } | |
| specialize (H0 Ht n). unfold Fixpoints.pred_subset in H0. | |
| apply H0. assumption. | |
| Qed. | |
| c, d : cand | |
| k : nat | |
| H : ~ Path k c d | |
| ============================ | |
| Fixpoints.greatest_fixed_point (cand * cand) (all_pairs cand_all) | |
| (all_pairs_universal cand_all cand_fin) (W k) (monotone_operator_w k) | |
| (c, d) = true | |
| I am trying to apply apply path_lfp in H to get ~ (Fixpoints.least_fixed_point | |
| (cand * cand) (all_pairs cand_all) | |
| (all_pairs_universal cand_all cand_fin) (O k) (monotone_operator k) (c, d) = true ) in the context but getting error | |
| "Statement without assumption". |
Author
Sign up for free
to join this conversation on GitHub.
Already have an account?
Sign in to comment
Full source code https://github.com/mukeshtiwari/formalized-voting/blob/master/Schulze_Dirk.v