Documentation

Lake.Util.Date

Date #

A year-mont-day date. Used by Lake's TOML parser and its toolchain version parser (for nightlies).

def Lake.lpad (s : String) (c : Char) (len : Nat) :
Equations
Instances For
    def Lake.rpad (s : String) (c : Char) (len : Nat) :
    Equations
    Instances For
      def Lake.zpad (n len : Nat) :
      Equations
      Instances For
        structure Lake.Date :

        A date (year-month-day).

        Instances For
          def Lake.instDecidableEqDate.decEq (x✝ x✝¹ : Date) :
          Decidable (x✝ = x✝¹)
          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            Equations
            Instances For
              Equations
              • One or more equations did not get rendered due to their size.
              Instances For
                @[reducible, inline]
                Equations
                Instances For
                  @[reducible, inline]
                  Equations
                  Instances For
                    def Lake.Date.maxDay (y m : Nat) :
                    Equations
                    Instances For
                      @[reducible, inline]
                      abbrev Lake.Date.IsValidDay (y m d : Nat) :
                      Equations
                      Instances For
                        def Lake.Date.ofValid? (year month day : Nat) :
                        Equations
                        Instances For
                          Equations
                          • One or more equations did not get rendered due to their size.
                          Instances For