- decl: Lean.Name → Lean.Meta.Origin
A global declaration in the environment.
- fvar: Lean.FVarId → Lean.Meta.Origin
A local hypothesis. When
contextual := trueis enabled, this fvar may exist in an extension of the current local context; it will not be used for rewriting by simp once it is out of scope but it may end up in theusedSimpstrace. - stx: Lean.Name → Lean.Syntax → Lean.Meta.Origin
A proof term provided directly to a call to
simp [ref, ...]whererefis the provided simp argument (of kindParser.Tactic.simpLemma). Theidis a unique identifier for the call. - other: Lean.Name → Lean.Meta.Origin
Some other origin.
nameshould not collide with the other types for erasure to work correctly, and simp trace will ignore this lemma. The other origins should be preferred if possible.
An Origin is an identifier for simp theorems which indicates roughly
what action the user took which lead to this theorem existing in the simp set.
Instances For
Equations
- Lean.Meta.instInhabitedOrigin = { default := Lean.Meta.Origin.decl default }
Equations
- Lean.Meta.instReprOrigin = { reprPrec := Lean.Meta.reprOrigin✝ }
A unique identifier corresponding to the origin.
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Meta.instBEqOrigin = { beq := fun a a_1 => Lean.Meta.Origin.key a == Lean.Meta.Origin.key a_1 }
Equations
- Lean.Meta.instHashableOrigin = { hash := fun a => hash (Lean.Meta.Origin.key a) }
- keys : Array Lean.Meta.DiscrTree.Key
It stores universe parameter names for universe polymorphic proofs. Recall that it is non-empty only when we elaborate an expression provided by the user. When
proofis just a constant, we can use the universe parameter names stored in the declaration.- proof : Lean.Expr
- priority : Nat
- post : Bool
permis true if lhs and rhs are identical modulo permutation of variables.perm : Booloriginis mainly relevant for producing trace messages. It is also viewed anidused to "erase"simptheorems fromSimpTheorems.origin : Lean.Meta.Origin- rfl : Bool
The fields levelParams and proof are used to encode the proof of the simp theorem.
If the proof is a global declaration c, we store Expr.const c [] at proof without the universe levels, and levelParams is set to #[]
When using the lemma, we create fresh universe metavariables.
Motivation: most simp theorems are global declarations, and this approach is faster and saves memory.
The field levelParams is not empty only when we elaborate an expression provided by the user, and it contains universe metavariables.
Then, we use abstractMVars to abstract the universe metavariables and create new fresh universe parameters that are stored at the field levelParams.
Instances For
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Meta.instBEqSimpTheorem = { beq := fun e₁ e₂ => e₁.proof == e₂.proof }
- lemmaNames : Lean.PHashSet Lean.Meta.Origin
- toUnfold : Lean.PHashSet Lean.Name
- erased : Lean.PHashSet Lean.Meta.Origin
- toUnfoldThms : Lean.PHashMap Lean.Name (Array Lean.Name)
Instances For
Equations
- Lean.Meta.instInhabitedSimpTheorems = { default := { pre := default, post := default, lemmaNames := default, toUnfold := default, erased := default, toUnfoldThms := default } }
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Return true if declName is tagged to be unfolded using unfoldDefinition? (i.e., without using equational theorems).
Equations
- Lean.Meta.SimpTheorems.isDeclToUnfold d declName = Lean.PersistentHashSet.contains d.toUnfold declName
Equations
- Lean.Meta.SimpTheorems.isLemma d thmId = Lean.PersistentHashSet.contains d.lemmaNames thmId
Register the equational theorems for the given definition.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
- thm: Lean.Meta.SimpTheorem → Lean.Meta.SimpEntry
- toUnfold: Lean.Name → Lean.Meta.SimpEntry
- toUnfoldThms: Lean.Name → Array Lean.Name → Lean.Meta.SimpEntry
Instances For
Equations
- Lean.Meta.instInhabitedSimpEntry = { default := Lean.Meta.SimpEntry.thm default }
Equations
- Lean.Meta.SimpExtension.getTheorems ext = do let a ← Lean.getEnv pure (Lean.ScopedEnvExtension.getState ext a)
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Meta.getSimpExtension? attrName = do let a ← ST.Ref.get Lean.Meta.simpExtensionMapRef pure (Lean.HashMap.find? a attrName)
Auxiliary method for adding a global declaration to a SimpTheorems datastructure.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Auxiliary method for creating simp theorems from a proof term val.
Equations
- One or more equations did not get rendered due to their size.
Auxiliary method for adding a local simp theorem to a SimpTheorems datastructure.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- One or more equations did not get rendered due to their size.
Equations
- Lean.Meta.SimpTheoremsArray.eraseTheorem thmsArray thmId = Array.map (fun thms => Lean.Meta.SimpTheorems.eraseCore thms thmId) thmsArray
Equations
- Lean.Meta.SimpTheoremsArray.isErased thmsArray thmId = Array.any thmsArray (fun thms => Lean.PersistentHashSet.contains thms.erased thmId) 0 (Array.size thmsArray)
Equations
- Lean.Meta.SimpTheoremsArray.isDeclToUnfold thmsArray declName = Array.any thmsArray (fun thms => Lean.Meta.SimpTheorems.isDeclToUnfold thms declName) 0 (Array.size thmsArray)
Equations
- One or more equations did not get rendered due to their size.