Skip to content

Commit

Permalink
Enable dynamic structuring by default
Browse files Browse the repository at this point in the history
  • Loading branch information
JLimperg committed Aug 7, 2024
1 parent 8ff1f48 commit 0444234
Show file tree
Hide file tree
Showing 2 changed files with 3 additions and 3 deletions.
2 changes: 1 addition & 1 deletion Aesop/Options/Public.lean
Original file line number Diff line number Diff line change
Expand Up @@ -162,7 +162,7 @@ structure Options where
-/
register_option aesop.dev.dynamicStructuring : Bool := {
descr := "(aesop) Only for use by Aesop developers. Enables dynamic script structuring."
defValue := false
defValue := true
}

end Aesop
4 changes: 2 additions & 2 deletions AesopTest/RulePattern.lean
Original file line number Diff line number Diff line change
Expand Up @@ -44,8 +44,8 @@ axiom triangle (a b : Int) : |a + b| ≤ |a| + |b|

example : |a + b| ≤ |c + d| := by
aesop!
guard_hyp fwd_1 : |c + d| ≤ |c| + |d|
guard_hyp fwd : |a + b| ≤ |a| + |b|
guard_hyp fwd : |c + d| ≤ |c| + |d|
guard_hyp fwd_1 : |a + b| ≤ |a| + |b|
falso

@[aesop safe apply (pattern := (0 : Nat))]
Expand Down

0 comments on commit 0444234

Please sign in to comment.