Documentation

Std.Internal.Parsec.Basic

Instances For
    instance Std.Internal.Parsec.instReprParseResult {α✝ ι✝ : Type} [Repr α✝] [Repr ι✝] :
    Equations
    • Std.Internal.Parsec.instReprParseResult = { reprPrec := Std.Internal.Parsec.reprParseResult✝ }
    Equations
    Instances For
      class Std.Internal.Parsec.Input (ι : Type) (elem idx : outParam Type) [DecidableEq idx] [DecidableEq elem] :
      Instances
        Equations
        @[inline]
        def Std.Internal.Parsec.bind {ι α β : Type} (f : Std.Internal.Parsec ι α) (g : αStd.Internal.Parsec ι β) :
        Equations
        Instances For
          @[always_inline]
          Equations
          • Std.Internal.Parsec.instMonad = Monad.mk
          @[inline]
          def Std.Internal.Parsec.tryCatch {α ι elem idx : Type} [DecidableEq idx] [DecidableEq elem] [Std.Internal.Parsec.Input ι elem idx] {β : Type} (p : Std.Internal.Parsec ι α) (csuccess : αStd.Internal.Parsec ι β) (cerror : UnitStd.Internal.Parsec ι β) :
          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            @[inline]
            def Std.Internal.Parsec.orElse {α ι elem idx : Type} [DecidableEq idx] [DecidableEq elem] [Std.Internal.Parsec.Input ι elem idx] (p : Std.Internal.Parsec ι α) (q : UnitStd.Internal.Parsec ι α) :
            Equations
            • p.orElse q = p.tryCatch pure q
            Instances For
              @[inline]
              Equations
              • One or more equations did not get rendered due to their size.
              Instances For
                @[always_inline]
                Equations
                @[inline]
                Equations
                • One or more equations did not get rendered due to their size.
                Instances For
                  @[specialize #[]]
                  partial def Std.Internal.Parsec.manyCore {α ι elem idx : Type} [DecidableEq idx] [DecidableEq elem] [Std.Internal.Parsec.Input ι elem idx] (p : Std.Internal.Parsec ι α) (acc : Array α) :
                  @[inline]
                  Equations
                  • p.many = p.manyCore #[]
                  Instances For
                    @[inline]
                    Equations
                    • p.many1 = do let __do_liftp p.manyCore #[__do_lift]
                    Instances For
                      @[inline]
                      Equations
                      • One or more equations did not get rendered due to their size.
                      Instances For
                        @[inline]
                        def Std.Internal.Parsec.satisfy {ι elem idx : Type} [DecidableEq idx] [DecidableEq elem] [Std.Internal.Parsec.Input ι elem idx] (p : elemBool) :
                        Equations
                        Instances For
                          @[inline]
                          Equations
                          • One or more equations did not get rendered due to their size.
                          Instances For
                            @[inline]
                            Equations
                            • One or more equations did not get rendered due to their size.
                            Instances For
                              @[inline]
                              Equations
                              • One or more equations did not get rendered due to their size.
                              Instances For
                                @[inline]
                                def Std.Internal.Parsec.peekD {ι elem idx : Type} [DecidableEq idx] [DecidableEq elem] [Std.Internal.Parsec.Input ι elem idx] (default : elem) :
                                Equations
                                • One or more equations did not get rendered due to their size.
                                Instances For
                                  @[inline]
                                  Equations
                                  • One or more equations did not get rendered due to their size.
                                  Instances For
                                    @[specialize #[]]
                                    @[inline]
                                    Equations
                                    • p.manyChars = p.manyCharsCore ""
                                    Instances For
                                      @[inline]
                                      Equations
                                      • p.many1Chars = do let __do_liftp p.manyCharsCore __do_lift.toString
                                      Instances For