Skip to content

Instantly share code, notes, and snippets.

View yoshihiro503's full-sized avatar

YOSHIHIRO Imai yoshihiro503

View GitHub Profile

cometbft/cometbft から派生した 0xPolygon/cometbft リポジトリを見ているが、どのタイミングで分岐したか知りたい

分岐点のコミットを探す

git clone https://github.com/0xPolygon/cometbft.git cometbft-polygonfork
cd cometbft-polygonfork/
git remote add upstream https://github.com/cometbft/cometbft.git
git fetch upstream

Alt text

#CUT
digraph G {
    aize ="4,4";
    subgraph cluster_public {
        label="Public";
        Start [shape=box];
        RegisterTasks [shape=box, layer=cluster_public];
        Stop [shape=box];

mathcomp analysisのtopology.vにおいて,

...
Module PropInFilter : PropInFilterSig.
  Definition t := prop_in_filter_proj.
  ...
End PropInFilter.
Notation prop_of := PropInFilter.t.
...
From mathcomp Require Import all_ssreflect.
Require Import JMeq.
Inductive sizseq (T:Type) : nat -> Type :=
| SizNil : sizseq T 0
| SizCons n : T -> sizseq T n -> sizseq T n.+1.
Lemma sizseq0nil_aux (T:Type) n : forall xs : sizseq T n, n = 0 -> JMeq xs (SizNil T).
Proof.
From mathcomp Require Import all_ssreflect.
Set Implicit Arguments.
Unset Strict Implicit.
Unset Printing Implicit Defensive.
(* :> を複数持つと予期せぬことがおきることがあるぞ *)
Structure S : Type := MakeS {
sort2 :> Type;
sort :> Type;
From mathcomp Require Import all_ssreflect.
Fixpoint evivn_rec pred_d m q :=
if m - pred_d is m'.+1 then edivn_rec pred_d m' q.+1 else (q, m).
Definition edivn m d := if d > 0 then edivn_rec d.-1 m 0 else (0, m).
Lemma edivn_recP1 q r m pred_d q0:
(q, r) = edivn_rec pred_d m q0 ->
r < pred_d.+1.
Require Import String List.
Import ListNotations.
Open Scope string_scope.
Definition aaa := 1+2.
Definition bbb := aaa * 5.
Definition foo x y:= 2*x + y.
Compute foo 1 2.
Require Import Arith Unicode.Utf8.
Definition f (n : nat) :=
n - 1.
Inductive reaches_1 : nat → Prop :=
| term_done : reaches_1 1
| term_more (n : nat) : reaches_1 (f n) → reaches_1 n.
Check reaches_1_ind.