Documentation

Lean.Meta.WHNF

Smart unfolding support #

@[extern lean_get_structural_rec_arg_pos]

Forward declaration. It is defined in the module src/Lean/Elab/PreDefinition/Structural/Eqns.lean. It is possible to avoid this hack if we move Structural.EqnInfo and Structural.eqnInfoExt to this module.

@[inline]
Equations
Instances For
    Equations
    Instances For

      Add auxiliary annotation to indicate the match-expression e must be reduced when performing smart unfolding.

      Equations
      Instances For

        Add auxiliary annotation to indicate expression e (a match alternative rhs) was successfully reduced by smart unfolding.

        Equations
        Instances For

          Helper methods #

          def Lean.Meta.isAuxDef (constName : Name) :
          Equations
          Instances For

            Helper functions for reducing recursors #

            def Lean.Meta.mkProjFn (ctorVal : ConstructorVal) (us : List Level) (params : Array Expr) (i : Nat) (major : Expr) :

            Create the ith projection major. It tries to use the auto-generated projection functions if available. Otherwise falls back to Expr.proj.

            Equations
            • One or more equations did not get rendered due to their size.
            Instances For

              Helper functions for reducing Quot.lift and Quot.ind #

              Helper function for extracting "stuck term" #

              Return some (Expr.mvar mvarId) if metavariable mvarId is blocking reduction.

              Weak Head Normal Form auxiliary combinators #

              @[specialize #[]]
              partial def Lean.Meta.whnfEasyCases (e : Expr) (k : ExprMetaM Expr) :

              Auxiliary combinator for handling easy WHNF cases. It takes a function for handling the "hard" cases as an argument

              Instances For

                The "match" compiler uses dependent if-then-else dite and other auxiliary declarations to compile match-expressions such as

                match v with
                | 'a' => 1
                | 'b' => 2
                | _   => 3
                

                because it is more efficient than using casesOn recursors. The method reduceMatcher? fails if these auxiliary definitions cannot be unfolded in the current transparency setting. This is problematic because tactics such as simp use TransparencyMode.reducible, and most users assume that expressions such as

                match 0 with
                | 0 => 1
                | 100 => 2
                | _ => 3
                

                should reduce in any transparency mode.

                Thus, if the transparency mode is .reducible or .instances, we first eagerly unfold dite constants used in the auxiliary match-declaration, and then use a custom canUnfoldAtMatcher predicate for whnfMatcher.

                Remark: we used to include dite (and ite) as auxiliary declarations to unfold at canUnfoldAtMatcher, but this is problematic because the dite/ite may occur in the discriminant. See issue #5388.

                This solution is not very modular because modifications at the match compiler require changes here. We claim this is defensible because it is reducing the auxiliary declaration defined by the match compiler.

                Remark: if the eager unfolding is problematic, we may cache the result. We may also consider not using dite in the match-compiler and use Decidable.casesOn, but it will require changes in how we generate equation lemmas.

                Alternative solution: tactics that use TransparencyMode.reducible should rely on the equations we generated for match-expressions. This solution is also not perfect because the match-expression above will not reduce during type checking when we are not using TransparencyMode.default or TransparencyMode.all.

                Auxiliary predicate for whnfMatcher. See comment above.

                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
                      Equations
                      Instances For

                        Reduce kernel projection Expr.proj .. expression.

                        Equations
                        Instances For

                          Apply beta-reduction, zeta-reduction (i.e., unfold let local-decls), iota-reduction, expand let-expressions, expand assigned meta-variables.

                          Equations
                          Instances For

                            Recall that _sunfold auxiliary definitions contains the markers: markSmartUnfoldingMatch (*) and markSmartUnfoldingMatchAlt (**). For example, consider the following definition

                            def r (i j : Nat) : Nat :=
                              i +
                                match j with
                                | Nat.zero => 1
                                | Nat.succ j =>
                                  i + match j with
                                      | Nat.zero => 2
                                      | Nat.succ j => r i j
                            

                            produces the following _sunfold auxiliary definition with the markers

                            def r._sunfold (i j : Nat) : Nat :=
                              i +
                                (*) match j with
                                | Nat.zero => (**) 1
                                | Nat.succ j =>
                                  i + (*) match j with
                                      | Nat.zero => (**) 2
                                      | Nat.succ j => (**) r i j
                            

                            match expressions marked with markSmartUnfoldingMatch (*) must be reduced, otherwise the resulting term is not definitionally equal to the given expression. The recursion may be interrupted as soon as the annotation markSmartUnfoldingAlt (**) is reached.

                            For example, the term r i j.succ.succ reduces to the definitionally equal term i + i * r i j

                            Equations
                            Instances For

                              Auxiliary method for unfolding a class projection.

                              Auxiliary method for unfolding a class projection when transparency is set to TransparencyMode.instances. Recall that class instance projections are not marked with [reducible] because we want them to be in "reducible canonical form".

                              partial def Lean.Meta.unfoldDefinition? (e : Expr) (ignoreTransparency : Bool := false) :

                              Unfold definition using "smart unfolding" if possible. If ignoreTransparency = true, then the definition is unfolded even if the transparency setting does not allow it.

                              Equations
                              • One or more equations did not get rendered due to their size.
                              Instances For
                                @[specialize #[]]
                                partial def Lean.Meta.whnfHeadPred (e : Expr) (pred : ExprMetaM Bool) :
                                def Lean.Meta.whnfUntil (e : Expr) (declName : Name) :
                                Equations
                                Instances For

                                  Try to reduce matcher/recursor/quot applications. We say they are all "morally" recursor applications.

                                  Equations
                                  • One or more equations did not get rendered due to their size.
                                  Instances For
                                    Equations
                                    Instances For
                                      unsafe def Lean.Meta.reduceNatNativeUnsafe (constName : Name) :
                                      Equations
                                      Instances For
                                        @[implemented_by Lean.Meta.reduceBoolNativeUnsafe]
                                        @[implemented_by Lean.Meta.reduceNatNativeUnsafe]
                                        opaque Lean.Meta.reduceNatNative (constName : Name) :
                                        Equations
                                        Instances For
                                          @[inline]
                                          def Lean.Meta.withNatValue {α : Type} (a : Expr) (k : NatMetaM (Option α)) :
                                          Equations
                                          • One or more equations did not get rendered due to their size.
                                          Instances For
                                            def Lean.Meta.reduceBinNatOp (f : NatNatNat) (a b : Expr) :
                                            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
                                                Instances For
                                                  Instances For
                                                    @[export lean_whnf]
                                                    partial def Lean.Meta.whnfImp (e : Expr) :

                                                    If e is a projection function that satisfies p, then reduce it

                                                    Equations
                                                    • One or more equations did not get rendered due to their size.
                                                    Instances For