diff options
Diffstat (limited to 'backends/lean/Base/Arith/Scalar.lean')
| -rw-r--r-- | backends/lean/Base/Arith/Scalar.lean | 47 | 
1 files changed, 23 insertions, 24 deletions
| diff --git a/backends/lean/Base/Arith/Scalar.lean b/backends/lean/Base/Arith/Scalar.lean index 86b2e216..c2e4e24e 100644 --- a/backends/lean/Base/Arith/Scalar.lean +++ b/backends/lean/Base/Arith/Scalar.lean @@ -8,30 +8,29 @@ open Lean Lean.Elab Lean.Meta  open Primitives  def scalarTacExtraPreprocess : Tactic.TacticM Unit := do -   Tactic.withMainContext do -   -- Inroduce the bounds for the isize/usize types -   let add (e : Expr) : Tactic.TacticM Unit := do -     let ty ← inferType e -     let _ ← Utils.addDeclTac (← Utils.mkFreshAnonPropUserName) e ty (asLet := false) -   add (← mkAppM ``Scalar.cMin_bound #[.const ``ScalarTy.Isize []]) -   add (← mkAppM ``Scalar.cMax_bound #[.const ``ScalarTy.Usize []]) -   add (← mkAppM ``Scalar.cMax_bound #[.const ``ScalarTy.Isize []]) -   -- Reveal the concrete bounds, simplify calls to [ofInt] -   Utils.simpAt true -                -- Unfoldings -                [``Scalar.min, ``Scalar.max, ``Scalar.cMin, ``Scalar.cMax, -                 ``I8.min, ``I16.min, ``I32.min, ``I64.min, ``I128.min, -                 ``I8.max, ``I16.max, ``I32.max, ``I64.max, ``I128.max, -                 ``U8.min, ``U16.min, ``U32.min, ``U64.min, ``U128.min, -                 ``U8.max, ``U16.max, ``U32.max, ``U64.max, ``U128.max, -                 ``Usize.min -                 ] -                 -- Simp lemmas -                 [``Scalar.ofInt_val_eq, ``Scalar.neq_to_neq_val, -                  ``Scalar.lt_equiv, ``Scalar.le_equiv, ``Scalar.eq_equiv] -                 -- Hypotheses -                 [] .wildcard -    +  Tactic.withMainContext do +  -- Inroduce the bounds for the isize/usize types +  let add (e : Expr) : Tactic.TacticM Unit := do +    let ty ← inferType e +    let _ ← Utils.addDeclTac (← Utils.mkFreshAnonPropUserName) e ty (asLet := false) +  add (← mkAppM ``Scalar.cMin_bound #[.const ``ScalarTy.Isize []]) +  add (← mkAppM ``Scalar.cMax_bound #[.const ``ScalarTy.Usize []]) +  add (← mkAppM ``Scalar.cMax_bound #[.const ``ScalarTy.Isize []]) +  -- Reveal the concrete bounds, simplify calls to [ofInt] +  Utils.simpAt true {} +               -- Unfoldings +               [``Scalar.min, ``Scalar.max, ``Scalar.cMin, ``Scalar.cMax, +                ``I8.min, ``I16.min, ``I32.min, ``I64.min, ``I128.min, +                ``I8.max, ``I16.max, ``I32.max, ``I64.max, ``I128.max, +                ``U8.min, ``U16.min, ``U32.min, ``U64.min, ``U128.min, +                ``U8.max, ``U16.max, ``U32.max, ``U64.max, ``U128.max, +                ``Usize.min +                ] +                -- Simp lemmas +                [``Scalar.ofInt_val_eq, ``Scalar.neq_to_neq_val, +                 ``Scalar.lt_equiv, ``Scalar.le_equiv, ``Scalar.eq_equiv] +                -- Hypotheses +                [] .wildcard  elab "scalar_tac_preprocess" : tactic =>    intTacPreprocess scalarTacExtraPreprocess | 
