Documentation

Aesop.Util.EqualUpToIds

  • allowAssignmentDiff : Bool

    Allow metavariables to be unassigned on one side of the comparison and assigned on the other. So when we compare two expressions and we encounter a metavariable ?x in one of them and a subexpression e in the other (at the same position), we consider ?x equal to e.

Instances For
    Instances For
      def Aesop.EqualUpToIdsM.run' {α : Type} (x : Aesop.EqualUpToIdsM α) (commonMCtx? : Option Lean.MetavarContext) (mctx₁ mctx₂ : Lean.MetavarContext) (allowAssignmentDiff : Bool) :
      Equations
      • One or more equations did not get rendered due to their size.
      Instances For
        def Aesop.EqualUpToIdsM.run {α : Type} (x : Aesop.EqualUpToIdsM α) (commonMCtx? : Option Lean.MetavarContext) (mctx₁ mctx₂ : Lean.MetavarContext) (allowAssignmentDiff : Bool) :
        Equations
        • x.run commonMCtx? mctx₁ mctx₂ allowAssignmentDiff = (fun (x : α × Aesop.EqualUpToIdsM.State) => x.fst) <$> x.run' commonMCtx? mctx₁ mctx₂ allowAssignmentDiff
        Instances For
          @[inline]
          Equations
          Instances For
            @[inline]
            Equations
            Instances For
              @[inline]
              Equations
              Instances For
                @[inline]
                Equations
                Instances For
                  @[specialize #[]]
                  Equations
                  • One or more equations did not get rendered due to their size.
                  Instances For
                    @[specialize #[]]
                    Equations
                    • One or more equations did not get rendered due to their size.
                    Instances For
                      Instances For
                        @[specialize #[]]
                        Instances For
                          @[implemented_by Aesop.EqualUpToIds.Unsafe.levelsEqualUpToIdsCore]
                          @[specialize #[]]
                          Instances For
                            @[specialize #[]]
                            Instances For
                              @[implemented_by Aesop.EqualUpToIds.Unsafe.exprsEqualUpToIdsCore₁]
                              @[implemented_by Aesop.EqualUpToIds.Unsafe.unassignedMVarsEqualUpToIdsCore]
                              @[specialize #[]]
                              Equations
                              • One or more equations did not get rendered due to their size.
                              Instances For
                                def Aesop.exprsEqualUpToIds (mctx₁ mctx₂ : Lean.MetavarContext) (lctx₁ lctx₂ : Lean.LocalContext) (localInstances₁ localInstances₂ : Lean.LocalInstances) (e₁ e₂ : Lean.Expr) (allowAssignmentDiff : Bool := false) :
                                Equations
                                • One or more equations did not get rendered due to their size.
                                Instances For
                                  def Aesop.exprsEqualUpToIds' (e₁ e₂ : Lean.Expr) (allowAssignmentDiff : Bool := false) :
                                  Equations
                                  • One or more equations did not get rendered due to their size.
                                  Instances For
                                    def Aesop.unassignedMVarsEqualUptoIds (commonMCtx? : Option Lean.MetavarContext) (mctx₁ mctx₂ : Lean.MetavarContext) (mvarId₁ mvarId₂ : Lean.MVarId) (allowAssignmentDiff : Bool := false) :
                                    Equations
                                    • One or more equations did not get rendered due to their size.
                                    Instances For
                                      def Aesop.unassignedMVarsEqualUptoIds' (commonMCtx? : Option Lean.MetavarContext) (mctx₁ mctx₂ : Lean.MetavarContext) (mvarId₁ mvarId₂ : Lean.MVarId) (allowAssignmentDiff : Bool := false) :
                                      Equations
                                      • One or more equations did not get rendered due to their size.
                                      Instances For
                                        def Aesop.tacticStatesEqualUpToIds (commonMCtx? : Option Lean.MetavarContext) (mctx₁ mctx₂ : Lean.MetavarContext) (goals₁ goals₂ : Array Lean.MVarId) (allowAssignmentDiff : Bool := false) :
                                        Equations
                                        • One or more equations did not get rendered due to their size.
                                        Instances For
                                          def Aesop.tacticStatesEqualUpToIds' (commonMCtx? : Option Lean.MetavarContext) (mctx₁ mctx₂ : Lean.MetavarContext) (goals₁ goals₂ : Array Lean.MVarId) (allowAssignmentDiff : Bool := false) :
                                          Equations
                                          • One or more equations did not get rendered due to their size.
                                          Instances For