Skip to content

Commit

Permalink
feat: add Simp.Config.implicitDefEqProofs
Browse files Browse the repository at this point in the history
This commit does **not** implement this feature.
  • Loading branch information
leodemoura committed Jun 29, 2024
1 parent d4d7c72 commit fb97275
Showing 1 changed file with 8 additions and 0 deletions.
8 changes: 8 additions & 0 deletions src/Init/MetaTypes.lean
Original file line number Diff line number Diff line change
Expand Up @@ -218,6 +218,14 @@ structure Config where
to find candidate `simp` theorems. It approximates Lean 3 `simp` behavior.
-/
index : Bool := true
/--
When `true` (default: `false`), `simp` will **not** create a proof for a rewriting rule associated
with an `rfl`-theorem.
Rewriting rules are provided by users by annotating theorems with the attribute `@[simp]`.
If the proof of the theorem is just `rfl` (reflexivity), and `implicitDefEqProofs := true`, `simp`
will **not** create a proof term which is an application of the annotated theorem.
-/
implicitDefEqProofs : Bool := false
deriving Inhabited, BEq

-- Configuration object for `simp_all`
Expand Down

0 comments on commit fb97275

Please sign in to comment.