Documentation

Lean.Compiler.LCNF.AlphaEqv

Alpha equivalence for LCNF Code

Equations
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
        @[inline]
        def Lean.Compiler.LCNF.AlphaEqv.withFVar {α : Type} (fvarId₁ fvarId₂ : FVarId) (x : EqvM α) :
        EqvM α
        Equations
        Instances For
          @[inline]
          Equations
          Instances For
            @[irreducible, specialize #[]]
            def Lean.Compiler.LCNF.AlphaEqv.withParams.go (params₁ params₂ : Array Param) (x : EqvM Bool) (h : params₂.size = params₁.size) (i : Nat) :
            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
                partial def Lean.Compiler.LCNF.AlphaEqv.eqv (code₁ code₂ : Code) :

                Return true if c₁ and c₂ are alpha equivalent.

                Equations
                Instances For