Documentation

Lean.Meta.Tactic.SplitIf

Instances For
    Equations
    Instances For
      Equations
      Instances For
        Instances For
          @[inline]
          Equations
          • One or more equations did not get rendered due to their size.
          Instances For
            Equations
            • One or more equations did not get rendered due to their size.
            Instances For
              def Lean.Meta.findSplit? (e : Expr) (kind : SplitKind := SplitKind.both) (exceptionSet : ExprSet := ) :

              Return an if-then-else or match-expr to split.

              Equations
              Instances For
                partial def Lean.Meta.findSplit?.go (kind : SplitKind := SplitKind.both) (exceptionSet : ExprSet := ) (e : Expr) :
                def Lean.Meta.findSplit?.find? (kind : SplitKind := SplitKind.both) (exceptionSet : ExprSet := ) (e : Expr) :
                Equations
                • One or more equations did not get rendered due to their size.
                Instances For

                  Default Simp.Context for simpIf methods. It contains all congruence theorems, but just the rewriting rules for reducing if expressions.

                  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
                        def Lean.Meta.simpIfTarget (mvarId : MVarId) (useDecide : Bool := false) :
                        Equations
                        • One or more equations did not get rendered due to their size.
                        Instances For
                          Equations
                          • One or more equations did not get rendered due to their size.
                          Instances For
                            Equations
                            • One or more equations did not get rendered due to their size.
                            Instances For
                              def Lean.Meta.splitIfLocalDecl? (mvarId : MVarId) (fvarId : FVarId) (hName? : Option Name := none) :
                              Equations
                              • One or more equations did not get rendered due to their size.
                              Instances For