Skip to content

Commit

Permalink
minor update
Browse files Browse the repository at this point in the history
  • Loading branch information
PratherConid committed Dec 27, 2024
1 parent ed277c2 commit d428dfa
Show file tree
Hide file tree
Showing 2 changed files with 15 additions and 2 deletions.
4 changes: 2 additions & 2 deletions Auto/Translation/Monomorphization.lean
Original file line number Diff line number Diff line change
Expand Up @@ -41,7 +41,7 @@ register_option auto.mono.ciInstDefEq.mode : Meta.TransparencyMode := {
}

register_option auto.mono.ciInstDefEq.maxHeartbeats : Nat := {
defValue := 1024
defValue := 2048
descr := "Heartbeats allocated to each unification of constant instance"
}

Expand All @@ -52,7 +52,7 @@ register_option auto.mono.termLikeDefEq.mode : Meta.TransparencyMode := {
}

register_option auto.mono.termLikeDefEq.maxHeartbeats : Nat := {
defValue := 1024
defValue := 2048
descr := "Heartbeats allocated to each unification of term-like expression"
}

Expand Down
13 changes: 13 additions & 0 deletions Test/Test_Regression.lean
Original file line number Diff line number Diff line change
Expand Up @@ -277,6 +277,9 @@ end UnfoldConst

section ConstInstDefEq

-- Effectively disable `termLikeDefEq`
set_option auto.mono.termLikeDefEq.mode "reducible"

def Nat.add₁ := Nat.add

example : Nat.add₁ = Nat.add := by
Expand Down Expand Up @@ -312,6 +315,16 @@ section ConstInstDefEq

end ConstInstDefEq

-- Definitional Equality from Term-like expressions

section TermLikeDefEq

set_option auto.tptp false
example (h : List.append [1, 2] [3, 4] = [2, 3]) : [1, 2, 3, 4] = [2, 3] := by
auto

end TermLikeDefEq

-- First Order

example : True := by
Expand Down

0 comments on commit d428dfa

Please sign in to comment.